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_map_hom (R : Type w) [Ring R] (C : Type u) [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] [CategoryTheory.Linear R C] (X : C) {X✝ Y✝ : Cᵒᵖ} (f : X✝ Y✝) :
    (((CategoryTheory.linearYoneda R C).obj X).map f).hom = CategoryTheory.Linear.leftComp R X f.unop

    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]