Pointwise right derived functors #
We define the pointwise right derived functors using the notion of pointwise left Kan extensions.
We show that if F : C ⥤ H
inverts W : MorphismProperty C
,
then it has a pointwise right derived functor.
Given F : C ⥤ H
, W : MorphismProperty C
and X : C
, we say that F
has a
pointwise right derived functor at X
if F
has a left Kan extension
at L.obj X
for any localization functor L : C ⥤ D
for W
. In the
definition, this is stated for L := W.Q
, see hasPointwiseRightDerivedFunctorAt_iff
for the more general equivalence.
- hasColimit' : W.Q.HasPointwiseLeftKanExtensionAt F (W.Q.obj X)
Use the more general
hasColimit
lemma instead, see alsohasPointwiseRightDerivedFunctorAt_iff
Instances
A functor F : C ⥤ H
has a pointwise right derived functor with respect to
W : MorphismProperty C
if it has a pointwise right derived functor at X
for any X : C
.
Equations
- F.HasPointwiseRightDerivedFunctor W = ∀ (X : C), F.HasPointwiseRightDerivedFunctorAt W X
Instances For
A right derived functor is a pointwise right derived functor when there exists a pointwise right derived functor.
Equations
Instances For
If L : C ⥤ D
is a localization functor for W
and e : F ≅ L ⋙ G
is an isomorphism,
then e.hom
makes G
a pointwise left Kan extension of F
along L
at L.obj Y
for any Y : C
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If L
is a localization functor for W
and e : F ≅ L ⋙ G
is an isomorphism,
then e.hom
makes G
a poinwise left Kan extension of F
along L
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Let L : C ⥤ D
be a localization functor for W
, if an extension E
of F : C ⥤ H
along L
is such that the natural transformation
E.hom : F ⟶ L ⋙ E.right
is an isomorphism, then E
is a pointwise
left Kan extension.