Continuous functional calculus #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we construct the continuous_functional_calculus
for a normal element a
of a
(unital) C⋆-algebra over ℂ
. This is a star algebra equivalence
C(spectrum ℂ a, ℂ) ≃⋆ₐ[ℂ] elemental_star_algebra ℂ a
which sends the (restriction of) the
identity map continuous_map.id ℂ
to the (unique) preimage of a
under the coercion of
elemental_star_algebra ℂ a
to A
.
Being a star algebra equivalence between C⋆-algebras, this map is continuous (even an isometry),
and by the Stone-Weierstrass theorem it is the unique star algebra equivalence which extends the
polynomial functional calculus (i.e., polynomial.aeval
).
For any continuous function f : spectrum ℂ a → ℂ
, this makes it possible to define an element
f a
(not valid notation) in the original algebra, which heuristically has the same eigenspaces as
a
and acts on eigenvector of a
for an eigenvalue λ
as multiplication by f λ
. This
description is perfectly accurate in finite dimension, but only heuristic in infinite dimension as
there might be no genuine eigenvector. In particular, when f
is a polynomial ∑ cᵢ Xⁱ
, then
f a
is ∑ cᵢ aⁱ
. Also, id a = a
.
This file also includes a proof of the spectral permanence theorem for (unital) C⋆-algebras
(see star_subalgebra.spectrum_eq
)
Main definitions #
continuous_functional_calculus : C(spectrum ℂ a, ℂ) ≃⋆ₐ[ℂ] elemental_star_algebra ℂ a
: this is the composition of the inverse of thegelfand_star_transform
with the natural isomorphism induced by the homeomorphismelemental_star_algebra.character_space_homeo
.elemental_star_algebra.character_space_homeo :
character_space ℂ (elemental_star_algebra ℂ a) ≃ₜ spectrum ℂ a: this homeomorphism is defined by evaluating a character
φat
a, and noting that
φ a ∈ spectrum ℂ asince
φ` is an algebra homomorphism. Moreover, this map is continuous and bijective and since the spaces involved are compact Hausdorff, it is a homeomorphism.
Main statements #
star_subalgebra.coe_is_unit
: forx : S
in a C⋆-subalgebraS
ofA
, then↑x : A
is a unit if and only ifx
is a unit.star_subalgebra.spectrum_eq
: spectral_permanence forx : S
, whereS
is a C⋆-subalgebra ofA
,spectrum ℂ x = spectrum ℂ (x : A)
.
Notes #
The result we have established here is the strongest possible, but it is likely not the version which will be most useful in practice. Future work will include developing an appropriate API for the continuous functional calculus (including one for real-valued functions with real argument that applies to self-adjoint elements of the algebra).
Equations
- elemental_star_algebra.normed_comm_ring a = {to_normed_ring := {to_has_norm := normed_ring.to_has_norm (subring_class.to_normed_ring (elemental_star_algebra R a)), to_ring := normed_ring.to_ring (subring_class.to_normed_ring (elemental_star_algebra R a)), to_metric_space := normed_ring.to_metric_space (subring_class.to_normed_ring (elemental_star_algebra R a)), dist_eq := _, norm_mul := _}, mul_comm := _}
Equations
This lemma is used in the proof of star_subalgebra.is_unit_of_is_unit_of_is_star_normal
,
which in turn is the key to spectral permanence star_subalgebra.spectrum_eq
, which is itself
necessary for the continuous functional calculus. Using the continuous functional calculus, this
lemma can be superseded by one that omits the is_star_normal
hypothesis.
This is the key lemma on the way to establishing spectral permanence for C⋆-algebras, which is
established in star_subalgebra.spectrum_eq
. This lemma is superseded by
star_subalgebra.coe_is_unit
, which does not require an is_star_normal
hypothesis and holds for
any closed star subalgebra.
For x : A
which is invertible in A
, the inverse lies in any unital C⋆-subalgebra S
containing x
.
For a unital C⋆-subalgebra S
of A
and x : S
, if ↑x : A
is invertible in A
, then
x
is invertible in S
.
Spectral permanence. The spectrum of an element is invariant of the (closed)
star_subalgebra
in which it is contained.
The natural map from character_space ℂ (elemental_star_algebra ℂ x)
to spectrum ℂ x
given
by evaluating φ
at x
. This is essentially just evaluation of the gelfand_transform
of x
,
but because we want something in spectrum ℂ x
, as opposed to
spectrum ℂ ⟨x, elemental_star_algebra.self_mem ℂ x⟩
there is slightly more work to do.
Equations
- elemental_star_algebra.character_space_to_spectrum x φ = ⟨⇑φ ⟨x, _⟩, _⟩
The homeomorphism between the character space of the unital C⋆-subalgebra generated by a
single normal element a : A
and spectrum ℂ a
.
Continuous functional calculus. Given a normal element a : A
of a unital C⋆-algebra,
the continuous functional calculus is a star_alg_equiv
from the complex-valued continuous
functions on the spectrum of a
to the unital C⋆-subalgebra generated by a
. Moreover, this
equivalence identifies (continuous_map.id ℂ).restrict (spectrum ℂ a))
with a
; see
continuous_functional_calculus_map_id
. As such it extends the polynomial functional calculus.