refactor: Fix imports and some lint

This commit is contained in:
jstoobysmith 2024-10-19 08:49:26 +00:00
parent 14bf127335
commit b2ac704d80
14 changed files with 47 additions and 69 deletions

View file

@ -105,6 +105,5 @@ lemma coMetric_apply_one : coMetric.hom (1 : ) = coMetricVal := by
change coMetric.hom.toFun (1 : ) = coMetricVal
simp [coMetric]
end Lorentz
end

View file

@ -46,7 +46,6 @@ lemma coCoToMatrix_symm_expand_tmul (M : Matrix (Fin 1 ⊕ Fin 3) (Fin 1 ⊕ Fin
rfl
· simp
/-- Equivalence of `complexContr ⊗ complexCo` to `4 x 4` complex matrices. -/
def contrCoToMatrix : (complexContr ⊗ complexCo).V ≃ₗ[]
Matrix (Fin 1 ⊕ Fin 3) (Fin 1 ⊕ Fin 3) :=