Left resolutions which preserve the zero object #
The structure LeftResolution allows to define a functorial
resolution of an object (see LeftResolution.chainComplexFunctor
in the file Algebra.Homology.LeftResolution.Basic). In
order to extend this resolution to complexes, we not only
need the functoriality but also that zero morphisms
are sent to zero. In this file, given ι : C ⥤ A,
we extend Λ : LeftResolution ι to idempotent completions as
Λ.karoubi : LeftResolution ((functorExtension₂ C A).obj ι), and
when both C and A are idempotent complete, we define
Λ.reduced : LeftResolution ι in such a way that the
functor Λ.reduced.F : A ⥤ C preserves zero morphisms.
For example, if A := ModuleCat R and C is the full subcategory
of flat R-modules, we may first define Λ by using the
functor which sends an R-module M to the free R-module
on the elements of M. Then, Λ.reduced.F.obj M will be obtained
from the free R-module on M by factoring out the direct factor
corresponding to the submodule spanned by the generator corresponding
to 0 : M (TODO).
Auxiliary definition for LeftResolution.karoubi.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Auxiliary definition for LeftResolution.karoubi.
Equations
Instances For
Auxiliary definition for LeftResolution.karoubi.
Equations
Instances For
The morphism (karoubi.π' Λ).app X is a retract of (toKaroubi _).map (Λ.π.app X).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Auxiliary definition for LeftResolution.karoubi.
Equations
Instances For
Given ι : C ⥤ A, this is the extension of Λ : LeftResolution ι to
LeftResolution ((functorExtension₂ C A).obj ι), where
(functorExtension₂ C A).obj ι : Karoubi C ⥤ Karoubi A is the extension of ι.
Equations
- Λ.karoubi = { F := CategoryTheory.Abelian.LeftResolution.karoubi.F Λ, π := CategoryTheory.Abelian.LeftResolution.karoubi.π Λ, epi_π_app := ⋯ }
Instances For
Given an additive functor ι : C ⥤ A between idempotent complete categories,
any Λ : LeftResolution ι induces a term Λ.reduced : LeftResolution ι
such that Λ.reduced.F preserves zero morphisms.
Equations
- One or more equations did not get rendered due to their size.