Zulip Chat Archive

Stream: new members

Topic: simple linear algebra


Monica Omar (Jan 18 2023 at 20:02):

I'm currently stuck on this one problem. Any help would be appreciated!

import analysis.inner_product_space.spectrum

open_locale big_operators
lemma hi {n : } {V : Type*} [inner_product_space  V]  [finite_dimensional  V] (T : V →ₗ[] V) (x : V)
  (hT : T.is_symmetric) (hn : finite_dimensional.finrank  V = n) (h :  i, 0  hT.eigenvalues hn i) :
  0   i : fin n, (real.sqrt (hT.eigenvalues hn i)  (x, hT.eigenvector_basis hn i_ℂ * hT.eigenvector_basis hn i, x_ℂ)).re := sorry

Ruben Van de Velde (Jan 18 2023 at 20:06):

Start with docs#finset.sum_nonneg?

Eric Wieser (Jan 18 2023 at 20:11):

 simp_rw [inner_conj_sym x, complex.norm_sq_eq_conj_mul_self, complex.smul_re,
    complex.of_real_re, smul_eq_mul],

makes some good progress, then it's a trivial inequality


Last updated: Dec 20 2023 at 11:08 UTC