refactor: Lint

This commit is contained in:
jstoobysmith 2024-11-11 07:22:36 +00:00
parent a8243f4e79
commit 081955c993
6 changed files with 35 additions and 34 deletions

View file

@ -278,11 +278,9 @@ lemma toSelfAdjoint_symm_basis (i : Fin 1 ⊕ Fin 3) :
## Topology
-/
instance : TopologicalSpace (ContrMod d) := TopologicalSpace.induced
ContrMod.toFin1dEquiv (Pi.topologicalSpace)
lemma toFin1dEquiv_isInducing : IsInducing (@ContrMod.toFin1dEquiv d) := by
exact { eq_induced := rfl }