Gelfand Duality #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
The gelfand_transform
is an algebra homomorphism from a topological 𝕜
-algebra A
to
C(character_space 𝕜 A, 𝕜)
. In the case where A
is a commutative complex Banach algebra, then
the Gelfand transform is actually spectrum-preserving (spectrum.gelfand_transform_eq
). Moreover,
when A
is a commutative C⋆-algebra over ℂ
, then the Gelfand transform is a surjective isometry,
and even an equivalence between C⋆-algebras.
Main definitions #
ideal.to_character_space
: constructs an element of the character space from a maximal ideal in a commutative complex Banach algebraweak_dual.character_space.comp_continuous_map
: The functorial map takingψ : A →⋆ₐ[ℂ] B
to a continuous functioncharacter_space ℂ B → character_space ℂ A
given by pre-composition withψ
.
Main statements #
spectrum.gelfand_transform_eq
: the Gelfand transform is spectrum-preserving when the algebra is a commutative complex Banach algebra.gelfand_transform_isometry
: the Gelfand transform is an isometry when the algebra is a commutative (unital) C⋆-algebra overℂ
.gelfand_transform_bijective
: the Gelfand transform is bijective when the algebra is a commutative (unital) C⋆-algebra overℂ
.
TODO #
- After
star_alg_equiv
is defined, realizegelfand_transform
as astar_alg_equiv
. - Prove that if
A
is the unital C⋆-algebra overℂ
generated by a fixed normal elementx
in a larger C⋆-algebraB
, thencharacter_space ℂ A
is homeomorphic tospectrum ℂ x
. - From the previous result, construct the continuous functional calculus.
- Show that if
X
is a compact Hausdorff space, thenX
is (canonically) homeomorphic tocharacter_space ℂ C(X, ℂ)
. - Conclude using the previous fact that the functors
C(⬝, ℂ)
andcharacter_space ℂ ⬝
along with the canonical homeomorphisms described above constitute a natural contravariant equivalence of the categories of compact Hausdorff spaces (with continuous maps) and commutative unital C⋆-algebras (with unital ⋆-algebra homomoprhisms); this is known as Gelfand duality.
Tags #
Gelfand transform, character space, C⋆-algebra
Every maximal ideal in a commutative complex Banach algebra gives rise to a character on that
algebra. In particular, the character, which may be identified as an algebra homomorphism due to
weak_dual.character_space.equiv_alg_hom
, is given by the composition of the quotient map and
the Gelfand-Mazur isomorphism normed_ring.alg_equiv_complex_of_complete
.
Equations
If a : A
is not a unit, then some character takes the value zero at a
. This is equivlaent
to gelfand_transform ℂ A a
takes the value zero at some character.
The Gelfand transform is spectrum-preserving.
The Gelfand transform is an isometry when the algebra is a C⋆-algebra over ℂ
.
The Gelfand transform is bijective when the algebra is a C⋆-algebra over ℂ
.
The Gelfand transform as a star_alg_equiv
between a commutative unital C⋆-algebra over ℂ
and the continuous functions on its character_space
.
The functorial map taking ψ : A →⋆ₐ[ℂ] B
to a continuous function
character_space ℂ B → character_space ℂ A
obtained by pre-composition with ψ
.
Equations
weak_dual.character_space.comp_continuous_map
sends the identity to the identity.
weak_dual.character_space.comp_continuous_map
is functorial.