Documentation

Mathlib.AlgebraicTopology.SimplicialCategory.Basic

Simplicial categories #

A simplicial category is a category C that is enriched over the category of simplicial sets in such a way that morphisms in C identify to the 0-simplices of the enriched hom.

TODO #

References #

@[reducible, inline]
abbrev CategoryTheory.SimplicialCategory (C : Type u) [Category.{v, u} C] :
Type (max (max u (v + 1)) v)

A simplicial category is a category C that is enriched over the category of simplicial sets in such a way that morphisms in C identify to the 0-simplices of the enriched hom.

Equations
Instances For
    @[reducible, inline]

    Abbreviation for the enriched hom of a simplicial category.

    Equations
    Instances For
      @[reducible, inline]

      Abbreviation for the enriched composition in a simplicial category.

      Equations
      Instances For

        The bijection (K ⟶ L) ≃ sHom K L _[0] for all objects K and L in a simplicial category.

        Equations
        Instances For
          @[reducible, inline]

          The bifunctor Cᵒᵖ ⥤ C ⥤ SSet.{v} which sends K : Cᵒᵖ and L : C to sHom K.unop L.

          Equations
          Instances For