Skip to content

Commit

Permalink
doc(linear_algebra/finite_dimensional): update doc to new definition (#…
Browse files Browse the repository at this point in the history
…10758)

`finite_dimensional` is now (since a couple of months) defined to be `module.finite`. The lines modified by this PR are about the old definition.
  • Loading branch information
riccardobrasca committed Dec 13, 2021
1 parent 108eb0b commit ee8de4c
Showing 1 changed file with 2 additions and 5 deletions.
7 changes: 2 additions & 5 deletions src/linear_algebra/finite_dimensional.lean
Expand Up @@ -77,9 +77,8 @@ open_locale classical cardinal

open cardinal submodule module function

/-- `finite_dimensional` vector spaces are defined to be noetherian modules.
Use `finite_dimensional.iff_fg` or `finite_dimensional.of_fintype_basis` to prove finite dimension
from another definition. -/
/-- `finite_dimensional` vector spaces are defined to be finite modules.
Use `finite_dimensional.of_fintype_basis` to prove finite dimension from another definition. -/
@[reducible] def finite_dimensional (K V : Type*) [division_ring K]
[add_comm_group V] [module K V] := module.finite K V

Expand All @@ -94,8 +93,6 @@ variables (K : Type u) (V : Type v) [division_ring K] [add_comm_group V] [module

variables (K V)

-- Without this apparently redundant instance we get typeclass search errors
-- in `analysis.normed_space.finite_dimension`.
instance finite_dimensional_pi {ι} [fintype ι] : finite_dimensional K (ι → K) :=
iff_fg.1 is_noetherian_pi

Expand Down

0 comments on commit ee8de4c

Please sign in to comment.