Documentation

Mathlib.CategoryTheory.Preadditive.InjectiveResolution

Injective resolutions #

An injective resolution I : InjectiveResolution Z of an object Z : C consists of an -indexed cochain complex I.cocomplex of injective objects, along with a quasi-isomorphism I.ι from the cochain complex consisting just of Z in degree zero to I.cocomplex.

Z ----> 0 ----> ... ----> 0 ----> ...
|       |                 |
|       |                 |
v       v                 v
I⁰ ---> I¹ ---> ... ----> Iⁿ ---> ...

An InjectiveResolution Z consists of a bundled -indexed cochain complex of injective objects, along with a quasi-isomorphism from the complex consisting of just Z supported in degree 0.

  • cocomplex : CochainComplex C

    the cochain complex involved in the resolution

  • injective (n : ) : Injective (self.cocomplex.X n)

    the cochain complex must be degreewise injective

  • hasHomology (i : ) : HomologicalComplex.HasHomology self.cocomplex i

    the cochain complex must have homology

  • ι : (CochainComplex.single₀ C).obj Z self.cocomplex

    the morphism from the single cochain complex with Z in degree 0

  • quasiIso : QuasiIso self

    the morphism from the single cochain complex with Z in degree 0 is a quasi-isomorphism

Instances For

    An object admits an injective resolution.

    Instances

      You will rarely use this typeclass directly: it is implied by the combination [EnoughInjectives C] and [Abelian C].

      Instances
        theorem CategoryTheory.InjectiveResolution.exact_succ {C : Type u} [Category.{v, u} C] [Limits.HasZeroObject C] [Limits.HasZeroMorphisms C] {Z : C} (I : InjectiveResolution Z) (n : ) :
        (ShortComplex.mk (I.cocomplex.d n (n + 1)) (I.cocomplex.d (n + 1) (n + 2)) ).Exact
        theorem CategoryTheory.InjectiveResolution.complex_d_comp {C : Type u} [Category.{v, u} C] [Limits.HasZeroObject C] [Limits.HasZeroMorphisms C] {Z : C} (I : InjectiveResolution Z) (n : ) :
        CategoryStruct.comp (I.cocomplex.d n (n + 1)) (I.cocomplex.d (n + 1) (n + 2)) = 0

        The (limit) kernel fork given by the composition Z ⟶ I.cocomplex.X 0 ⟶ I.cocomplex.X 1 when I : InjectiveResolution Z.

        Equations
        Instances For

          Z is the kernel of I.cocomplex.X 0 ⟶ I.cocomplex.X 1 when I : InjectiveResolution Z.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For