Documentation

Mathlib.AlgebraicTopology.SimplicialSet.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 [GJ09], 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 #

The nerve of a category

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

    Given a functor C ⥤ D, we obtain a morphism nerve C ⟶ nerve D of simplicial sets.

    Equations
    Instances For

      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
        @[simp]
        theorem CategoryTheory.nerveFunctor_map {X✝ Y✝ : Cat} (F : X✝ Y✝) :

        The 0-simplices of the nerve of a category are equivalent to the objects of the category.

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

          Nerves of finite non-empty ordinals are representable functors.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem CategoryTheory.nerve.δ_obj {C : Type u} [Category.{v, u} C] {n : } (i : Fin (n + 2)) (x : ComposableArrows C (n + 1)) (j : Fin (n + 1)) :
            theorem CategoryTheory.nerve.σ_obj {C : Type u} [Category.{v, u} C] {n : } (i : Fin (n + 1)) (x : ComposableArrows C n) (j : Fin (n + 2)) :
            theorem CategoryTheory.nerve.δ₂_mk₂_eq {C : Type u} [Category.{v, u} C] {X₀ X₁ X₂ : C} (f : X₀ X₁) (g : X₁ X₂) :
            theorem CategoryTheory.nerve.δ₀_mk₂_eq {C : Type u} [Category.{v, u} C] {X₀ X₁ X₂ : C} (f : X₀ X₁) (g : X₁ X₂) :

            Bijection between edges in the nerve of category and morphisms in the category.

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

              Constructor for edges in the nerve of a category. (See also homEquiv.)

              Equations
              Instances For
                @[simp]
                @[simp]
                theorem CategoryTheory.nerve.homEquiv_edgeMk {C : Type u} [Category.{v, u} C] {x y : C} (f : x y) :
                theorem CategoryTheory.nerve.nonempty_compStruct_iff {C : Type u} [Category.{v, u} C] {x₀ x₁ x₂ : C} (f₀₁ : x₀ x₁) (f₁₂ : x₁ x₂) (f₀₂ : x₀ x₂) :
                Nonempty ((edgeMk f₀₁).CompStruct (edgeMk f₁₂) (edgeMk f₀₂)) CategoryStruct.comp f₀₁ f₁₂ = f₀₂
                theorem CategoryTheory.nerve.homEquiv_comp {C : Type u} [Category.{v, u} C] {x₀ x₁ x₂ : ComposableArrows C 0} {e₀₁ : SSet.Edge x₀ x₁} {e₁₂ : SSet.Edge x₁ x₂} {e₀₂ : SSet.Edge x₀ x₂} (h : e₀₁.CompStruct e₁₂ e₀₂) :
                CategoryStruct.comp (homEquiv e₀₁) (homEquiv e₁₂) = homEquiv e₀₂
                @[simp]
                theorem CategoryTheory.nerve.homEquiv_edgeMk_map_nerveMap {C : Type u} [Category.{v, u} C] {D : Type u} [Category.{v, u} D] {x y : C} (f : x y) (F : Functor C D) :