Exact sequences #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In a category with zero morphisms, images, and equalizers we say that f : A ⟶ B
and g : B ⟶ C
are exact if f ≫ g = 0
and the natural map image f ⟶ kernel g
is an epimorphism.
In any preadditive category this is equivalent to the homology at B
vanishing.
However in general it is weaker than other reasonable definitions of exactness, particularly that
- the inclusion map
image.ι f
is a kernel ofg
or image f ⟶ kernel g
is an isomorphism orimage_subobject f = kernel_subobject f
. However when the category is abelian, these all become equivalent; these results are found incategory_theory/abelian/exact.lean
.
Main results #
- Suppose that cokernels exist and that
f
andg
are exact. Ifs
is any kernel fork overg
andt
is any cokernel cofork overf
, thenfork.ι s ≫ cofork.π t = 0
. - Precomposing the first morphism with an epimorphism retains exactness. Postcomposing the second morphism with a monomorphism retains exactness.
- If
f
andg
are exact andi
is an isomorphism, thenf ≫ i.hom
andi.inv ≫ g
are also exact.
Future work #
- Short exact sequences, split exact sequences, the splitting lemma (maybe only for abelian categories?)
- Two adjacent maps in a chain complex are exact iff the homology vanishes
- w : f ≫ g = 0
- epi : category_theory.epi (image_to_kernel f g _)
Two morphisms f : A ⟶ B
, g : B ⟶ C
are called exact if w : f ≫ g = 0
and the natural map
image_to_kernel f g w : image_subobject f ⟶ kernel_subobject g
is an epimorphism.
In any preadditive category, this is equivalent to w : f ≫ g = 0
and homology f g w ≅ 0
.
In an abelian category, this is equivalent to image_to_kernel f g w
being an isomorphism,
and hence equivalent to the usual definition,
image_subobject f = kernel_subobject g
.
In any preadditive category,
composable morphisms f g
are exact iff they compose to zero and the homology vanishes.
A reformulation of preadditive.exact_of_iso_of_exact
that does not involve the arrow
category.
The dual of this lemma is only true when V
is abelian, see abelian.exact_epi_comp_iff
.
- reflects : ∀ {A B C : V} (f : A ⟶ B) (g : B ⟶ C), category_theory.exact (F.map f) (F.map g) → category_theory.exact f g
A functor reflects exact sequences if any composable pair of morphisms that is mapped to an exact pair is itself exact.
Instances of this typeclass
Instances of other typeclasses for category_theory.functor.reflects_exact_sequences
- category_theory.functor.reflects_exact_sequences.has_sizeof_inst