Spectral objects in triangulated categories #
In this file, we introduce the category SpectralObject C ι of spectral
objects in a pretriangulated category C indexed by the category ι.
TODO (@joelriou) #
- construct the spectral object indexed by
WithTop (WithBot ℤ)consisting of all truncations of an object of a triangulated category equipped with a t-structure - define a similar notion of spectral objects in abelian categories, show that
by applying an homological functor
C ⥤ Ato a spectral object in the triangulated categoryC, we obtain a spectral object in the abelian categoryA - construct the spectral sequence attached to a spectral object in an abelian category
References #
A spectral object in a pretriangulated category C indexed by a category ι consists
of a functor ω₁ : ComposableArrows ι 1 ⥤ C, and a functorial distinguished triangle
from the category ComposableArrows ι 2, which must be of the form
ω₁.obj (mk₁ f) ⟶ ω₁.obj (mk₁ (f ≫ g)) ⟶ ω₁.obj (mk₁ g) ⟶ ... when evaluated
on mk₂ f g : ComposableArrows ι 2.
- ω₁ : Functor (ComposableArrows ι 1) C
A functor from
ComposableArrows ι 1to the pretriangulated category. - δ' : (ComposableArrows.functorArrows ι 1 2 2 _proof_1 _proof_2).comp self.ω₁ ⟶ (ComposableArrows.functorArrows ι 0 1 2 _proof_3 _proof_1).comp (self.ω₁.comp (shiftFunctor C 1))
The connecting homomorphism of the spectral object.
- distinguished' (D : ComposableArrows ι 2) : Pretriangulated.Triangle.mk (self.ω₁.map ((ComposableArrows.mapFunctorArrows ι 0 1 0 2 2 _proof_3 _proof_4 _proof_5 _proof_1 _proof_2).app D)) (self.ω₁.map ((ComposableArrows.mapFunctorArrows ι 0 2 1 2 2 _proof_4 _proof_1 _proof_3 _proof_2 _proof_2).app D)) (self.δ'.app D) ∈ Pretriangulated.distinguishedTriangles
Instances For
The functorial (distinguished) triangle attached to a spectral object in a pretriangulated category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The connecting homomorphism X.ω₁.obj (mk₁ g) ⟶ (X.ω₁.obj (mk₁ f))⟦(1 : ℤ)⟧
of a spectral object X in a pretriangulated category when f : i ⟶ j and g : j ⟶ k
are composable.
Equations
- X.δ f g = X.δ'.app (CategoryTheory.ComposableArrows.mk₂ f g)
Instances For
The distinguished triangle attached to a spectral object E : SpectralObjet C ι
and composable morphisms f : i ⟶ j and g : j ⟶ k in ι.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The image of a spectral by a triangulated functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The type of morphisms between spectral objects in pretriangulated categories.
The natural transformation that is part of a morphism between spectral objects.
- comm {i j k : ι} (f : i ⟶ j) (g : j ⟶ k) : CategoryStruct.comp (X.δ f g) ((shiftFunctor C 1).map (self.hom.app (ComposableArrows.mk₁ f))) = CategoryStruct.comp (self.hom.app (ComposableArrows.mk₁ g)) (Y.δ f g)
Instances For
Equations
- One or more equations did not get rendered due to their size.
The functor between categories of spectral objects that is induced by a triangulated functor.
Equations
- One or more equations did not get rendered due to their size.