Documentation

Mathlib.CategoryTheory.Linear.Basic

Linear categories #

An R-linear category is a category in which X ⟶ Y is an R-module in such a way that composition of morphisms is R-linear in both variables.

Note that sometimes in the literature a "linear category" is further required to be abelian.

Implementation #

Corresponding to the fact that we need to have an AddCommGroup X structure in place to talk about a Module R X structure, we need Preadditive C as a prerequisite typeclass for Linear R C. This makes for longer signatures than would be ideal.

Future work #

It would be nice to have a usable framework of enriched categories in which this just became a category enriched in Module R.

class CategoryTheory.Linear (R : Type w) [Semiring R] (C : Type u) [Category.{v, u} C] [Preadditive C] :
Type (max (max u v) w)

A category is called R-linear if P ⟶ Q is an R-module such that composition is R-linear in both variables.

Instances
    Equations
    Equations
    instance CategoryTheory.Linear.inducedCategory {C : Type u} [Category.{v, u} C] [Preadditive C] {R : Type w} [Semiring R] [Linear R C] {D : Type u'} (F : DC) :
    Equations
    Equations
    def CategoryTheory.Linear.leftComp {C : Type u} [Category.{v, u} C] [Preadditive C] (R : Type w) [Semiring R] [Linear R C] {X Y : C} (Z : C) (f : X Y) :
    (Y Z) →ₗ[R] X Z

    Composition by a fixed left argument as an R-linear map.

    Equations
    Instances For
      @[simp]
      theorem CategoryTheory.Linear.leftComp_apply {C : Type u} [Category.{v, u} C] [Preadditive C] (R : Type w) [Semiring R] [Linear R C] {X Y : C} (Z : C) (f : X Y) (g : Y Z) :
      def CategoryTheory.Linear.rightComp {C : Type u} [Category.{v, u} C] [Preadditive C] (R : Type w) [Semiring R] [Linear R C] (X : C) {Y Z : C} (g : Y Z) :
      (X Y) →ₗ[R] X Z

      Composition by a fixed right argument as an R-linear map.

      Equations
      Instances For
        @[simp]
        theorem CategoryTheory.Linear.rightComp_apply {C : Type u} [Category.{v, u} C] [Preadditive C] (R : Type w) [Semiring R] [Linear R C] (X : C) {Y Z : C} (g : Y Z) (f : X Y) :
        instance CategoryTheory.Linear.instEpiHSMulHomOfInvertible {C : Type u} [Category.{v, u} C] [Preadditive C] (R : Type w) [Semiring R] [Linear R C] {X Y : C} (f : X Y) [Epi f] (r : R) [Invertible r] :
        Epi (r f)
        instance CategoryTheory.Linear.instMonoHSMulHomOfInvertible {C : Type u} [Category.{v, u} C] [Preadditive C] (R : Type w) [Semiring R] [Linear R C] {X Y : C} (f : X Y) [Mono f] (r : R) [Invertible r] :
        Mono (r f)
        def CategoryTheory.Linear.homCongr (k : Type u_1) {C : Type u_2} [Category.{u_3, u_2} C] [Semiring k] [Preadditive C] [Linear k C] {X Y W Z : C} (f₁ : X Y) (f₂ : W Z) :
        (X W) ≃ₗ[k] Y Z

        Given isomorphic objects X ≅ Y, W ≅ Z in a k-linear category, we have a k-linear isomorphism between Hom(X, W) and Hom(Y, Z).

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem CategoryTheory.Linear.homCongr_apply (k : Type u_1) {C : Type u_2} [Category.{u_3, u_2} C] [Semiring k] [Preadditive C] [Linear k C] {X Y W Z : C} (f₁ : X Y) (f₂ : W Z) (f : X W) :
          (homCongr k f₁ f₂) f = CategoryStruct.comp (CategoryStruct.comp f₁.inv f) f₂.hom
          theorem CategoryTheory.Linear.homCongr_symm_apply (k : Type u_1) {C : Type u_2} [Category.{u_3, u_2} C] [Semiring k] [Preadditive C] [Linear k C] {X Y W Z : C} (f₁ : X Y) (f₂ : W Z) (f : Y Z) :
          (homCongr k f₁ f₂).symm f = CategoryStruct.comp f₁.hom (CategoryStruct.comp f f₂.inv)
          @[simp]
          theorem CategoryTheory.Linear.units_smul_comp {C : Type u} [Category.{v, u} C] [Preadditive C] {R : Type w} [Semiring R] [Linear R C] {X Y Z : C} (r : Rˣ) (f : X Y) (g : Y Z) :
          @[simp]
          theorem CategoryTheory.Linear.comp_units_smul {C : Type u} [Category.{v, u} C] [Preadditive C] {R : Type w} [Semiring R] [Linear R C] {X Y Z : C} (f : X Y) (r : Rˣ) (g : Y Z) :
          def CategoryTheory.Linear.comp {C : Type u} [Category.{v, u} C] [Preadditive C] {S : Type w} [CommSemiring S] [Linear S C] (X Y Z : C) :
          (X Y) →ₗ[S] (Y Z) →ₗ[S] X Z

          Composition as a bilinear map.

          Equations
          Instances For
            @[simp]
            theorem CategoryTheory.Linear.comp_apply {C : Type u} [Category.{v, u} C] [Preadditive C] {S : Type w} [CommSemiring S] [Linear S C] (X Y Z : C) (f : X Y) :
            (comp X Y Z) f = leftComp S Z f