Subcomplexes of a simplicial set #
Given a simplicial set X, this file defines the type X.Subcomplex
of subcomplexes of X as an abbreviation for Subpresheaf X.
It also introduces a coercion from X.Subcomplex to SSet.
Implementation note #
SSet.{u} is defined as Cᵒᵖ ⥤ Type u, but it is not an abbreviation.
This is the reason why Subpresheaf.ι is redefined here as Subcomplex.ι
so that this morphism appears as a morphism in SSet instead of a morphism
in the category of presheaves.
The complete lattice of subcomplexes of a simplicial set.
Equations
Instances For
The underlying simplicial set of a subcomplex.
Equations
Instances For
Equations
- SSet.Subcomplex.instCoeOut = { coe := fun (S : X.Subcomplex) => S.toSSet }
If A : Subcomplex X, this is the inclusion A ⟶ X in the category SSet.
Equations
Instances For
Given an inequality S₁ ≤ S₂ between subcomplexes of a simplicial set,
this is the induced morphism in the category SSet.
Equations
Instances For
This is the isomorphism of simplicial sets corresponding to an equality of subcomplexes.
Equations
- SSet.Subcomplex.eqToIso h = { hom := SSet.Subcomplex.homOfLE ⋯, inv := SSet.Subcomplex.homOfLE ⋯, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The functor which sends A : X.Subcomplex to A.toSSet.
Equations
- SSet.Subcomplex.toSSetFunctor = { obj := fun (A : X.Subcomplex) => A.toSSet, map := fun {X_1 Y : X.Subcomplex} (h : X_1 ⟶ Y) => SSet.Subcomplex.homOfLE ⋯, map_id := ⋯, map_comp := ⋯ }
Instances For
If X : SSet, this is the isomorphism of simplicial sets
from ⊤ : X.Subcomplex to X.
Equations
- SSet.Subcomplex.topIso X = CategoryTheory.NatIso.ofComponents (fun (n : SimplexCategoryᵒᵖ) => (Equiv.Set.univ (X.obj n)).toIso) ⋯
Instances For
If X is a simplicial set, then the empty subcomplex of X is an initial
object in SSet.
Instances For
The subcomplex of a simplicial set that is generated by a simplex.
Instances For
The range of a morphism of simplicial sets, as a subcomplex.
Equations
Instances For
The morphism X ⟶ Subcomplex.range f induced by f : X ⟶ Y.
Equations
Instances For
Given a morphism of simplicial sets f : X ⟶ Y whose
range is ≤ B for some B : Y.Subcomplex, this is the
induced morphism X ⟶ B.
Equations
Instances For
The preimage of a subcomplex by a morphism of simplicial sets.
Instances For
The image of a subcomplex by a morphism of simplicial sets.
Equations
- A.image f = CategoryTheory.Subpresheaf.image A f
Instances For
Given a morphism of simplicial sets f : X ⟶ Y and a subcomplex A of X,
this is the induced morphism from A to A.image f.
Equations
- A.toImage f = SSet.Subcomplex.lift (CategoryTheory.CategoryStruct.comp A.ι f) ⋯
Instances For
Given a morphism of simplicial sets p : Y ⟶ X and
A : X.Subcomplex, this is the induced morphism
(A.preimage p : SSet) ⟶ (A : SSet).
Equations
- A.fromPreimage p = SSet.Subcomplex.lift (CategoryTheory.CategoryStruct.comp (A.preimage p).ι p) ⋯