Commit 2025-01-10 18:19 0479fde8
View on Github →feat(CategoryTheory/Shift/Opposite and CategoryTheory/Shift/Pullback): CommShift
structures on adjunctions are compatible with opposites and pullbacks (#20363)
Suppose that we use categories C
and D
equiped with a shifts by an additive monoid A
, functors F,F' : C ⥤ D
, a functor G : D ⥤ C
, a natural transformation τ : F ⟶ F'
and an adjunction adj
between F
and G
.
- For any map of additive monoids
φ : B →+ A
, we define type synonymsPullbackShift.functor F φ
forF
,PullbackShift.natTrans τ φ
forτ
, andPullbackShift.adjunction adj φ
foradj
. We then prove that aCommShift
structure onF
(resp.τ
, resp.adj
) induces aCommShift
structure onPullbackShift.functor F φ
(resp.PullbackShift.natTrans τ φ
, resp.PullbackShift.adjunction adj φ
). - Similarly, we define type synonyms
OppositeShift.functor A F
forF.op
,OppositeShift.natTrans A τ
forτ.op
andOppositeShift.adjunction A adj
foradj.op
, and prove that aCommShift
structure onF
(resp.τ
, resp.adj
) induces aCommShift
structure onOppositeShift.functor A F
(resp.OppositeShift.natTrans A τ
, resp.OppositeShift.adjunction A adj
) for the naive shifts on the opposite categories. - The point of the second part is to reserve
F.op
etc to carryCommShift
structures for the modified shift on the opposite categories used in the theory of (pre)triangulated categories. We illustrate this by simplifying the definition of the instancecommShiftOpInt
(aCommShift ℤ
instance onF.op
for the modified shifts) in the fileTriangulated.Opposite.Functor
.
- depends on: #20364