Documentation

Mathlib.CategoryTheory.Abelian.EpiWithInjectiveKernel

Epimorphisms with an injective kernel #

In this file, we define the class of morphisms epiWithInjectiveKernel in an abelian category. We show that this property of morphisms is multiplicative.

This shall be used in the file Mathlib.Algebra.Homology.Factorizations.Basic in order to define morphisms of cochain complexes which satisfy this property degreewise.

A morphism g : X ⟶ Y is epi with an injective kernel iff there exists a morphism f : I ⟶ X with I injective such that f ≫ g = 0 and the short complex I ⟶ X ⟶ Y has a splitting.

instance CategoryTheory.Abelian.instIsMultiplicativeEpiWithInjectiveKernel {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Abelian C] :
CategoryTheory.Abelian.epiWithInjectiveKernel.IsMultiplicative
Equations
  • =