refactor: TensorStruct to TensorSpeciesStruct

This commit is contained in:
jstoobysmith 2024-10-21 11:53:22 +00:00
parent a44a538d85
commit b92796cb2f
9 changed files with 24 additions and 24 deletions

View file

@ -8,7 +8,7 @@ import HepLean.Tensors.Tree.Basic
# The commutativity of Permutations and contractions.
There is very likely a better way to do this using `TensorStruct.contrMap_tprod`.
There is very likely a better way to do this using `TensorSpeciesStruct.contrMap_tprod`.
-/
@ -18,10 +18,10 @@ open MonoidalCategory
open OverColor
open HepLean.Fin
namespace TensorStruct
namespace TensorSpeciesStruct
noncomputable section
variable (S : TensorStruct)
variable (S : TensorSpeciesStruct)
lemma contrFin1Fin1_naturality {n : } {c c1 : Fin n.succ.succ → S.C}
{i : Fin n.succ.succ} {j : Fin n.succ} (h : c1 (i.succAbove j) = S.τ (c1 i))
@ -236,11 +236,11 @@ lemma contrMap_naturality {n : } {c c1 : Fin n.succ.succ → S.C}
rfl
end
end TensorStruct
end TensorSpeciesStruct
namespace TensorTree
variable {S : TensorStruct}
variable {S : TensorSpeciesStruct}
/-- Permuting indices, and then contracting is equivalent to contracting and then permuting,
once care is taking about ensuring one is contracting the same idices. -/