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 #
- show that the fullsubcategory attached to
P
(such thatP.IsTriangulated
) is a pretriangulated category.
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.
- ext₁' (T : Pretriangulated.Triangle C) : T ∈ Pretriangulated.distinguishedTriangles → P T.obj₂ → P T.obj₃ → P.isoClosure T.obj₁
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.
- ext₂' (T : Pretriangulated.Triangle C) : T ∈ Pretriangulated.distinguishedTriangles → P T.obj₁ → P T.obj₃ → P.isoClosure T.obj₂
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.
- ext₃' (T : Pretriangulated.Triangle C) : T ∈ Pretriangulated.distinguishedTriangles → P T.obj₁ → P T.obj₂ → P.isoClosure T.obj₃
Instances
The property that P : ObjectProperty C
is a triangulated subcategory
(of a pretriangulated category C
).
- exists_zero : ∃ (Z : C), Limits.IsZero Z ∧ P Z
- ext₂' (T : Pretriangulated.Triangle C) : T ∈ Pretriangulated.distinguishedTriangles → P T.obj₁ → P T.obj₃ → P.isoClosure T.obj₂
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
Alias of CategoryTheory.ObjectProperty.IsTriangulated
.
The property that P : ObjectProperty C
is a triangulated subcategory
(of a pretriangulated category C
).
Instances For
Alias of CategoryTheory.ObjectProperty.IsTriangulatedClosed₂.mk'
.
Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₁
.
Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₁'
.
Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₂
.
Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₂'
.
Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₃
.
Alias of CategoryTheory.ObjectProperty.ext_of_isTriangulatedClosed₃'
.
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.)
Instances For
Alias of CategoryTheory.ObjectProperty.trW_iff
.
Alias of CategoryTheory.ObjectProperty.trW_iff'
.
Alias of CategoryTheory.ObjectProperty.trW.mk
.
Alias of CategoryTheory.ObjectProperty.trW.mk'
.
Alias of CategoryTheory.ObjectProperty.trW.shift
.
Alias of CategoryTheory.ObjectProperty.trW_iff_of_distinguished
.