Documentation

Mathlib.CategoryTheory.Linear.FunctorCategory

Linear structure on functor categories #

If C and D are categories and D is R-linear, then C ⥤ D is also R-linear.

Equations

Application of a natural transformation at a fixed object, as group homomorphism

Equations
Instances For
    @[simp]
    theorem CategoryTheory.NatTrans.app_smul {R : Type u_1} [Semiring R] {C : Type u_2} {D : Type u_3} [CategoryTheory.Category.{u_5, u_2} C] [CategoryTheory.Category.{u_4, u_3} D] [CategoryTheory.Preadditive D] [CategoryTheory.Linear R D] {F G : CategoryTheory.Functor C D} (X : C) (r : R) (α : F G) :
    (r α).app X = r α.app X