refactor: Some golfing

This commit is contained in:
jstoobysmith 2024-10-19 10:57:09 +00:00
parent ae7f8dea1e
commit 2cb219773e
7 changed files with 12 additions and 30 deletions

View file

@ -146,7 +146,6 @@ lemma contrIso_comm_aux_3 {n : } {c c1 : Fin n.succ.succ → S.C}
((HepLean.Fin.finExtractOnePerm ((Hom.toEquiv σ).symm i) (Hom.toEquiv σ)).symm j))).hom) ≫
(S.F.map (extractTwo i j σ)) := by
rw [← Functor.map_comp, ← Functor.map_comp]
apply congrArg
rfl
exact congrArg (λ f => Action.Hom.hom f) h1
@ -234,8 +233,7 @@ lemma contrMap_naturality {n : } {c c1 : Fin n.succ.succ → S.C}
erw [CategoryTheory.Category.id_comp, CategoryTheory.Category.comp_id]
erw [CategoryTheory.Category.comp_id]
rw [S.contr.naturality]
simp only [Nat.succ_eq_add_one, extractOne_homToEquiv, Monoidal.tensorUnit_obj,
Monoidal.tensorUnit_map, Category.comp_id]
rfl
end
end TensorStruct