refactor: Rename TensorSpeciesStruct to TensorSpecies
This commit is contained in:
parent
ef0d857cb7
commit
271745c11a
9 changed files with 25 additions and 26 deletions
|
@ -22,7 +22,7 @@ open TensorProduct
|
|||
|
||||
namespace TensorTree
|
||||
|
||||
variable {S : TensorSpeciesStruct}
|
||||
variable {S : TensorSpecies}
|
||||
|
||||
/-!
|
||||
|
||||
|
|
|
@ -21,7 +21,7 @@ open HepLean.Fin
|
|||
|
||||
namespace TensorTree
|
||||
|
||||
variable {S : TensorSpeciesStruct}
|
||||
variable {S : TensorSpecies}
|
||||
|
||||
/-- A structure containing two pairs of indices (i, j) and (k, l) to be sequentially
|
||||
contracted in a tensor. -/
|
||||
|
@ -168,7 +168,7 @@ lemma contrSwapHom_contrMapSnd_tprod (x : (i : (𝟭 Type).obj (OverColor.mk c).
|
|||
(x (q.swap.i.succAbove (q.swap.j.succAbove (q.swap.k.succAbove q.swap.l))))))) •
|
||||
((lift.obj S.FDiscrete).map q.contrSwapHom).hom ((PiTensorProduct.tprod S.k) fun k =>
|
||||
x (q.swap.i.succAbove (q.swap.j.succAbove (q.swap.k.succAbove (q.swap.l.succAbove k)))))) := by
|
||||
rw [contrMapSnd,TensorSpeciesStruct.contrMap_tprod]
|
||||
rw [contrMapSnd,TensorSpecies.contrMap_tprod]
|
||||
change ((lift.obj S.FDiscrete).map q.contrSwapHom).hom
|
||||
(_ • ((PiTensorProduct.tprod S.k) fun k =>
|
||||
x (q.swap.i.succAbove (q.swap.j.succAbove
|
||||
|
@ -214,7 +214,7 @@ lemma contrMapFst_contrMapSnd_swap :
|
|||
(S.F.map q.contrSwapHom).hom
|
||||
(q.swap.contrMapSnd.hom ((S.contrMap c q.swap.i q.swap.j _).hom
|
||||
((PiTensorProduct.tprod S.k) x)))
|
||||
rw [TensorSpeciesStruct.contrMap_tprod, TensorSpeciesStruct.contrMap_tprod]
|
||||
rw [TensorSpecies.contrMap_tprod, TensorSpecies.contrMap_tprod]
|
||||
simp only [Nat.succ_eq_add_one, Monoidal.tensorUnit_obj, Action.instMonoidalCategory_tensorUnit_V,
|
||||
Equivalence.symm_inverse, Action.functorCategoryEquivalence_functor,
|
||||
Action.FunctorCategoryEquivalence.functor_obj_obj, Functor.comp_obj, Discrete.functor_obj_eq_as,
|
||||
|
@ -226,7 +226,7 @@ lemma contrMapFst_contrMapSnd_swap :
|
|||
((lift.obj S.FDiscrete).map q.contrSwapHom).hom
|
||||
(q.swap.contrMapSnd.hom ((PiTensorProduct.tprod S.k)
|
||||
fun k => x (q.swap.i.succAbove (q.swap.j.succAbove k))))
|
||||
rw [contrMapSnd, TensorSpeciesStruct.contrMap_tprod, q.contrSwapHom_contrMapSnd_tprod]
|
||||
rw [contrMapSnd, TensorSpecies.contrMap_tprod, q.contrSwapHom_contrMapSnd_tprod]
|
||||
rw [smul_smul, smul_smul]
|
||||
congr 1
|
||||
/- The contractions. -/
|
||||
|
|
|
@ -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. -/
|
||||
|
|
|
@ -19,7 +19,7 @@ open HepLean.Fin
|
|||
|
||||
namespace TensorTree
|
||||
|
||||
variable {S : TensorSpeciesStruct} {n n' n2 : ℕ}
|
||||
variable {S : TensorSpecies} {n n' n2 : ℕ}
|
||||
{c : Fin n → S.C} {c' : Fin n' → S.C} (c2 : Fin n2 → S.C)
|
||||
(σ : OverColor.mk c ⟶ OverColor.mk c')
|
||||
|
||||
|
|
|
@ -19,7 +19,7 @@ open HepLean.Fin
|
|||
|
||||
namespace TensorTree
|
||||
|
||||
variable {S : TensorSpeciesStruct} {n n2 : ℕ}
|
||||
variable {S : TensorSpecies} {n n2 : ℕ}
|
||||
(c : Fin n → S.C) (c2 : Fin n2 → S.C)
|
||||
|
||||
/-- The permutation that arises when moving a commuting terms in a `prod` node.
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue