Documentation

Mathlib.Algebra.Homology.DerivedCategory.SingleTriangle

The distinguished triangle of a short exact sequence in an abelian category #

Given a short exact short complex S in an abelian category, we construct the associated distinguished triangle in the derived category: (singleFunctor C 0).obj S.X₁ ⟶ (singleFunctor C 0).obj S.X₂ ⟶ (singleFunctor C 0).obj S.X₃ ⟶ ...

TODO #

The connecting homomorphism (singleFunctor C 0).obj S.X₃ ⟶ ((singleFunctor C 0).obj S.X₁)⟦(1 : ℤ)⟧ in the derived category of C when S is a short exact short complex in C.

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

    The (distinguished) triangle in the derived category of C given by a short exact short complex in C.

    Equations
    Instances For

      Given a short exact complex S in C that is short exact (hS), this is the canonical isomorphism between the triangle hS.singleTriangle in the derived category and the triangle attached to the corresponding short exact sequence of cochain complexes after the application of the single functor.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        theorem CategoryTheory.ShortComplex.ShortExact.singleTriangle_distinguished {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Abelian C] [HasDerivedCategory C] {S : CategoryTheory.ShortComplex C} (hS : S.ShortExact) :
        hS.singleTriangle CategoryTheory.Pretriangulated.distinguishedTriangles

        The distinguished triangle in the derived category of C given by a short exact short complex in C.