refactor: Rename TensorSpeciesStruct to TensorSpecies
This commit is contained in:
parent
ef0d857cb7
commit
271745c11a
9 changed files with 25 additions and 26 deletions
|
@ -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
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue