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

@ -81,7 +81,7 @@ instance : DecidableEq Color := fun x y =>
noncomputable section
/-- The tensor structure for complex Lorentz tensors. -/
def complexLorentzTensor : TensorSpeciesStruct where
def complexLorentzTensor : TensorSpecies where
C := Fermion.Color
G := SL(2, )
G_group := inferInstance

View file

@ -59,7 +59,7 @@ lemma coMetric_expand : {Lorentz.coMetric | μ ν}ᵀ.tensor =
lemma coMetric_symm : {Lorentz.coMetric | μ ν = Lorentz.coMetric | ν μ}ᵀ := by
simp only [Nat.succ_eq_add_one, Nat.reduceAdd, Fin.isValue, perm_tensor]
rw [coMetric_expand]
simp only [TensorSpeciesStruct.F, Nat.succ_eq_add_one, Nat.reduceAdd, Functor.id_obj, Fin.isValue,
simp only [TensorSpecies.F, Nat.succ_eq_add_one, Nat.reduceAdd, Functor.id_obj, Fin.isValue,
map_sub]
congr 1
congr 1