Skip to content

Commit

Permalink
feat(data/matrix/rank): rank of a matrix is the rank of its column sp…
Browse files Browse the repository at this point in the history
…ace (#18778)

This is a TODO comment in this file left from #10826. Proving the link to the row space is harder, and only easy to prove for `is_R_or_C`; so I've left it for another time.
  • Loading branch information
eric-wieser committed Apr 13, 2023
1 parent 5ac1dab commit 2140728
Showing 1 changed file with 6 additions and 1 deletion.
7 changes: 6 additions & 1 deletion src/data/matrix/rank.lean
Original file line number Diff line number Diff line change
Expand Up @@ -19,7 +19,7 @@ This definition does not depend on the choice of basis, see `matrix.rank_eq_finr
## TODO
* Show that `matrix.rank` is equal to the row-rank and column-rank
* Show that `matrix.rank` is equal to the row-rank, and that `rank Aᵀ = rank A`.
-/

Expand Down Expand Up @@ -110,4 +110,9 @@ lemma rank_le_height [strong_rank_condition R] {m n : ℕ} (A : matrix (fin m) (
A.rank ≤ m :=
A.rank_le_card_height.trans $ (fintype.card_fin m).le

/-- The rank of a matrix is the rank of the space spanned by its columns. -/
lemma rank_eq_finrank_span_cols (A : matrix m n R) :
A.rank = finrank R (submodule.span R (set.range Aᵀ)) :=
by rw [rank, matrix.range_to_lin']

end matrix

0 comments on commit 2140728

Please sign in to comment.