Documentation

Mathlib.Algebra.Category.Grp.Yoneda

Yoneda embeddings #

This file defines a few Yoneda embeddings for the category of commutative groups.

The CommGrpCat-valued coyoneda embedding.

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

    The AddCommGrpCat-valued coyoneda embedding.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      @[simp]
      theorem CommGrpCat.coyoneda_map_app {X✝ Y✝ : CommGrpCatᵒᵖ} (f : X✝ Y✝) (N : CommGrpCat) :
      @[simp]
      theorem CommGrpCat.coyoneda_obj_map (M : CommGrpCatᵒᵖ) {X✝ Y✝ : CommGrpCat} (f : X✝ Y✝) :

      The CommGrpCat-valued coyoneda embedding composed with the forgetful functor is the usual coyoneda embedding.

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

        The AddCommGrpCat-valued coyoneda embedding composed with the forgetful functor is the usual coyoneda embedding.

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

          The Hom bifunctor sending a type X and a commutative group G to the commutative group X → G with pointwise operations.

          This is also the coyoneda embedding of Type into CommGrpCat-valued presheaves of commutative groups.

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

            The Hom bifunctor sending a type X and a commutative group G to the commutative group X → G with pointwise operations.

            This is also the coyoneda embedding of Type into AddCommGrpCat-valued presheaves of commutative groups.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[simp]
              @[simp]
              theorem AddCommGrpCat.coyonedaType_map_app {X✝ Y✝ : Type uᵒᵖ} (f : X✝ Y✝) (G : AddCommGrpCat) :
              (coyonedaType.map f).app G = ofHom (Pi.addMonoidHom fun (i : Opposite.unop Y✝) => Pi.evalAddMonoidHom (fun (a : Opposite.unop X✝) => G) (f.unop i))
              @[simp]
              theorem AddCommGrpCat.coyonedaType_obj_map (X : Type uᵒᵖ) {X✝ Y✝ : AddCommGrpCat} (f : X✝ Y✝) :
              (coyonedaType.obj X).map f = ofHom (Pi.addMonoidHom fun (i : Opposite.unop X) => (Hom.hom f).comp (Pi.evalAddMonoidHom (fun (a : Opposite.unop X) => X✝) i))
              @[simp]
              theorem CommGrpCat.coyonedaType_obj_map (X : Type uᵒᵖ) {X✝ Y✝ : CommGrpCat} (f : X✝ Y✝) :
              (coyonedaType.obj X).map f = ofHom (Pi.monoidHom fun (i : Opposite.unop X) => (Hom.hom f).comp (Pi.evalMonoidHom (fun (a : Opposite.unop X) => X✝) i))
              @[simp]
              theorem CommGrpCat.coyonedaType_map_app {X✝ Y✝ : Type uᵒᵖ} (f : X✝ Y✝) (G : CommGrpCat) :
              (coyonedaType.map f).app G = ofHom (Pi.monoidHom fun (i : Opposite.unop Y✝) => Pi.evalMonoidHom (fun (a : Opposite.unop X✝) => G) (f.unop i))