refactor: Move Lemmas

This commit is contained in:
jstoobysmith 2024-11-10 07:00:48 +00:00
parent b0c5ed894f
commit a9143f79b6
2 changed files with 18 additions and 12 deletions

View file

@ -274,6 +274,23 @@ lemma toSelfAdjoint_symm_basis (i : Fin 1 ⊕ Fin 3) :
refine (LinearEquiv.symm_apply_eq toSelfAdjoint).mpr ?_
rw [toSelfAdjoint_stdBasis]
/-!
## Topology
-/
instance : TopologicalSpace (ContrMod d) := TopologicalSpace.induced
ContrMod.toFin1dEquiv (Pi.topologicalSpace)
lemma toFin1dEquiv_isInducing : IsInducing (@ContrMod.toFin1dEquiv d) := by
exact { eq_induced := rfl }
lemma toFin1dEquiv_symm_isInducing : IsInducing ((@ContrMod.toFin1dEquiv d).symm) := by
let x := Equiv.toHomeomorphOfIsInducing (@ContrMod.toFin1dEquiv d).toEquiv
toFin1dEquiv_isInducing
exact Homeomorph.isInducing x.symm
end ContrMod
/-- The module for covariant (up-index) complex Lorentz vectors. -/