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

Commit ef18740

Browse files
committed
feat(linear_algebra/eigenspace): generalized eigenvectors span the entire space (#4111)
1 parent 4e41445 commit ef18740

File tree

4 files changed

+196
-66
lines changed

4 files changed

+196
-66
lines changed

docs/references.bib

Lines changed: 13 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,19 @@
44
% %
55
%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
66
7+
@book{axler2015,
8+
Author = {Sheldon Axler},
9+
Title = {Linear algebra done right. 3rd ed.},
10+
FJournal = {Undergraduate Texts in Mathematics},
11+
Journal = {Undergraduate Texts Math.},
12+
ISSN = {0172-6056; 2197-5604/e},
13+
Edition = {3rd ed.},
14+
ISBN = {978-3-319-11079-0/hbk; 978-3-319-11080-6/ebook},
15+
Pages = {xvii + 340},
16+
Year = {2015},
17+
Publisher = {Springer},
18+
}
19+
720
@article {MR1167694,
821
AUTHOR = {Blass, Andreas},
922
TITLE = {A game semantics for linear logic},

src/linear_algebra/basic.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1221,6 +1221,10 @@ lemma range_cod_restrict (p : submodule R M) (f : M₂ →ₗ[R] M) (hf) :
12211221
range (cod_restrict p f hf) = comap p.subtype f.range :=
12221222
map_cod_restrict _ _ _ _
12231223

1224+
lemma ker_restrict {p : submodule R M} {f : M →ₗ[R] M} (hf : ∀ x : M, x ∈ p → f x ∈ p) :
1225+
ker (f.restrict hf) = (f.dom_restrict p).ker :=
1226+
by rw [restrict_eq_cod_restrict_dom_restrict, ker_cod_restrict]
1227+
12241228
lemma map_comap_eq (f : M →ₗ[R] M₂) (q : submodule R M₂) :
12251229
map f (comap f q) = range f ⊓ q :=
12261230
le_antisymm (le_inf (map_mono le_top) (map_comap_le _ _)) $

0 commit comments

Comments
 (0)