Documentation

Mathlib.CategoryTheory.Bicategory.SingleObj

Promoting a monoidal category to a single object bicategory. #

A monoidal category can be thought of as a bicategory with a single object.

The objects of the monoidal category become the 1-morphisms, with composition given by tensor product, and the morphisms of the monoidal category become the 2-morphisms.

We verify that the endomorphisms of that single object recovers the original monoidal category.

One could go much further: the bicategory of monoidal categories (equipped with monoidal functors and monoidal natural transformations) is equivalent to the bicategory consisting of

Promote a monoidal category to a bicategory with a single object. (The objects of the monoidal category become the 1-morphisms, with composition given by tensor product, and the morphisms of the monoidal category become the 2-morphisms.)

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

    The unique object in the bicategory obtained by "promoting" a monoidal category.

    Equations
    Instances For

      The monoidal functor from the endomorphisms of the single object when we promote a monoidal category to a single object bicategory, to the original monoidal category.

      We subsequently show this is an equivalence.

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

        The equivalence between the endomorphisms of the single object when we promote a monoidal category to a single object bicategory, and the original monoidal category.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem CategoryTheory.MonoidalSingleObj.endMonoidalStarFunctorEquivalence_counitIso (C : Type u_1) [Category.{u_2, u_1} C] [MonoidalCategory C] :
          (endMonoidalStarFunctorEquivalence C).counitIso = Iso.refl ({ obj := fun (X : C) => X, map := fun {X Y : C} (f : X Y) => f, map_id := , map_comp := }.comp (endMonoidalStarFunctor C))