Documentation

Mathlib.CategoryTheory.Preadditive.Yoneda.Basic

The Yoneda embedding for preadditive categories #

The Yoneda embedding for preadditive categories sends an object Y to the presheaf sending an object X to the group of morphisms X ⟶ Y. At each point, we get an additional End Y-module structure.

We also show that this presheaf is additive and that it is compatible with the normal Yoneda embedding in the expected way and deduce that the preadditive Yoneda embedding is fully faithful.

TODO #

@[simp]
theorem CategoryTheory.preadditiveYonedaObj_map {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (Y : C) :
∀ {X Y_1 : Cᵒᵖ} (f : X Y_1), (CategoryTheory.preadditiveYonedaObj Y).map f = ModuleCat.ofHom { toAddHom := { toFun := fun (g : X.unop Y) => CategoryTheory.CategoryStruct.comp f.unop g, map_add' := }, map_smul' := }

The Yoneda embedding for preadditive categories sends an object Y to the presheaf sending an object X to the End Y-module of morphisms X ⟶ Y.

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

    The Yoneda embedding for preadditive categories sends an object Y to the presheaf sending an object X to the group of morphisms X ⟶ Y. At each point, we get an additional End Y-module structure, see preadditiveYonedaObj.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.preadditiveCoyonedaObj_map {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (X : Cᵒᵖ) :
      ∀ {X_1 Y : C} (f : X_1 Y), (CategoryTheory.preadditiveCoyonedaObj X).map f = ModuleCat.ofHom { toAddHom := { toFun := fun (g : X.unop X_1) => CategoryTheory.CategoryStruct.comp g f, map_add' := }, map_smul' := }

      The Yoneda embedding for preadditive categories sends an object X to the copresheaf sending an object Y to the End X-module of morphisms X ⟶ Y.

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

        The Yoneda embedding for preadditive categories sends an object X to the copresheaf sending an object Y to the group of morphisms X ⟶ Y. At each point, we get an additional End X-module structure, see preadditiveCoyonedaObj.

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

          Composing the preadditive yoneda embedding with the forgetful functor yields the regular Yoneda embedding.

          @[simp]

          Composing the preadditive yoneda embedding with the forgetful functor yields the regular Yoneda embedding.

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