Skip to content

Commit

Permalink
Update Mathlib/LinearAlgebra/Basis/Exact.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Andrew Yang <[email protected]>
  • Loading branch information
chrisflav and erdOne authored Jan 7, 2025
1 parent db207ba commit 2a19ed1
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/Basis/Exact.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ import Mathlib.LinearAlgebra.Basis.Basic
/-!
# Basis from a split exact sequence
Let `0 → K → M → P → 0` be an exact sequence of `R`-modules, let `s : M → K` be a
Let `0 → K → M → P → 0` be a split exact sequence of `R`-modules, let `s : M → K` be a
retraction of `f` and `v` be a basis of `M` indexed by `κ ⊕ σ`. Then
if `s vᵢ = 0` for `i : κ` and `(s vⱼ)ⱼ` is linear independent for `j : σ`, then
the images of `vᵢ` for `i : κ` form a basis of `P`.
Expand Down

0 comments on commit 2a19ed1

Please sign in to comment.