The (naive) shift on the opposite category #
If C
is a category equipped with a shift by a monoid A
, the opposite category
can be equipped with a shift such that the shift functor by n
is (shiftFunctor C n).op
.
This is the "naive" opposite shift, which we shall set on a category OppositeShift C A
,
which is a type synonym for Cᵒᵖ
.
However, for the application to (pre)triangulated categories, we would like to
define the shift on Cᵒᵖ
so that shiftFunctor Cᵒᵖ n
for n : ℤ
identifies to
(shiftFunctor C (-n)).op
rather than (shiftFunctor C n).op
. Then, the construction
of the shift on Cᵒᵖ
shall combine the shift on OppositeShift C A
and another
construction of the "pullback" of a shift by a monoid morphism like n ↦ -n
.
Construction of the naive shift on the opposite category of a category C
:
the shiftfunctor by n
is (shiftFunctor C n).op
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The category OppositeShift C A
is the opposite category Cᵒᵖ
equipped
with the naive shift: shiftFunctor (OppositeShift C A) n
is (shiftFunctor C n).op
.
Equations
Instances For
Equations
- CategoryTheory.instCategoryOppositeShift C A = id inferInstance
Equations
- CategoryTheory.instPreadditiveOppositeShift C A = id inferInstance
Given a CommShift
structure on F
, this is the corresponding CommShift
structure on
F.op
(for the naive shifts on the opposite categories).
Equations
- F.commShiftOp A = { iso := fun (a : A) => (CategoryTheory.NatIso.op (F.commShiftIso a)).symm, zero := ⋯, add := ⋯ }
Instances For
Given a CommShift
structure on F.op
(for the naive shifts on the opposite categories),
this is the corresponding CommShift
structure on F
.
Equations
- F.commShiftUnop A = { iso := fun (a : A) => CategoryTheory.NatIso.removeOp (F.op.commShiftIso a).symm, zero := ⋯, add := ⋯ }