The shift induced on a localized category #
Let C be a category equipped with a shift by a monoid A. A morphism property W
on C satisfies W.IsCompatibleWithShift A when for all a : A,
a morphism f is in W iff f⟦a⟧' is. When this compatibility is satisfied,
then the corresponding localized category can be equipped with
a shift by A, and the localization functor is compatible with the shift.
A morphism property W on a category C is compatible with the shift by a
monoid A when for all a : A, a morphism f belongs to W
if and only if f⟦a⟧' does.
the condition that for all
a : A, the morphism propertyWis not changed when we take its inverse image by the shift functor bya
Instances
The morphism of localizer from W to W given by the functor shiftFunctor C a
when a : A and W is compatible with the shift by A.
Equations
- W.shiftLocalizerMorphism a = { functor := CategoryTheory.shiftFunctor C a, map := ⋯ }
Instances For
When L : C ⥤ D is a localization functor with respect to a morphism property W
that is compatible with the shift by a monoid A on C, this is the induced
shift on the category D.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The localization functor L : C ⥤ D is compatible with the shift.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The localized category W.Localization is endowed with the induced shift.
Equations
The localization functor W.Q : C ⥤ W.Localization is compatible with the shift.
Equations
The localized category W.Localization' is endowed with the induced shift.
Equations
The localization functor W.Q' : C ⥤ W.Localization' is compatible with the shift.
Equations
Auxiliary definition for Functor.commShiftOfLocalization.
Equations
- One or more equations did not get rendered due to their size.
Instances For
In the context of localization of categories, if a functor is induced by a functor which commutes with the shift, then this functor commutes with the shift.
Equations
- L.commShiftOfLocalization W A F F' = { commShiftIso := CategoryTheory.Functor.commShiftOfLocalization.iso L W F F', commShiftIso_zero := ⋯, commShiftIso_add := ⋯ }
Instances For
This is the commutation of a functor G to shifts by an additive monoid M when
e : Φ.functor ⋙ L₂ ≅ L₁ ⋙ G is an isomorphism, Φ is a localizer morphism and
L₁ is a localization functor. We assume that all categories involved
are equipped with shifts and that L₁, L₂ and Φ.functor commute to them.
Equations
- Φ.commShift M L₁ L₂ G e = L₁.commShiftOfLocalization W₁ M (Φ.functor.comp L₂) G
Instances For
Equations
- Φ.instCommShiftLocalizedFunctor L₁ L₂ = Φ.commShift M L₁ L₂ (Φ.localizedFunctor L₁ L₂) (CategoryTheory.CatCommSq.iso Φ.functor L₁ L₂ (Φ.localizedFunctor L₁ L₂))