refactor: Lint

This commit is contained in:
jstoobysmith 2024-10-03 11:25:00 +00:00
parent f555bc6722
commit 31422a5e1d
2 changed files with 5 additions and 4 deletions

View file

@ -50,12 +50,10 @@ lemma toEquiv_symm_apply (m : f ⟶ g) (i : g.left) :
f.hom ((toEquiv m).symm i) = g.hom i := by
simpa [toEquiv, types_comp] using congrFun m.inv.w i
lemma toEquiv_comp_hom (m : f ⟶ g) : g.hom ∘ (toEquiv m) = f.hom := by
lemma toEquiv_comp_hom (m : f ⟶ g) : g.hom ∘ (toEquiv m) = f.hom := by
ext x
simpa [types_comp, toEquiv] using congrFun m.hom.w x
end Hom
instance (C : Type) : MonoidalCategoryStruct (OverColor C) where
@ -284,6 +282,5 @@ def colorFun : OverColor Color ⥤ Rep SL(2, ) where
Equiv.cast_apply, cast_cast, cast_inj]
rfl
end
end Fermion