Documentation

Mathlib.CategoryTheory.PUnit

The category Discrete PUnit #

We define star : C ⥤ Discrete PUnit sending everything to PUnit.star, show that any two functors to Discrete PUnit are naturally isomorphic, and construct the equivalence (Discrete PUnit ⥤ C) ≌ C.

The constant functor sending everything to PUnit.star.

Equations
Instances For
    @[simp]
    theorem CategoryTheory.Functor.star_map_down_down (C : Type u) [Category.{v, u} C] {X✝ Y✝ : C} (x✝ : X✝ Y✝) :
    =
    @[simp]
    theorem CategoryTheory.Functor.star_obj_as (C : Type u) [Category.{v, u} C] (x✝ : C) :
    ((star C).obj x✝).as = PUnit.unit

    Any two functors to Discrete PUnit are isomorphic.

    Equations
    Instances For

      Any two functors to Discrete PUnit are equal. You probably want to use punitExt instead of this.

      @[reducible, inline]

      The functor from Discrete PUnit sending everything to the given object.

      Equations
      Instances For

        Functors from Discrete PUnit are equivalent to the category itself.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem CategoryTheory.Functor.equiv_functor_obj {C : Type u} [Category.{v, u} C] (F : Functor (Discrete PUnit.{w + 1}) C) :
          equiv.functor.obj F = F.obj { as := PUnit.unit }
          @[simp]
          theorem CategoryTheory.Functor.equiv_functor_map {C : Type u} [Category.{v, u} C] {X✝ Y✝ : Functor (Discrete PUnit.{w + 1}) C} (θ : X✝ Y✝) :
          equiv.functor.map θ = θ.app { as := PUnit.unit }

          A category being equivalent to PUnit is equivalent to it having a unique morphism between any two objects. (In fact, such a category is also a groupoid; see CategoryTheory.Groupoid.ofHomUnique)