Documentation

Mathlib.CategoryTheory.Preadditive.LeftExact

Left exactness of functors between preadditive categories #

We show that a functor is left exact in the sense that it preserves finite limits, if it preserves kernels. The dual result holds for right exact functors and cokernels.

Main results #

def CategoryTheory.Functor.isLimitMapConeBinaryFanOfPreservesKernels {C : Type u₁} [Category.{v₁, u₁} C] [Preadditive C] {D : Type u₂} [Category.{v₂, u₂} D] [Preadditive D] (F : Functor C D) [F.PreservesZeroMorphisms] {X Y Z : C} (π₁ : Z X) (π₂ : Z Y) [Limits.PreservesLimit (Limits.parallelPair π₂ 0) F] (i : Limits.IsLimit (Limits.BinaryFan.mk π₁ π₂)) :
Limits.IsLimit (F.mapCone (Limits.BinaryFan.mk π₁ π₂))

A functor between preadditive categories which preserves kernels preserves that an arbitrary binary fan is a limit.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem CategoryTheory.Functor.preservesBinaryProduct_of_preservesKernels {C : Type u₁} [Category.{v₁, u₁} C] [Preadditive C] {D : Type u₂} [Category.{v₂, u₂} D] [Preadditive D] (F : Functor C D) [F.PreservesZeroMorphisms] [∀ {X Y : C} (f : X Y), Limits.PreservesLimit (Limits.parallelPair f 0) F] {X Y : C} :

    A kernel preserving functor between preadditive categories preserves any pair being a limit.

    A kernel preserving functor between preadditive categories preserves binary products.

    A functor between preadditive categories preserves the equalizer of two morphisms if it preserves all kernels.

    A functor between preadditive categories preserves all equalizers if it preserves all kernels.

    A functor between preadditive categories which preserves kernels preserves all finite limits.

    def CategoryTheory.Functor.isColimitMapCoconeBinaryCofanOfPreservesCokernels {C : Type u₁} [Category.{v₁, u₁} C] [Preadditive C] {D : Type u₂} [Category.{v₂, u₂} D] [Preadditive D] (F : Functor C D) [F.PreservesZeroMorphisms] {X Y Z : C} (ι₁ : X Z) (ι₂ : Y Z) [Limits.PreservesColimit (Limits.parallelPair ι₂ 0) F] (i : Limits.IsColimit (Limits.BinaryCofan.mk ι₁ ι₂)) :
    Limits.IsColimit (F.mapCocone (Limits.BinaryCofan.mk ι₁ ι₂))

    A functor between preadditive categories which preserves cokernels preserves finite coproducts.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem CategoryTheory.Functor.preservesCoproduct_of_preservesCokernels {C : Type u₁} [Category.{v₁, u₁} C] [Preadditive C] {D : Type u₂} [Category.{v₂, u₂} D] [Preadditive D] (F : Functor C D) [F.PreservesZeroMorphisms] [∀ {X Y : C} (f : X Y), Limits.PreservesColimit (Limits.parallelPair f 0) F] {X Y : C} :

      A cokernel preserving functor between preadditive categories preserves any pair being a colimit.

      A cokernel preserving functor between preadditive categories preserves binary coproducts.

      A functor between preadditive categories preserves the coequalizer of two morphisms if it preserves all cokernels.

      A functor between preadditive categories preserves all coequalizers if it preserves all kernels.

      A functor between preadditive categories which preserves kernels preserves all finite limits.