Short exact sequences, and splittings. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
short_exact f g
is the proposition that 0 ⟶ A -f⟶ B -g⟶ C ⟶ 0
is an exact sequence.
We define when a short exact sequence is left-split, right-split, and split.
See also #
In algebra.homology.short_exact.abelian
we show that in an abelian category
a left-split short exact sequences admits a splitting.
- mono : category_theory.mono f
- epi : category_theory.epi g
- exact : category_theory.exact f g
If f : A ⟶ B
and g : B ⟶ C
then short_exact f g
is the proposition saying
the resulting diagram 0 ⟶ A ⟶ B ⟶ C ⟶ 0
is an exact sequence.
- left_split : ∃ (φ : B ⟶ A), f ≫ φ = 𝟙 A
- epi : category_theory.epi g
- exact : category_theory.exact f g
An exact sequence A -f⟶ B -g⟶ C
is left split
if there exists a morphism φ : B ⟶ A
such that f ≫ φ = 𝟙 A
and g
is epi.
Such a sequence is automatically short exact (i.e., f
is mono).
- right_split : ∃ (χ : C ⟶ B), χ ≫ g = 𝟙 C
- mono : category_theory.mono f
- exact : category_theory.exact f g
An exact sequence A -f⟶ B -g⟶ C
is right split
if there exists a morphism φ : C ⟶ B
such that f ≫ φ = 𝟙 A
and f
is mono.
Such a sequence is automatically short exact (i.e., g
is epi).
- split : ∃ (φ : B ⟶ A) (χ : C ⟶ B), f ≫ φ = 𝟙 A ∧ χ ≫ g = 𝟙 C ∧ f ≫ g = 0 ∧ χ ≫ φ = 0 ∧ φ ≫ f + g ≫ χ = 𝟙 B
An exact sequence A -f⟶ B -g⟶ C
is split if there exist
φ : B ⟶ A
and χ : C ⟶ B
such that:
f ≫ φ = 𝟙 A
χ ≫ g = 𝟙 C
f ≫ g = 0
χ ≫ φ = 0
φ ≫ f + g ≫ χ = 𝟙 B
Such a sequence is automatically short exact (i.e., f
is mono and g
is epi).
The sequence A ⟶ A ⊞ B ⟶ B
is exact.
The sequence B ⟶ A ⊞ B ⟶ A
is exact.
- iso : B ≅ A ⊞ C
- comp_iso_eq_inl : f ≫ self.iso.hom = category_theory.limits.biprod.inl
- iso_comp_snd_eq : self.iso.hom ≫ category_theory.limits.biprod.snd = g
A splitting of a sequence A -f⟶ B -g⟶ C
is an isomorphism
to the short exact sequence 0 ⟶ A ⟶ A ⊞ C ⟶ C ⟶ 0
such that
the vertical maps on the left and the right are the identity.
Instances for category_theory.splitting
- category_theory.splitting.has_sizeof_inst
If h
is a splitting of A -f⟶ B -g⟶ C
,
then h.section : C ⟶ B
is the morphism satisfying h.section ≫ g = 𝟙 C
.
Instances for category_theory.splitting.section
If h
is a splitting of A -f⟶ B -g⟶ C
,
then h.retraction : B ⟶ A
is the morphism satisfying f ≫ h.retraction = 𝟙 A
.
Equations
Instances for category_theory.splitting.retraction
The retraction in a splitting is a split mono.
Equations
- h.split_mono = {retraction := h.retraction, id' := _}
The section in a splitting is a split epi.
A short exact sequence of the form X -f⟶ Y -0⟶ Z
where f
is an iso and Z
is zero
has a splitting.