Functorial resolutions give derivability structures #
In this file, we provide a constructor for right derivability structures.
We assume that Φ : LocalizerMorphism W₁ W₂
is given by
a fully faithful functor Φ.functor : C₁ ⥤ C₂
and that we have a resolution
functor ρ : C₂ ⥤ C₁
with a natural transformation i : 𝟭 C₂ ⟶ ρ ⋙ Φ.functor
such that W₂ (i.app X₂)
for any X₂ : C₂
. If we assume
that W₁
is induced by W₂
, that W₂
is multiplicative and has
the two out of three property, then Φ
is a right derivability structure.
If Φ : LocalizerMorphism W₁ W₂
corresponds to a class W₁
that is
the inverse image of W₂
by the functor Φ.functor
and that we
have functorial right resolutions, then this is a morphism of localizers
in the other direction.
Equations
- CategoryTheory.LocalizerMorphism.functorialRightResolutions.localizerMorphismInv hi hW₁ = { functor := ρ, map := ⋯ }
Instances For
If Φ : LocalizerMorphism W₁ W₂
corresponds to a class W₁
that is
induced by W₂
via the fully faithful functor Φ.functor
and we
have functorial right resolutions given by a functor ρ : C₂ ⥤ C₁
, then
this is the natural transformation 𝟭 C₁ ⟶ Φ.functor ⋙ ρ
induced
by i : 𝟭 C₂ ⟶ ρ ⋙ Φ.functor
.