Zulip Chat Archive

Stream: Is there code for X?

Topic: non_zero_eigenvalues_eq_rank_range


Ivรกn Renison (Jun 18 2025 at 07:28):

Hi, do we have something like this?

import Mathlib.Analysis.InnerProductSpace.Spectrum

variable {๐•œ : Type*} [RCLike ๐•œ]
variable {E : Type*} [NormedAddCommGroup E] [InnerProductSpace ๐•œ E] [FiniteDimensional ๐•œ E]
variable {T : E โ†’โ‚—[๐•œ] E}
variable {n : โ„•}

lemma LinearMap.IsSymmetric.non_zero_eigenvalues_eq_rank_range (hT : T.IsSymmetric)
    (hn : Module.finrank ๐•œ E = n) :
    Finset.card {i : Fin n | hT.eigenvalues hn i โ‰  0} = Module.finrank ๐•œ (LinearMap.range T) :=
  sorry

It does not need to be with exactly that statement. Actually, probably there is a better way to state it, maybe using the complement.
And if it is not, do you have some suggestions on how to prove it?


Last updated: Dec 20 2025 at 21:32 UTC