Documentation

Mathlib.CategoryTheory.Triangulated.Subcategory

Triangulated subcategories #

In this file, given a pretriangulated category C and P : ObjectProperty C, we introduce a typeclass P.IsTriangulated to express that P is a triangulated subcategory of C. When P is a triangulated subcategory, we introduce a class of morphisms P.trW : MorphismProperty C consisting of the morphisms whose "cone" belongs to P (up to isomorphisms), and we show that it has both calculus of left and right fractions.

TODO #

Implementation notes #

In the definition of P.IsTriangulated, 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. the subtype of ObjectProperty C consisting of triangulated subcategories 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 #

Given P : ObjectProperty C with C a pretriangulated category, this is the property that whenever X₁ ⟶ X₂ ⟶ X₃ ⟶ X₁⟦1⟧ is a distinguished triangle such that P X₂ and P X₃ hold, then P.isoClosure X₁ holds.

Instances

    Given P : ObjectProperty C with C a pretriangulated category, this is the property that whenever X₁ ⟶ X₂ ⟶ X₃ ⟶ X₁⟦1⟧ is a distinguished triangle such that P X₁ and P X₃ hold, then P.isoClosure X₂ holds.

    Instances

      Given P : ObjectProperty C with C a pretriangulated category, this is the property that whenever X₁ ⟶ X₂ ⟶ X₃ ⟶ X₁⟦1⟧ is a distinguished triangle such that P X₁ and P X₂ hold, then P.isoClosure X₃ holds.

      Instances

        The property that P : ObjectProperty C is a triangulated subcategory (of a pretriangulated category C).

        Instances

          Given P : ObjectProperty C with C a pretriangulated category, this is the class of morphisms whose cone satisfies P. (The name trW contains the prefix tr for "triangulated", and W is a letter that is often used to refer to classes of morphisms with respect to which we may consider the localized category.)

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem CategoryTheory.ObjectProperty.trW.shift {C : Type u_1} [Category.{u_2, u_1} C] [Limits.HasZeroObject C] [HasShift C ] [Preadditive C] [∀ (n : ), (shiftFunctor C n).Additive] [Pretriangulated C] {P : ObjectProperty C} [P.IsStableUnderShift ] {X₁ X₂ : C} {f : X₁ X₂} (hf : P.trW f) (n : ) :
            P.trW ((shiftFunctor C n).map f)
            theorem CategoryTheory.ObjectProperty.trW.unshift {C : Type u_1} [Category.{u_2, u_1} C] [Limits.HasZeroObject C] [HasShift C ] [Preadditive C] [∀ (n : ), (shiftFunctor C n).Additive] [Pretriangulated C] (P : ObjectProperty C) [P.IsStableUnderShift ] {X₁ X₂ : C} {f : X₁ X₂} {n : } (hf : P.trW ((shiftFunctor C n).map f)) :
            P.trW f
            @[deprecated CategoryTheory.ObjectProperty.IsTriangulated (since := "2025-07-21")]

            Alias of CategoryTheory.ObjectProperty.IsTriangulated.


            The property that P : ObjectProperty C is a triangulated subcategory (of a pretriangulated category C).

            Equations
            Instances For
              @[deprecated CategoryTheory.ObjectProperty.IsTriangulatedClosed₂.mk' (since := "2025-07-21")]

              Alias of CategoryTheory.ObjectProperty.IsTriangulatedClosed₂.mk'.

              @[deprecated CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₁ (since := "2025-07-21")]

              Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₁.

              @[deprecated CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₁' (since := "2025-07-21")]

              Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₁'.

              @[deprecated CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₂ (since := "2025-07-21")]

              Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₂.

              @[deprecated CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₂' (since := "2025-07-21")]

              Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₂'.

              @[deprecated CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₃ (since := "2025-07-21")]

              Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₃.

              @[deprecated CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₃' (since := "2025-07-21")]

              Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₃'.

              @[deprecated CategoryTheory.ObjectProperty.trW (since := "2025-07-21")]

              Alias of CategoryTheory.ObjectProperty.trW.


              Given P : ObjectProperty C with C a pretriangulated category, this is the class of morphisms whose cone satisfies P. (The name trW contains the prefix tr for "triangulated", and W is a letter that is often used to refer to classes of morphisms with respect to which we may consider the localized category.)

              Equations
              Instances For
                @[deprecated CategoryTheory.ObjectProperty.trW_iff (since := "2025-07-21")]

                Alias of CategoryTheory.ObjectProperty.trW_iff.

                @[deprecated CategoryTheory.ObjectProperty.trW_iff' (since := "2025-07-21")]

                Alias of CategoryTheory.ObjectProperty.trW_iff'.

                @[deprecated CategoryTheory.ObjectProperty.trW.mk (since := "2025-07-21")]

                Alias of CategoryTheory.ObjectProperty.trW.mk.

                @[deprecated CategoryTheory.ObjectProperty.trW.mk' (since := "2025-07-21")]

                Alias of CategoryTheory.ObjectProperty.trW.mk'.

                @[deprecated CategoryTheory.ObjectProperty.trW_isoClosure (since := "2025-07-21")]

                Alias of CategoryTheory.ObjectProperty.trW_isoClosure.

                @[deprecated CategoryTheory.ObjectProperty.trW_of_isIso (since := "2025-07-21")]

                Alias of CategoryTheory.ObjectProperty.trW_of_isIso.

                @[deprecated CategoryTheory.ObjectProperty.smul_mem_trW_iff (since := "2025-07-21")]

                Alias of CategoryTheory.ObjectProperty.smul_mem_trW_iff.

                @[deprecated CategoryTheory.ObjectProperty.trW.shift (since := "2025-07-21")]
                theorem CategoryTheory.Triangulated.Subcategory.W.shift {C : Type u_1} [Category.{u_2, u_1} C] [Limits.HasZeroObject C] [HasShift C ] [Preadditive C] [∀ (n : ), (shiftFunctor C n).Additive] [Pretriangulated C] {P : ObjectProperty C} [P.IsStableUnderShift ] {X₁ X₂ : C} {f : X₁ X₂} (hf : P.trW f) (n : ) :
                P.trW ((shiftFunctor C n).map f)

                Alias of CategoryTheory.ObjectProperty.trW.shift.

                @[deprecated CategoryTheory.ObjectProperty.trW.unshift (since := "2025-07-21")]
                theorem CategoryTheory.Triangulated.Subcategory.W.unshift {C : Type u_1} [Category.{u_2, u_1} C] [Limits.HasZeroObject C] [HasShift C ] [Preadditive C] [∀ (n : ), (shiftFunctor C n).Additive] [Pretriangulated C] (P : ObjectProperty C) [P.IsStableUnderShift ] {X₁ X₂ : C} {f : X₁ X₂} {n : } (hf : P.trW ((shiftFunctor C n).map f)) :
                P.trW f

                Alias of CategoryTheory.ObjectProperty.trW.unshift.