Documentation

Mathlib.Analysis.CStarAlgebra.Spectrum

Spectral properties in C⋆-algebras #

In this file, we establish various properties related to the spectrum of elements in C⋆-algebras. In particular, we show that the spectrum of a unitary element is contained in the unit circle in , the spectrum of a selfadjoint element is real, the spectral radius of a selfadjoint element or normal element is its norm, among others.

An essential feature of C⋆-algebras is spectral permanence. This is the property that the spectrum of an element in a closed subalgebra is the same as the spectrum of the element in the whole algebra. For Banach algebras more generally, and even for Banach ⋆-algebras, this fails.

A consequence of spectral permanence is that one may always enlarge the C⋆-algebra (via a unital embedding) while preserving the spectrum of any element. In addition, it allows us to make sense of the spectrum of elements in non-unital C⋆-algebras by considering them as elements in the Unitization of the C⋆-algebra, or indeed any unital C⋆-algebra. Of course, one may do this (that is, consider the spectrum of an element in a non-unital by embedding it in a unital algebra) for any Banach algebra, but the downside in that setting is that embedding in different unital algebras results in varying spectra.

In Mathlib, we don't define the spectrum of an element in a non-unital C⋆-algebra, and instead simply consider the quasispectrum so as to avoid depending on a choice of unital algebra. However, we can still establish a form of spectral permanence.

Main statements #

TODO #

theorem unitary.spectrum_subset_circle {𝕜 : Type u_1} [NormedField 𝕜] {E : Type u_2} [NormedRing E] [StarRing E] [CStarRing E] [NormedAlgebra 𝕜 E] [CompleteSpace E] (u : { x : E // x unitary E }) :
spectrum 𝕜 u Metric.sphere 0 1
theorem spectrum.subset_circle_of_unitary {𝕜 : Type u_1} [NormedField 𝕜] {E : Type u_2} [NormedRing E] [StarRing E] [CStarRing E] [NormedAlgebra 𝕜 E] [CompleteSpace E] {u : E} (h : u unitary E) :

In a C⋆-algebra, the spectral radius of a self-adjoint element is equal to its norm. See IsSelfAdjoint.toReal_spectralRadius_eq_norm for a version involving spectralRadius ℝ a.

theorem IsSelfAdjoint.mem_spectrum_eq_re {A : Type u_1} [NormedRing A] [NormedAlgebra A] [CompleteSpace A] [StarRing A] [CStarRing A] [StarModule A] {a : A} (ha : IsSelfAdjoint a) {z : } (hz : z spectrum a) :
z = z.re

Any element of the spectrum of a selfadjoint is real.

theorem selfAdjoint.mem_spectrum_eq_re {A : Type u_1} [NormedRing A] [NormedAlgebra A] [CompleteSpace A] [StarRing A] [CStarRing A] [StarModule A] (a : { x : A // x selfAdjoint A }) {z : } (hz : z spectrum a) :
z = z.re

Any element of the spectrum of a selfadjoint is real.

theorem IsSelfAdjoint.im_eq_zero_of_mem_spectrum {A : Type u_1} [NormedRing A] [NormedAlgebra A] [CompleteSpace A] [StarRing A] [CStarRing A] [StarModule A] {a : A} (ha : IsSelfAdjoint a) {z : } (hz : z spectrum a) :
z.im = 0

Any element of the spectrum of a selfadjoint is real.

The spectrum of a selfadjoint is real

The spectrum of a selfadjoint is real

The complement of the spectrum of a selfadjoint element in a C⋆-algebra is connected.

theorem StarSubalgebra.coe_isUnit {A : Type u_1} [NormedRing A] [NormedAlgebra A] [CompleteSpace A] [StarRing A] [CStarRing A] [StarModule A] (S : StarSubalgebra A) [hS : IsClosed S] {a : { x : A // x S }} :

For a unital C⋆-subalgebra S of A and x : S, if ↑x : A is invertible in A, then x is invertible in S.

theorem StarSubalgebra.mem_spectrum_iff {A : Type u_1} [NormedRing A] [NormedAlgebra A] [CompleteSpace A] [StarRing A] [CStarRing A] [StarModule A] (S : StarSubalgebra A) [hS : IsClosed S] {a : { x : A // x S }} {z : } :
theorem StarSubalgebra.spectrum_eq {A : Type u_1} [NormedRing A] [NormedAlgebra A] [CompleteSpace A] [StarRing A] [CStarRing A] [StarModule A] (S : StarSubalgebra A) [hS : IsClosed S] {a : { x : A // x S }} :

Spectral permanence. The spectrum of an element is invariant of the (closed) StarSubalgebra in which it is contained.

A non-unital star algebra homomorphism of complex C⋆-algebras is norm contractive.

A non-unital star algebra homomorphism of complex C⋆-algebras is norm contractive.

Non-unital star algebra homomorphisms between C⋆-algebras are continuous linear maps. See note [lower instance priority]

@[instance 100]
noncomputable instance WeakDual.Complex.instStarHomClass {F : Type u_1} {A : Type u_2} [NormedRing A] [NormedAlgebra A] [CompleteSpace A] [StarRing A] [CStarRing A] [StarModule A] [FunLike F A ] [hF : AlgHomClass F A ] :

This instance is provided instead of StarHomClass to avoid type class inference loops. See note [lower instance priority]

Equations
  • =

This is not an instance to avoid type class inference loops. See WeakDual.Complex.instStarHomClass.