Documentation

Mathlib.CategoryTheory.Triangulated.Subcategory

Triangulated subcategories #

In this file, we introduce the notion of triangulated subcategory of a pretriangulated category.

TODO #

Implementation notes #

In the definition of Triangulated.Subcategory, we do not assume that the predicate on objects is closed under isomorphisms (i.e. that the subcategory is "strictly full"). Part of the theory would be more convenient under this stronger assumption (e.g. Subcategory C would be a lattice), but some applications require this: for example, the subcategory of bounded below complexes in the homotopy category of an additive category is not closed under isomorphisms.

References #

A triangulated subcategory of a pretriangulated category C consists of a predicate P : C → Prop which contains a zero object, is stable by shifts, and such that if X₁ ⟶ X₂ ⟶ X₃ ⟶ X₁⟦1⟧ is a distinguished triangle such that if X₁ and X₃ satisfy P then X₂ is isomorphic to an object satisfying P.

Instances For
    def CategoryTheory.Triangulated.Subcategory.mk' {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Limits.HasZeroObject C] [CategoryTheory.HasShift C ] [CategoryTheory.Preadditive C] [∀ (n : ), (CategoryTheory.shiftFunctor C n).Additive] [CategoryTheory.Pretriangulated C] (P : CProp) (zero : P 0) (shift : ∀ (X : C) (n : ), P XP ((CategoryTheory.shiftFunctor C n).obj X)) (ext₂ : TCategoryTheory.Pretriangulated.distinguishedTriangles, P T.obj₁P T.obj₃P T.obj₂) :

    An alternative constructor for "strictly full" triangulated subcategory.

    Equations
    Instances For
      instance CategoryTheory.Triangulated.Subcategory.instClosedUnderIsomorphismsPMk' {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Limits.HasZeroObject C] [CategoryTheory.HasShift C ] [CategoryTheory.Preadditive C] [∀ (n : ), (CategoryTheory.shiftFunctor C n).Additive] [CategoryTheory.Pretriangulated C] (P : CProp) (zero : P 0) (shift : ∀ (X : C) (n : ), P XP ((CategoryTheory.shiftFunctor C n).obj X)) (ext₂ : TCategoryTheory.Pretriangulated.distinguishedTriangles, P T.obj₁P T.obj₃P T.obj₂) :
      Equations
      • =