Skip to content

Commit

Permalink
feat(linear_algebra/eigenspace): generalized eigenvectors span the en…
Browse files Browse the repository at this point in the history
…tire space (#4111)
  • Loading branch information
abentkamp committed Sep 24, 2020
1 parent 4e41445 commit ef18740
Show file tree
Hide file tree
Showing 4 changed files with 196 additions and 66 deletions.
13 changes: 13 additions & 0 deletions docs/references.bib
Expand Up @@ -4,6 +4,19 @@
% %
%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
@book{axler2015,
Author = {Sheldon Axler},
Title = {Linear algebra done right. 3rd ed.},
FJournal = {Undergraduate Texts in Mathematics},
Journal = {Undergraduate Texts Math.},
ISSN = {0172-6056; 2197-5604/e},
Edition = {3rd ed.},
ISBN = {978-3-319-11079-0/hbk; 978-3-319-11080-6/ebook},
Pages = {xvii + 340},
Year = {2015},
Publisher = {Springer},
}

@article {MR1167694,
AUTHOR = {Blass, Andreas},
TITLE = {A game semantics for linear logic},
Expand Down
4 changes: 4 additions & 0 deletions src/linear_algebra/basic.lean
Expand Up @@ -1221,6 +1221,10 @@ lemma range_cod_restrict (p : submodule R M) (f : M₂ →ₗ[R] M) (hf) :
range (cod_restrict p f hf) = comap p.subtype f.range :=
map_cod_restrict _ _ _ _

lemma ker_restrict {p : submodule R M} {f : M →ₗ[R] M} (hf : ∀ x : M, x ∈ p → f x ∈ p) :
ker (f.restrict hf) = (f.dom_restrict p).ker :=
by rw [restrict_eq_cod_restrict_dom_restrict, ker_cod_restrict]

lemma map_comap_eq (f : M →ₗ[R] M₂) (q : submodule R M₂) :
map f (comap f q) = range f ⊓ q :=
le_antisymm (le_inf (map_mono le_top) (map_comap_le _ _)) $
Expand Down

0 comments on commit ef18740

Please sign in to comment.