Split simplicial objects #
In this file, we introduce the notion of split simplicial object.
If C
is a category that has finite coproducts, a splitting
s : Splitting X
of a simplical object X
in C
consists
of the datum of a sequence of objects s.N : ℕ → C
(which
we shall refer to as "nondegenerate simplices") and a
sequence of morphisms s.ι n : s.N n → X _[n]
that have
the property that a certain canonical map identifies X _[n]
with the coproduct of objects s.N i
indexed by all possible
epimorphisms [n] ⟶ [i]
in SimplexCategory
. (We do not
assume that the morphisms s.ι n
are monomorphisms: in the
most common categories, this would be a consequence of the
axioms.)
Simplicial objects equipped with a splitting form a category
SimplicialObject.Split C
.
References #
- [Stacks: Splitting simplicial objects] https://stacks.math.columbia.edu/tag/017O
The index set which appears in the definition of split simplicial objects.
Instances For
The element in Splitting.IndexSet Δ
attached to an epimorphism f : Δ ⟶ Δ'
.
Instances For
The epimorphism in SimplexCategory
associated to A : Splitting.IndexSet Δ
Instances For
The distinguished element in Splitting.IndexSet Δ
which corresponds to the
identity of Δ
.
Instances For
The condition that an element Splitting.IndexSet Δ
is the distinguished
element Splitting.IndexSet.Id Δ
.
Instances For
Given A : IndexSet Δ₁
, if p.unop : unop Δ₂ ⟶ unop Δ₁
is an epi, this
is the obvious element in A : IndexSet Δ₂
associated to the composition
of epimorphisms p.unop ≫ A.e
.
Instances For
When A : IndexSet Δ
and θ : Δ → Δ'
is a morphism in SimplexCategoryᵒᵖ
,
an element in IndexSet Δ'
can be defined by using the epi-mono factorisation
of θ.unop ≫ A.e
.
Instances For
Given a sequences of objects N : ℕ → C
in a category C
, this is
a family of objects indexed by the elements A : Splitting.IndexSet Δ
.
The Δ
-simplices of a split simplicial objects shall identify to the
coproduct of objects in such a family.
Instances For
The coproduct of the family summand N Δ
Instances For
The inclusion of a summand in the coproduct.
Instances For
The canonical morphism coprod N Δ ⟶ X.obj Δ
attached to a sequence
of objects N
and a sequence of morphisms N n ⟶ X _[n]
.
Instances For
- N : ℕ → C
- ι : (n : ℕ) → SimplicialObject.Splitting.N s n ⟶ X.obj (Opposite.op (SimplexCategory.mk n))
- map_isIso : ∀ (Δ : SimplexCategoryᵒᵖ), CategoryTheory.IsIso (SimplicialObject.Splitting.map X s.ι Δ)
A splitting of a simplicial object X
consists of the datum of a sequence
of objects N
, a sequence of morphisms ι : N n ⟶ X _[n]
such that
for all Δ : SimplexCategoryᵒᵖ
, the canonical map Splitting.map X ι Δ
is an isomorphism.
Instances For
The isomorphism on simplices given by the axiom Splitting.map_isIso
Instances For
Via the isomorphism s.iso Δ
, this is the inclusion of a summand
in the direct sum decomposition given by the splitting s : Splitting X
.
Instances For
As it is stated in Splitting.hom_ext
, a morphism f : X ⟶ Y
from a split
simplicial object to any simplicial object is determined by its restrictions
s.φ f n : s.N n ⟶ Y _[n]
to the distinguished summands in each degree n
.
Instances For
The map X.obj Δ ⟶ Z
obtained by providing a family of morphisms on all the
terms of decomposition given by a splitting s : Splitting X
Instances For
A simplicial object that is isomorphic to a split simplicial object is split.
Instances For
- s : SimplicialObject.Splitting s.X
The category SimplicialObject.Split C
is the category of simplicial objects
in C
equipped with a splitting, and morphisms are morphisms of simplicial objects
which are compatible with the splittings.
Instances For
The object in SimplicialObject.Split C
attached to a splitting s : Splitting X
of a simplicial object X
.
Instances For
- F : S₁.X ⟶ S₂.X
- f : (n : ℕ) → SimplicialObject.Splitting.N S₁.s n ⟶ SimplicialObject.Splitting.N S₂.s n
- comm : ∀ (n : ℕ), CategoryTheory.CategoryStruct.comp (SimplicialObject.Splitting.ι S₁.s n) (s.F.app (Opposite.op (SimplexCategory.mk n))) = CategoryTheory.CategoryStruct.comp (SimplicialObject.Split.Hom.f s n) (SimplicialObject.Splitting.ι S₂.s n)
Morphisms in SimplicialObject.Split C
are morphisms of simplicial objects that
are compatible with the splittings.
Instances For
The functor SimplicialObject.Split C ⥤ SimplicialObject C
which forgets
the splitting.
Instances For
The functor SimplicialObject.Split C ⥤ C
which sends a simplicial object equipped
with a splitting to its nondegenerate n
-simplices.
Instances For
The inclusion of each summand in the coproduct decomposition of simplices
in split simplicial objects is a natural transformation of functors
SimplicialObject.Split C ⥤ C