Left derived functors #
In this file, given a functor F : C ⥤ H
, and L : C ⥤ D
that is a
localization functor for W : MorphismProperty C
, we define
F.totalLeftDerived L W : D ⥤ H
as the right Kan extension of F
along L
: it is defined if the type class F.HasLeftDerivedFunctor W
asserting the existence of a right Kan extension is satisfied.
(The name totalLeftDerived
is to avoid name-collision with
Functor.leftDerived
which are the left derived functors in
the context of abelian categories.)
Given LF : D ⥤ H
and α : L ⋙ RF ⟶ F
, we also introduce a type class
F.IsLeftDerivedFunctor α W
saying that α
is a right Kan extension of F
along the localization functor L
.
(This file was obtained by dualizing the results in the file
CategoryTheory.Functor.Derived.RightDerived
.)
References #
- https://ncatlab.org/nlab/show/derived+functor
A functor LF : D ⥤ H
is a left derived functor of F : C ⥤ H
if it is equipped with a natural transformation α : L ⋙ LF ⟶ F
which makes it a right Kan extension of F
along L
,
where L : C ⥤ D
is a localization functor for W : MorphismProperty C
.
- isRightKanExtension : LF.IsRightKanExtension α
Instances
Constructor for natural transformations to a left derived functor.
Equations
- LF.leftDerivedLift α W G β = LF.liftOfIsRightKanExtension α G β
Instances For
The natural transformation LF' ⟶ LF
on left derived functors that is
induced by a natural transformation F' ⟶ F
.
Equations
- LF'.leftDerivedNatTrans LF α' α W τ = LF.leftDerivedLift α W LF' (CategoryTheory.CategoryStruct.comp α' τ)
Instances For
The natural isomorphism LF' ≅ LF
on left derived functors that is
induced by a natural isomorphism F' ≅ F
.
Equations
- LF'.leftDerivedNatIso LF α' α W τ = { hom := LF'.leftDerivedNatTrans LF α' α W τ.hom, inv := LF.leftDerivedNatTrans LF' α α' W τ.inv, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Uniqueness (up to a natural isomorphism) of the left derived functor.
Equations
- LF'.leftDerivedUnique LF α α'₂ W = LF.leftDerivedNatIso LF' α α'₂ W (CategoryTheory.Iso.refl F)
Instances For
A functor F : C ⥤ H
has a left derived functor with respect to
W : MorphismProperty C
if it has a right Kan extension along
W.Q : C ⥤ W.Localization
(or any localization functor L : C ⥤ D
for W
, see hasLeftDerivedFunctor_iff
).
- hasRightKanExtension' : W.Q.HasRightKanExtension F
Instances
Given a functor F : C ⥤ H
, and a localization functor L : D ⥤ H
for W
,
this is the left derived functor D ⥤ H
of F
, i.e. the right Kan extension
of F
along L
.
Equations
- F.totalLeftDerived L W = L.rightKanExtension F
Instances For
The canonical natural transformation L ⋙ F.totalLeftDerived L W ⟶ F
.
Equations
- F.totalLeftDerivedCounit L W = L.rightKanExtensionCounit F