Finite dimension of vector spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Definition of the rank of a module, or dimension of a vector space, as a natural number.
Main definitions #
Defined is finite_dimensional.finrank
, the dimension of a finite dimensional space, returning a
nat
, as opposed to module.rank
, which returns a cardinal
. When the space has infinite
dimension, its finrank
is by convention set to 0
.
The definition of finrank
does not assume a finite_dimensional
instance, but lemmas might.
Import linear_algebra.finite_dimensional
to get access to these additional lemmas.
Formulas for the dimension are given for linear equivs, in linear_equiv.finrank_eq
Implementation notes #
Most results are deduced from the corresponding results for the general dimension (as a cardinal),
in dimension.lean
. Not all results have been ported yet.
You should not assume that there has been any effort to state lemmas as generally as possible.
The rank of a module as a natural number.
Defined by convention to be 0
if the space has infinite rank.
For a vector space V
over a field K
, this is the same as the finite dimension
of V
over K
.
Equations
A finite dimensional space is nontrivial if it has positive finrank
.
A finite dimensional space is nontrivial if it has finrank
equal to the successor of a
natural number.
A (finite dimensional) space that is a subsingleton has zero finrank
.
If a vector space (or module) has a finite basis, then its dimension (or rank) is equal to the cardinality of the basis.
If a vector space (or module) has a finite basis, then its dimension (or rank) is equal to the
cardinality of the basis. This lemma uses a finset
instead of indexed types.
A ring satisfying strong_rank_condition
(such as a division_ring
) is one-dimensional as a
module over itself.
The vector space of functions on a fintype ι has finrank equal to the cardinality of ι.
The vector space of functions on fin n
has finrank equal to n
.
The dimension of a finite dimensional space is preserved under linear equivalence.
Pushforwards of finite-dimensional submodules along a linear_equiv
have the same finrank.
The dimensions of the domain and range of an injective linear map are equal.
The rank of a set of vectors as a natural number.
Equations
- set.finrank K s = finite_dimensional.finrank K ↥(submodule.span K s)
A finite family of vectors is linearly independent if and only if its cardinality equals the dimension of its span.
A family of finrank K V
vectors forms a basis if they span the whole space.
Equations
- basis_of_top_le_span_of_card_eq_finrank b le_span card_eq = basis.mk _ le_span
A finset of finrank K V
vectors forms a basis if they span the whole space.
Equations
- finset_basis_of_top_le_span_of_card_eq_finrank le_span card_eq = basis_of_top_le_span_of_card_eq_finrank coe _ _
A set of finrank K V
vectors forms a basis if they span the whole space.
Equations
- set_basis_of_top_le_span_of_card_eq_finrank le_span card_eq = basis_of_top_le_span_of_card_eq_finrank coe _ _
We now give characterisations of finrank K V = 1
and finrank K V ≤ 1
.
If there is a nonzero vector and every other vector is a multiple of it, then the module has dimension one.
If every vector is a multiple of some v : V
, then V
has dimension at most one.