Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 036527a

Browse files
committed
feat(linear_algebra/finite_dimensional): eq_of_le_of_findim_eq (#4005)
Add a variant of `eq_top_of_findim_eq`, where instead of proving a submodule equal to `⊤`, it's shown equal to another finite-dimensional submodule with the same dimension that contains it. The two lemmas are related by the `comap_subtype` lemmas, so the proof is short, but it still seems useful to have this form.
1 parent be3b175 commit 036527a

File tree

1 file changed

+13
-0
lines changed

1 file changed

+13
-0
lines changed

src/linear_algebra/finite_dimensional.lean

Lines changed: 13 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -587,6 +587,19 @@ end
587587

588588
end linear_equiv
589589

590+
namespace finite_dimensional
591+
592+
/-- If a submodule is less than or equal to a finite-dimensional
593+
submodule with the same dimension, they are equal. -/
594+
lemma eq_of_le_of_findim_eq {S₁ S₂ : submodule K V} [finite_dimensional K S₂] (hle : S₁ ≤ S₂)
595+
(hd : findim K S₁ = findim K S₂) : S₁ = S₂ :=
596+
begin
597+
rw ←linear_equiv.findim_eq (submodule.comap_subtype_equiv_of_le hle) at hd,
598+
exact le_antisymm hle (submodule.comap_subtype_eq_top.1 (eq_top_of_findim_eq hd))
599+
end
600+
601+
end finite_dimensional
602+
590603
namespace linear_map
591604
open finite_dimensional
592605

0 commit comments

Comments
 (0)