Documentation

Mathlib.Algebra.Homology.LeftResolution.Reduced

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
    @[simp]
    theorem CategoryTheory.Abelian.LeftResolution.karoubi.F'_map_f {A : Type u_1} {C : Type u_2} [Category.{u_3, u_2} C] [Category.{u_4, u_1} A] {ι : Functor C A} (Λ : LeftResolution ι) [Preadditive C] [Preadditive A] {X Y : A} (f : X Y) :
    ((F' Λ).map f).f = Λ.F.map f - Λ.F.map 0
    @[simp]
    @[simp]
    theorem CategoryTheory.Abelian.LeftResolution.karoubi.F_map_f {A : Type u_1} {C : Type u_2} [Category.{u_3, u_2} C] [Category.{u_4, u_1} A] {ι : Functor C A} (Λ : LeftResolution ι) [Preadditive C] [Preadditive A] {X✝ Y✝ : Idempotents.Karoubi A} (f : X✝ Y✝) :
    ((F Λ).map f).f = Λ.F.map f.f - Λ.F.map 0

    Auxiliary definition for LeftResolution.karoubi.

    Equations
    Instances For
      @[simp]

      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

        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
        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.
          Instances For