Documentation

Mathlib.CategoryTheory.Linear.LinearFunctor

Linear Functors #

An additive functor between two R-linear categories is called linear if the induced map on hom types is a morphism of R-modules.

Implementation details #

Functor.Linear is a Prop-valued class, defined by saying that for every two objects X and Y, the map F.map : (X ⟶ Y) → (F.obj X ⟶ F.obj Y) is a morphism of R-modules.

An additive functor F is R-linear provided F.map is an R-module morphism.

  • map_smul {X Y : C} (f : X Y) (r : R) : F.map (r f) = r F.map f

    the functor induces a linear map on morphisms

Instances
    @[simp]
    theorem CategoryTheory.Functor.map_smul {R : Type u_1} [Semiring R] {C : Type u_2} {D : Type u_3} [Category.{u_4, u_2} C] [Category.{u_5, u_3} D] [Preadditive C] [Preadditive D] [CategoryTheory.Linear R C] [CategoryTheory.Linear R D] (F : Functor C D) [Linear R F] {X Y : C} (r : R) (f : X Y) :
    F.map (r f) = r F.map f
    @[simp]
    theorem CategoryTheory.Functor.map_units_smul {R : Type u_1} [Semiring R] {C : Type u_2} {D : Type u_3} [Category.{u_4, u_2} C] [Category.{u_5, u_3} D] [Preadditive C] [Preadditive D] [CategoryTheory.Linear R C] [CategoryTheory.Linear R D] (F : Functor C D) [Linear R F] {X Y : C} (r : Rˣ) (f : X Y) :
    F.map (r f) = r F.map f

    F.mapLinearMap is an R-linear map whose underlying function is F.map.

    Equations
    Instances For
      @[simp]
      theorem CategoryTheory.Functor.mapLinearMap_apply (R : Type u_1) [Semiring R] {C : Type u_2} {D : Type u_3} [Category.{u_4, u_2} C] [Category.{u_5, u_3} D] [Preadditive C] [Preadditive D] [CategoryTheory.Linear R C] [CategoryTheory.Linear R D] (F : Functor C D) [Linear R F] [F.Additive] {X Y : C} (a✝ : X Y) :
      (mapLinearMap R F) a✝ = (↑F.mapAddHom).toFun a✝