Skip to content

Commit

Permalink
feat(analysis/normed_space/star/gelfand_duality): functoriality of `c…
Browse files Browse the repository at this point in the history
…haracter_space ℂ` (#16835)

This is one of the two contravariant functors involved in Gelfand duality.
  • Loading branch information
j-loreaux committed Oct 14, 2022
1 parent 71429ce commit e0ce218
Showing 1 changed file with 42 additions and 0 deletions.
42 changes: 42 additions & 0 deletions src/analysis/normed_space/star/gelfand_duality.lean
Expand Up @@ -24,6 +24,8 @@ and even an equivalence between C⋆-algebras.
* `ideal.to_character_space` : constructs an element of the character space from a maximal ideal in
a commutative complex Banach algebra
* `weak_dual.character_space.comp_continuous_map`: The functorial map taking `ψ : A →⋆ₐ[ℂ] B` to a
continuous function `character_space ℂ B → character_space ℂ A` given by pre-composition with `ψ`.
## Main statements
Expand Down Expand Up @@ -164,3 +166,43 @@ begin
end

end complex_cstar_algebra

section functoriality

namespace weak_dual

namespace character_space

variables {A B C : Type*}
variables [normed_ring A] [normed_algebra ℂ A] [complete_space A] [star_ring A]
variables [normed_ring B] [normed_algebra ℂ B] [complete_space B] [star_ring B]
variables [normed_ring C] [normed_algebra ℂ C] [complete_space C] [star_ring C]

/-- The functorial map taking `ψ : A →⋆ₐ[ℂ] B` to a continuous function
`character_space ℂ B → character_space ℂ A` obtained by pre-composition with `ψ`. -/
@[simps]
noncomputable def comp_continuous_map (ψ : A →⋆ₐ[ℂ] B) :
C(character_space ℂ B, character_space ℂ A) :=
{ to_fun := λ φ, equiv_alg_hom.symm ((equiv_alg_hom φ).comp (ψ.to_alg_hom)),
continuous_to_fun := continuous.subtype_mk (continuous_of_continuous_eval $
λ a, map_continuous $ gelfand_transform ℂ B (ψ a)) _ }

variables (A)

/-- `weak_dual.character_space.comp_continuous_map` sends the identity to the identity. -/
@[simp] lemma comp_continuous_map_id :
comp_continuous_map (star_alg_hom.id ℂ A) = continuous_map.id (character_space ℂ A) :=
continuous_map.ext $ λ a, ext $ λ x, rfl

variables {A}

/-- `weak_dual.character_space.comp_continuous_map` is functorial. -/
@[simp] lemma comp_continuous_map_comp (ψ₂ : B →⋆ₐ[ℂ] C) (ψ₁ : A →⋆ₐ[ℂ] B) :
comp_continuous_map (ψ₂.comp ψ₁) = (comp_continuous_map ψ₁).comp (comp_continuous_map ψ₂) :=
continuous_map.ext $ λ a, ext $ λ x, rfl

end character_space

end weak_dual

end functoriality

0 comments on commit e0ce218

Please sign in to comment.