Documentation

Mathlib.AlgebraicTopology.Nerve

The nerve of a category #

This file provides the definition of the nerve of a category C, which is a simplicial set nerve C (see [goerss-jardine-2009], Example I.1.4). By definition, the type of n-simplices of nerve C is ComposableArrows C n, which is the category Fin (n + 1) ⥤ C.

References #

@[simp]
theorem CategoryTheory.nerve_map (C : Type u) [CategoryTheory.Category.{v, u} C] :
∀ {X Y : SimplexCategoryᵒᵖ} (f : X Y) (x : CategoryTheory.ComposableArrows C X.unop.len), (CategoryTheory.nerve C).map f x = x.whiskerLeft (SimplexCategory.toCat.map f.unop)

The nerve of a category

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    Equations
    • CategoryTheory.instCategoryObjOppositeSimplexCategoryNerve = inferInstance

    The nerve of a category, as a functor Cat ⥤ SSet

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For