Documentation

Mathlib.LinearAlgebra.Matrix.HermitianFunctionalCalculus

Continuous Functional Calculus for Hermitian Matrices #

This file defines an instance of the continuous functional calculus for Hermitian matrices over an RCLike field 𝕜.

Main Results #

Tags #

spectral theorem, diagonalization theorem, continuous functional calculus

theorem Matrix.finite_real_spectrum {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {A : Matrix n n 𝕜} :
(spectrum A).Finite
instance Matrix.instFiniteElemRealSpectrum {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {A : Matrix n n 𝕜} :
Equations
  • =
theorem Matrix.IsHermitian.eigenvalues_eq_spectrum_real {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {a : Matrix n n 𝕜} (ha : a.IsHermitian) :
spectrum a = Set.range ha.eigenvalues

The -spectrum of a Hermitian matrix over RCLike field is the range of the eigenvalue function

@[simp]
theorem Matrix.IsHermitian.cfcAux_apply {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {A : Matrix n n 𝕜} (hA : A.IsHermitian) (g : C((spectrum A), )) :
hA.cfcAux g = hA.eigenvectorUnitary * Matrix.diagonal (RCLike.ofReal g fun (i : n) => hA.eigenvalues i, ) * star hA.eigenvectorUnitary
noncomputable def Matrix.IsHermitian.cfcAux {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {A : Matrix n n 𝕜} (hA : A.IsHermitian) :

The star algebra homomorphism underlying the instance of the continuous functional calculus of a Hermitian matrix. This is an auxiliary definition and is not intended for use outside of this file.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem Matrix.IsHermitian.closedEmbedding_cfcAux {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {A : Matrix n n 𝕜} (hA : A.IsHermitian) :
    ClosedEmbedding hA.cfcAux
    theorem Matrix.IsHermitian.cfcAux_id {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {A : Matrix n n 𝕜} (hA : A.IsHermitian) :

    Instance of the continuous functional calculus for a Hermitian matrix over 𝕜 with RCLike 𝕜.

    Equations
    • =
    noncomputable def Matrix.IsHermitian.cfc {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {A : Matrix n n 𝕜} (hA : A.IsHermitian) (f : ) :
    Matrix n n 𝕜

    The continuous functional calculus of a Hermitian matrix as a triple product using the spectral theorem. Note that this actually operates on bare functions since every function is continuous on the spectrum of a matrix, since the spectrum is finite. This is shown to be equal to the generic continuous functional calculus API in Matrix.IsHermitian.cfc_eq. In general, users should prefer the generic API, especially because it will make rewriting easier.

    Equations
    Instances For
      theorem Matrix.IsHermitian.cfc_eq {n : Type u_1} {𝕜 : Type u_2} [RCLike 𝕜] [Fintype n] [DecidableEq n] {A : Matrix n n 𝕜} (hA : A.IsHermitian) (f : ) :
      cfc f A = hA.cfc f