Documentation

Mathlib.LinearAlgebra.Eigenspace.Minpoly

Eigenvalues are the roots of the minimal polynomial. #

Tags #

eigenvalue, minimal polynomial

theorem Module.End.aeval_apply_of_hasEigenvector {K : Type v} {V : Type w} [Field K] [AddCommGroup V] [Module K V] {f : Module.End K V} {p : Polynomial K} {μ : K} {x : V} (h : Module.End.HasEigenvector f μ x) :
theorem Module.End.isRoot_of_hasEigenvalue {K : Type v} {V : Type w} [Field K] [AddCommGroup V] [Module K V] {f : Module.End K V} {μ : K} (h : Module.End.HasEigenvalue f μ) :

An endomorphism of a finite-dimensional vector space has finitely many eigenvalues.

Equations