Exactness of a pair #
For two maps
f : M → N
andg : N → P
, withZero P
,Function.Exact f g
says thatSet.range f = Set.preimage g {0}
For additive maps
f : M →+ N
andg : N →+ P
,Exact f g
says thatrange f = ker g
For linear maps
f : M →ₗ[R] N
andg : N →ₗ[R] P
,Exact f g
says thatrange f = ker g
TODO : #
generalize to
SemilinearMap
, evenSemilinearMapClass
add the multiplicative case (
Function.Exact
will becomeFunction.AddExact
?)
When we have a commutative diagram from a sequence of two maps to another,
such that the left vertical map is surjective, the middle vertical map is bijective and the right
vertical map is injective, then the upper row is exact iff the lower row is.
See ShortComplex.exact_iff_of_epi_of_isIso_of_mono
in the file
Algebra.Homology.ShortComplex.Exact
for the categorical version of this result.
Given an exact sequence 0 → M → N → P
, giving a section P → N
is equivalent to giving a
splitting N ≃ M × P
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given an exact sequence M → N → P → 0
, giving a retraction N → M
is equivalent to giving a
splitting N ≃ M × P
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equivalent characterizations of split exact sequences. Also known as the Splitting lemma.
A necessary and sufficient condition for an exact sequence to descend to a quotient.
When we have a commutative diagram from a sequence of two linear maps to another,
such that the left vertical map is surjective, the middle vertical map is bijective and the right
vertical map is injective, then the upper row is exact iff the lower row is.
See ShortComplex.exact_iff_of_epi_of_isIso_of_mono
in the file
Algebra.Homology.ShortComplex.Exact
for the categorical version of this result.
The linear equivalence (N ⧸ LinearMap.range f) ≃ₗ[A] P
associated to
an exact sequence M → N → P → 0
of R
-modules.
Equations
- h.linearEquivOfSurjective hg = LinearEquiv.ofBijective ((LinearMap.range f).liftQ g ⋯) ⋯