Documentation

Mathlib.CategoryTheory.Linear.Yoneda

The Yoneda embedding for R-linear categories #

The Yoneda embedding for R-linear categories C, sends an object X : C to the ModuleCat R-valued presheaf on C, with value on Y : Cᵒᵖ given by ModuleCat.of R (unop Y ⟶ X).

TODO: linearYoneda R C is R-linear. TODO: In fact, linearYoneda itself is additive and R-linear.

The Yoneda embedding for R-linear categories C, sending an object X : C to the ModuleCat R-valued presheaf on C, with value on Y : Cᵒᵖ given by ModuleCat.of R (unop Y ⟶ X).

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CategoryTheory.linearYoneda_obj_obj_carrier (R : Type w) [Ring R] (C : Type u) [Category.{v, u} C] [Preadditive C] [Linear R C] (X : C) (Y : Cᵒᵖ) :
    (((linearYoneda R C).obj X).obj Y) = (Opposite.unop Y X)
    @[simp]
    theorem CategoryTheory.linearYoneda_map_app (R : Type w) [Ring R] (C : Type u) [Category.{v, u} C] [Preadditive C] [Linear R C] {X₁ X₂ : C} (f : X₁ X₂) (Y : Cᵒᵖ) :
    @[simp]
    theorem CategoryTheory.linearYoneda_obj_map (R : Type w) [Ring R] (C : Type u) [Category.{v, u} C] [Preadditive C] [Linear R C] (X : C) {X✝ Y✝ : Cᵒᵖ} (f : X✝ Y✝) :

    The Yoneda embedding for R-linear categories C, sending an object Y : Cᵒᵖ to the ModuleCat R-valued copresheaf on C, with value on X : C given by ModuleCat.of R (unop Y ⟶ X).

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.linearCoyoneda_obj_map (R : Type w) [Ring R] (C : Type u) [Category.{v, u} C] [Preadditive C] [Linear R C] (Y : Cᵒᵖ) {X✝ Y✝ : C} (f : X✝ Y✝) :
      @[simp]
      theorem CategoryTheory.linearCoyoneda_obj_obj_carrier (R : Type w) [Ring R] (C : Type u) [Category.{v, u} C] [Preadditive C] [Linear R C] (Y : Cᵒᵖ) (X : C) :
      (((linearCoyoneda R C).obj Y).obj X) = (Opposite.unop Y X)
      @[simp]
      theorem CategoryTheory.linearCoyoneda_map_app (R : Type w) [Ring R] (C : Type u) [Category.{v, u} C] [Preadditive C] [Linear R C] {Y₁ Y₂ : Cᵒᵖ} (f : Y₁ Y₂) (X : C) :