Eigenvectors and eigenvalues #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines eigenspaces, eigenvalues, and eigenvalues, as well as their generalized counterparts. We follow Axler's approach [Axl15] because it allows us to derive many properties without choosing a basis and without using matrices.
An eigenspace of a linear map f for a scalar μ is the kernel of the map (f - μ • id). The
nonzero elements of an eigenspace are eigenvectors x. They have the property f x = μ • x. If
there are eigenvectors for a scalar μ, the scalar μ is called an eigenvalue.
There is no consensus in the literature whether 0 is an eigenvector. Our definition of
has_eigenvector permits only nonzero vectors. For an eigenvector x that may also be 0, we
write x ∈ f.eigenspace μ.
A generalized eigenspace of a linear map f for a natural number k and a scalar μ is the kernel
of the map (f - μ • id) ^ k. The nonzero elements of a generalized eigenspace are generalized
eigenvectors x. If there are generalized eigenvectors for a natural number k and a scalar μ,
the scalar μ is called a generalized eigenvalue.
The fact that the eigenvalues are the roots of the minimal polynomial is proved in
linear_algebra.eigenspace.minpoly.
The existence of eigenvalues over an algebraically closed field
(and the fact that the generalized eigenspaces then span) is deferred to
linear_algebra.eigenspace.is_alg_closed.
References #
Tags #
eigenspace, eigenvector, eigenvalue, eigen
The submodule eigenspace f μ for a linear map f and a scalar μ consists of all vectors x
such that f x = μ • x. (Def 5.36 of [Axl15])
Equations
- f.eigenspace μ = linear_map.ker (f - ⇑(algebra_map R (module.End R M)) μ)
Instances for module.End.eigenspace
A nonzero element of an eigenspace is an eigenvector. (Def 5.7 of [Axl15])
Equations
- f.has_eigenvector μ x = (x ∈ f.eigenspace μ ∧ x ≠ 0)
A scalar μ is an eigenvalue for a linear map f if there are nonzero vectors x
such that f x = μ • x. (Def 5.5 of [Axl15])
Equations
- f.has_eigenvalue a = (f.eigenspace a ≠ ⊥)
The eigenvalues of the endomorphism f, as a subtype of R.
Equations
- f.eigenvalues = {μ // f.has_eigenvalue μ}
Instances for module.End.eigenvalues
Equations
The eigenspaces of a linear operator form an independent family of subspaces of V. That is,
any eigenspace has trivial intersection with the span of all the other eigenspaces.
Eigenvectors corresponding to distinct eigenvalues of a linear operator are linearly independent. (Lemma 5.10 of [Axl15])
We use the eigenvalues as indexing set to ensure that there is only one eigenvector for each
eigenvalue in the image of xs.
The generalized eigenspace for a linear map f, a scalar μ, and an exponent k ∈ ℕ is the
kernel of (f - μ • id) ^ k. (Def 8.10 of [Axl15]). Furthermore, a generalized eigenspace for
some exponent k is contained in the generalized eigenspace for exponents larger than k.
Equations
- f.generalized_eigenspace μ = {to_fun := λ (k : ℕ), linear_map.ker ((f - ⇑(algebra_map R (module.End R M)) μ) ^ k), monotone' := _}
A nonzero element of a generalized eigenspace is a generalized eigenvector. (Def 8.9 of [Axl15])
Equations
- f.has_generalized_eigenvector μ k x = (x ≠ 0 ∧ x ∈ ⇑(f.generalized_eigenspace μ) k)
A scalar μ is a generalized eigenvalue for a linear map f and an exponent k ∈ ℕ if there
are generalized eigenvectors for f, k, and μ.
Equations
- f.has_generalized_eigenvalue μ k = (⇑(f.generalized_eigenspace μ) k ≠ ⊥)
The generalized eigenrange for a linear map f, a scalar μ, and an exponent k ∈ ℕ is the
range of (f - μ • id) ^ k.
Equations
- f.generalized_eigenrange μ k = linear_map.range ((f - ⇑(algebra_map R (module.End R M)) μ) ^ k)
The exponent of a generalized eigenvalue is never 0.
The union of the kernels of (f - μ • id) ^ k over all k.
Equations
- f.maximal_generalized_eigenspace μ = ⨆ (k : ℕ), ⇑(f.generalized_eigenspace μ) k
If there exists a natural number k such that the kernel of (f - μ • id) ^ k is the
maximal generalized eigenspace, then this value is the least such k. If not, this value is not
meaningful.
Equations
For an endomorphism of a Noetherian module, the maximal eigenspace is always of the form kernel
(f - μ • id) ^ k for some k.
A generalized eigenvalue for some exponent k is also
a generalized eigenvalue for exponents larger than k.
The eigenspace is a subspace of the generalized eigenspace.
All eigenvalues are generalized eigenvalues.
All generalized eigenvalues are eigenvalues.
Generalized eigenvalues are actually just eigenvalues.
Every generalized eigenvector is a generalized eigenvector for exponent finrank K V.
(Lemma 8.11 of [Axl15])
Generalized eigenspaces for exponents at least finrank K V are equal to each other.
If f maps a subspace p into itself, then the generalized eigenspace of the restriction
of f to p is the part of the generalized eigenspace of f that lies in p.
If p is an invariant submodule of an endomorphism f, then the μ-eigenspace of the
restriction of f to p is a submodule of the μ-eigenspace of f.
Generalized eigenrange and generalized eigenspace for exponent finrank K V are disjoint.
If an invariant subspace p of an endomorphism f is disjoint from the μ-eigenspace of f,
then the restriction of f to p has trivial μ-eigenspace.
The generalized eigenspace of an eigenvalue has positive dimension for positive exponents.
A linear map maps a generalized eigenrange into itself.