Skip to content

Commit

Permalink
fix Shift.Adjunction
Browse files Browse the repository at this point in the history
  • Loading branch information
morel committed Jan 6, 2025
1 parent 40999e1 commit a739e23
Showing 1 changed file with 5 additions and 5 deletions.
10 changes: 5 additions & 5 deletions Mathlib/CategoryTheory/Shift/Adjunction.lean
Original file line number Diff line number Diff line change
Expand Up @@ -197,8 +197,8 @@ The property for `CommShift` structures on `F` and `G` to be compatible with an
adjunction `F ⊣ G`.
-/
class CommShift : Prop where
commShift_unit' : NatTrans.CommShift adj.unit A := by infer_instance
commShift_counit' : NatTrans.CommShift adj.counit A := by infer_instance
commShift_unit : NatTrans.CommShift adj.unit A := by infer_instance
commShift_counit : NatTrans.CommShift adj.counit A := by infer_instance

open CommShift in
attribute [instance] commShift_unit commShift_counit
Expand Down Expand Up @@ -229,7 +229,7 @@ namespace CommShift
/-- Constructor for `Adjunction.CommShift`. -/
lemma mk' (h : NatTrans.CommShift adj.unit A) :
adj.CommShift A where
commShift_counit' := ⟨fun a ↦ by
commShift_counit := ⟨fun a ↦ by
ext
simp only [Functor.comp_obj, Functor.id_obj, NatTrans.comp_app,
Functor.commShiftIso_comp_hom_app, whiskerRight_app, assoc, whiskerLeft_app,
Expand Down Expand Up @@ -512,8 +512,8 @@ instance [h : E.inverse.CommShift A] : E.symm.functor.CommShift A := h
/-- Constructor for `Equivalence.CommShift`. -/
lemma mk' (h : NatTrans.CommShift E.unitIso.hom A) :
E.CommShift A where
commShift_unit' := h
commShift_counit' := (Adjunction.CommShift.mk' E.toAdjunction A h).commShift_counit
commShift_unit := h
commShift_counit := (Adjunction.CommShift.mk' E.toAdjunction A h).commShift_counit

/--
The forward functor of the identity equivalence is compatible with shifts.
Expand Down

0 comments on commit a739e23

Please sign in to comment.