feat: Writing toDualRep in terms of contrOneTwoLeft
This commit is contained in:
parent
5d21f74062
commit
2c26584cfc
5 changed files with 49 additions and 13 deletions
|
@ -120,7 +120,8 @@ lemma contrOneTwoLeft_unitTensor {c1 : S.C} (x : S.F.obj (OverColor.mk ![c1]))
|
|||
Action.instMonoidalCategory_leftUnitor_hom_hom, Monoidal.tensorUnit_obj,
|
||||
Action.instMonoidalCategory_whiskerRight_hom, Functor.comp_obj, Discrete.functor_obj_eq_as,
|
||||
Function.comp_apply, Action.instMonoidalCategory_associator_inv_hom, Equivalence.symm_inverse,
|
||||
Action.functorCategoryEquivalence_functor, Action.FunctorCategoryEquivalence.functor_obj_obj]
|
||||
Action.functorCategoryEquivalence_functor, Action.FunctorCategoryEquivalence.functor_obj_obj,
|
||||
forgetLiftAppCon_inv_apply_expand]
|
||||
erw [pairIsoSep_inv_unitTensor (S := S) (c := c1)]
|
||||
change (S.F.mapIso (mkIso _)).hom.hom _ = _
|
||||
rw [Discrete.rep_iso_apply_iff, Discrete.rep_iso_inv_apply_iff]
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue