Documentation

Mathlib.CategoryTheory.Abelian.NonPreadditive

Every NonPreadditiveAbelian category is preadditive #

In mathlib, we define an abelian category as a preadditive category with a zero object, kernels and cokernels, products and coproducts and in which every monomorphism and epimorphism is normal.

While virtually every interesting abelian category has a natural preadditive structure (which is why it is included in the definition), preadditivity is not actually needed: Every category that has all of the other properties appearing in the definition of an abelian category admits a preadditive structure. This is the construction we carry out in this file.

The proof proceeds in roughly five steps:

  1. Prove some results (for example that all equalizers exist) that would be trivial if we already had the preadditive structure but are a bit of work without it.
  2. Develop images and coimages to show that every monomorphism is the kernel of its cokernel.

The results of the first two steps are also useful for the "normal" development of abelian categories, and will be used there.

  1. For every object A, define a "subtraction" morphism σ : A ⨯ A ⟶ A and use it to define subtraction on morphisms as f - g := prod.lift f g ≫ σ.
  2. Prove a small number of identities about this subtraction from the definition of σ.
  3. From these identities, prove a large number of other identities that imply that defining f + g := f - (0 - g) indeed gives an abelian group structure on morphisms such that composition is bilinear.

The construction is non-trivial and it is quite remarkable that this abelian group structure can be constructed purely from the existence of a few limits and colimits. Even more remarkably, since abelian categories admit exactly one preadditive structure (see subsingletonPreadditiveOfHasBinaryBiproducts), the construction manages to exactly reconstruct any natural preadditive structure the category may have.

References #

We call a category NonPreadditiveAbelian if it has a zero object, kernels, cokernels, binary products and coproducts, and every monomorphism and every epimorphism is normal.

Instances

    In a NonPreadditiveAbelian category, an epi is the cokernel of its kernel. More precisely: If f is an epimorphism and s is some limit kernel cone on f, then f is a cokernel of Fork.ι s.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      In a NonPreadditiveAbelian category, a mono is the kernel of its cokernel. More precisely: If f is a monomorphism and s is some colimit cokernel cocone on f, then f is a kernel of Cofork.π s.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[inline, reducible]

        The composite A ⟶ A ⨯ A ⟶ cokernel (Δ A), where the first map is (𝟙 A, 0) and the second map is the canonical projection into the cokernel.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[inline, reducible]

          The composite A ⨯ A ⟶ cokernel (diag A) ⟶ A given by the natural projection into the cokernel followed by the inverse of r. In the category of modules, using the normal kernels and cokernels, this map is equal to the map (a, b) ↦ a - b, hence the name σ for "subtraction".

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For

            σ is a cokernel of Δ X.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              theorem CategoryTheory.NonPreadditiveAbelian.σ_comp {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.NonPreadditiveAbelian C] {X : C} {Y : C} (f : X Y) :
              CategoryTheory.CategoryStruct.comp CategoryTheory.NonPreadditiveAbelian.σ f = CategoryTheory.CategoryStruct.comp (CategoryTheory.Limits.prod.map f f) CategoryTheory.NonPreadditiveAbelian.σ

              This is the key identity satisfied by σ.

              Subtraction of morphisms in a NonPreadditiveAbelian category.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                Negation of morphisms in a NonPreadditiveAbelian category.

                Equations
                • CategoryTheory.NonPreadditiveAbelian.hasNeg = { neg := fun (f : X Y) => 0 - f }
                Instances For

                  Addition of morphisms in a NonPreadditiveAbelian category.

                  Equations
                  • CategoryTheory.NonPreadditiveAbelian.hasAdd = { add := fun (f g : X Y) => f - -g }
                  Instances For
                    theorem CategoryTheory.NonPreadditiveAbelian.sub_sub_sub {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.NonPreadditiveAbelian C] {X : C} {Y : C} (a : X Y) (b : X Y) (c : X Y) (d : X Y) :
                    a - c - (b - d) = a - b - (c - d)
                    theorem CategoryTheory.NonPreadditiveAbelian.sub_add {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.NonPreadditiveAbelian C] {X : C} {Y : C} (a : X Y) (b : X Y) (c : X Y) :
                    a - b + c = a - (b - c)
                    theorem CategoryTheory.NonPreadditiveAbelian.add_assoc {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.NonPreadditiveAbelian C] {X : C} {Y : C} (a : X Y) (b : X Y) (c : X Y) :
                    a + b + c = a + (b + c)

                    Every NonPreadditiveAbelian category is preadditive.

                    Equations
                    • CategoryTheory.NonPreadditiveAbelian.preadditive = { homGroup := fun (X Y : C) => AddCommGroup.mk , add_comp := , comp_add := }
                    Instances For