Documentation

Mathlib.CategoryTheory.Products.Unitor

The left/right unitor equivalences 1 × C ≌ C and C × 1 ≌ C. #

The left unitor functor 1 × C ⥤ C

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

    The right unitor functor C × 1 ⥤ C

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.prod.leftInverseUnitor_map (C : Type u) [CategoryTheory.Category.{v, u} C] :
      ∀ {X Y : C} (f : X Y), (CategoryTheory.prod.leftInverseUnitor C).map f = (CategoryTheory.CategoryStruct.id ((fun (X : C) => ({ as := PUnit.unit }, X)) X).1, f)

      The left inverse unitor C ⥤ 1 × C

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

        The right inverse unitor C ⥤ C × 1

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

          The equivalence of categories expressing left unity of products of categories.

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

            The equivalence of categories expressing right unity of products of categories.

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