Some results on free modules over rings satisfying strong rank condition #
This file contains some results on free modules over rings satisfying strong rank condition.
Most of them are generalized from the same result assuming the base ring being a division ring,
and are moved from the files Mathlib/LinearAlgebra/Dimension/DivisionRing.lean
and Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean.
The ι indexed basis on V, where ι is an empty type and V is zero-dimensional.
See also Module.finBasis.
Equations
Instances For
A vector space has dimension at most 1 if and only if there is a
single vector of which all vectors are multiples.
A vector space has dimension 1 if and only if there is a
single non-zero vector of which all vectors are multiples.
A submodule has dimension at most 1 if and only if there is a
single vector in the submodule such that the submodule is contained in
its span.
A submodule has dimension 1 if and only if there is a
single non-zero vector in the submodule such that the submodule is contained in
its span.
A submodule has dimension at most 1 if and only if there is a
single vector, not necessarily in the submodule, such that the
submodule is contained in its span.
A module has dimension 1 iff there is some v : V so {v} is a basis.
See also Module.Basis.nonempty_unique_index_of_finrank_eq_one
A module has dimension 1 iff there is some nonzero v : V so every vector is a multiple of v.
A finite-dimensional module has dimension at most 1 iff
there is some v : V so every vector is a multiple of v.
Alias of the reverse direction of Subalgebra.bot_eq_top_iff_rank_eq_one.
Alias of the reverse direction of Subalgebra.bot_eq_top_iff_finrank_eq_one.