Documentation

Mathlib.CategoryTheory.Monoidal.Yoneda

Yoneda embedding of Mon_ C #

We show that monoid objects are exactly those whose yoneda presheaf is a presheaf of monoids, by constructing the yoneda embedding Mon_ C ⥤ Cᵒᵖ ⥤ MonCat.{v} and showing that it is fully faithful and its (essential) image is the representable functors.

If X represents a presheaf of monoids, then X is a monoid object.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[deprecated Mon_Class.ofRepresentableBy (since := "2025-03-07")]

    Alias of Mon_Class.ofRepresentableBy.


    If X represents a presheaf of monoids, then X is a monoid object.

    Equations
    Instances For
      @[reducible]

      If X is a monoid object, then Hom(Y, X) has a monoid structure.

      Equations
      Instances For

        If X is a monoid object, then Hom(-, X) is a presheaf of monoids.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem yonedaMonObj_map {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.ChosenFiniteProducts C] (X : C) [Mon_Class X] {Y₁ Y₂ : Cᵒᵖ} (φ : Y₁ Y₂) :
          (yonedaMonObj X).map φ = MonCat.ofHom { toFun := fun (x : Opposite.unop Y₁ X) => CategoryTheory.CategoryStruct.comp φ.unop x, map_one' := , map_mul' := }

          If X represents a presheaf of monoids F, then Hom(-, X) is isomorphic to F as a presheaf of monoids.

          Equations
          Instances For

            The yoneda embedding of Mon_C into presheaves of monoids.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[simp]
              theorem yonedaMon_map_app {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.ChosenFiniteProducts C] {X₁ X₂ : Mon_ C} (ψ : X₁ X₂) (Y : Cᵒᵖ) :
              (yonedaMon.map ψ).app Y = MonCat.ofHom { toFun := fun (x : Opposite.unop Y X₁.X) => CategoryTheory.CategoryStruct.comp x ψ.hom, map_one' := , map_mul' := }

              The yoneda embedding for Mon_C is fully faithful.

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

                If X represents a presheaf of commutative groups, then X is a commutative group object.