refactor: Rename TensorSpeciesStruct to TensorSpecies

This commit is contained in:
jstoobysmith 2024-10-21 12:24:17 +00:00
parent ef0d857cb7
commit 271745c11a
9 changed files with 25 additions and 26 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 `TensorSpeciesStruct.contrMap_tprod`.
There is very likely a better way to do this using `TensorSpecies.contrMap_tprod`.
-/
@ -18,10 +18,10 @@ open MonoidalCategory
open OverColor
open HepLean.Fin
namespace TensorSpeciesStruct
namespace TensorSpecies
noncomputable section
variable (S : TensorSpeciesStruct)
variable (S : TensorSpecies)
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 TensorSpeciesStruct
end TensorSpecies
namespace TensorTree
variable {S : TensorSpeciesStruct}
variable {S : TensorSpecies}
/-- Permuting indices, and then contracting is equivalent to contracting and then permuting,
once care is taking about ensuring one is contracting the same idices. -/