Short exact sequences in abelian categories #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In an abelian category, a left-split or right-split short exact sequence admits a splitting.
To construct a splitting of A -f⟶ B -g⟶ C
it suffices to supply
a morphism i : B ⟶ A ⊞ C
such that f ≫ i
is the canonical map biprod.inl : A ⟶ A ⊞ C
and
i ≫ q = g
, where q
is the canonical map biprod.snd : A ⊞ C ⟶ C
,
together with proofs that f
is mono and g
is epi.
The morphism i
is then automatically an isomorphism.
Equations
- category_theory.splitting.mk' h i h1 h2 = {iso := category_theory.as_iso i _, comp_iso_eq_inl := _, iso_comp_snd_eq := h2}
To construct a splitting of A -f⟶ B -g⟶ C
it suffices to supply
a morphism i : A ⊞ C ⟶ B
such that p ≫ i = f
where p
is the canonical map
biprod.inl : A ⟶ A ⊞ C
, and i ≫ g
is the canonical map biprod.snd : A ⊞ C ⟶ C
,
together with proofs that f
is mono and g
is epi.
The morphism i
is then automatically an isomorphism.
Equations
- category_theory.splitting.mk'' h i h1 h2 = {iso := (category_theory.as_iso i).symm, comp_iso_eq_inl := _, iso_comp_snd_eq := _}
A short exact sequence that is left split admits a splitting.
Equations
A short exact sequence that is right split admits a splitting.