Zulip Chat Archive
Stream: Is there code for X?
Topic: Eigenspaces of diagonalizable maps
Andrew Yang (Feb 21 2025 at 04:53):
Do we have the description of eigenspaces of a diagonalizable map?
Concretely:
import Mathlib
variable {K V : Type*} [Field K] [AddCommGroup V] [Module K V]
variable {ι : Type*} [DecidableEq ι] [Fintype ι] (b : Basis ι K V)
variable (μ : ι → K) (f : Module.End K V) (H : ∀ i, f.HasEigenvector (μ i) (b i))
example (l : K) : f.eigenspace l =
(Finsupp.supported K _ { j | μ j = l }).comap b.repr := sorry
Last updated: May 02 2025 at 03:31 UTC