Commit 2024-01-01 14:48 0b41ea95
View on Github →chore: Reorganize results about rank
and finrank
. (#9349)
The files Mathlib.LinearAlgebra.FreeModule.Rank
, Mathlib.LinearAlgebra.FreeModule.Finite.Rank
, Mathlib.LinearAlgebra.Dimension
and Mathlib.LinearAlgebra.Finrank
were reorganized into a
folder Mathlib.LinearAlgebra.Dimension
, containing the following files
Basic.lean
: Contains the definition ofModule.rank
.Finrank.lean
: Contains the definition ofFiniteDimensional.finrank
.StrongRankCondition.lean
: Contains results aboutrank
andfinrank
over rings satisfying strong rank conditionFree.lean
: Contains results aboutrank
andfinrank
of free modulesFinite.lean
: Contains conditions or consequences forrank
to be finite or zeroConstructions.lean
: Contains the calculation of therank
of various constructions.DivisionRing.lean
: Contains results aboutrank
andfinrank
of spaces over division rings.LinearMap.lean
: Contains results aboutLinearMap.rank
API changes:IsNoetherian.rank_lt_aleph0
andFiniteDimensional.rank_lt_aleph0
are replaced withrank_lt_aleph0
.Module.Free.finite_basis
was renamed toModule.Finite.finite_basis
.FiniteDimensional.finrank_eq_rank
was renamed tofinrank_eq_rank
.rank_eq_cardinal_basis
andrank_eq_cardinal_basis'
were removed in favour ofBasis.mk_eq_mk
andBasis.mk_eq_mk''
.