Ideals of continuous functions #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
For a topological semiring R and a topological space X there is a Galois connection between
ideal C(X, R) and set X given by sending each I : ideal C(X, R) to
{x : X | ∀ f ∈ I, f x = 0}ᶜ and mapping s : set X to the ideal with carrier
{f : C(X, R) | ∀ x ∈ sᶜ, f x = 0}, and we call these maps continuous_map.set_of_ideal and
continuous_map.ideal_of_set. As long as R is Hausdorff, continuous_map.set_of_ideal I is open,
and if, in addition, X is locally compact, then continuous_map.set_of_ideal s is closed.
When R = 𝕜 with is_R_or_C 𝕜 and X is compact Hausdorff, then this Galois connection can be
improved to a true Galois correspondence (i.e., order isomorphism) between the type opens X and
the subtype of closed ideals of C(X, 𝕜). Because we do not have a bundled type of closed ideals,
we simply register this as a Galois insertion between ideal C(X, 𝕜) and opens X, which is
continuous_map.ideal_opens_gi. Consequently, the maximal ideals of C(X, 𝕜) are precisely those
ideals corresponding to (complements of) singletons in X.
In addition, when X is locally compact and 𝕜 is a nontrivial topological integral domain, then
there is a natural continuous map from X to character_space 𝕜 C(X, 𝕜) given by point evaluation,
which is herein called weak_dual.character_space.continuous_map_eval. Again, when X is compact
Hausdorff and is_R_or_C 𝕜, more can be obtained. In particular, in that context this map is
bijective, and since the domain is compact and the codomain is Hausdorff, it is a homeomorphism,
herein called weak_dual.character_space.homeo_eval.
Main definitions #
continuous_map.ideal_of_set: ideal of functions which vanish on the complement of a set.continuous_map.set_of_ideal: complement of the set on which all functions in the ideal vanish.continuous_map.opens_of_ideal:continuous_map.set_of_idealas a term ofopens X.continuous_map.ideal_opens_gi: The Galois insertioncontinuous_map.opens_of_idealandλ s, continuous_map.ideal_of_set ↑s.weak_dual.character_space.continuous_map_eval: the natural continuous map from a locally compact topological spaceXto thecharacter_space 𝕜 C(X, 𝕜)which sendsx : Xto point evaluation atx, with modest hypothesis on𝕜.weak_dual.character_space.homeo_eval: this isweak_dual.character_space.continuous_map_evalupgraded to a homeomorphism whenXis compact Hausdorff andis_R_or_C 𝕜.
Main statements #
continuous_map.ideal_of_set_of_ideal_eq_closure: whenXis compact Hausdorff andis_R_or_C 𝕜,ideal_of_set 𝕜 (set_of_ideal I) = I.closurefor any idealI : ideal C(X, 𝕜).continuous_map.set_of_ideal_of_set_eq_interior: whenXis compact Hausdorff andis_R_or_C 𝕜,set_of_ideal (ideal_of_set 𝕜 s) = interior sfor anys : set X.continuous_map.ideal_is_maximal_iff: whenXis compact Hausdorff andis_R_or_C 𝕜, a closed ideal ofC(X, 𝕜)is maximal if and only if it isideal_of_set 𝕜 {x}ᶜfor somex : X.
Implementation details #
Because there does not currently exist a bundled type of closed ideals, we don't provide the actual
order isomorphism described above, and instead we only consider the Galois insertion
continuous_map.ideal_opens_gi.
Tags #
ideal, continuous function, compact, Hausdorff
Given a topological ring R and s : set X, construct the ideal in C(X, R) of functions
which vanish on the complement of s.
Given an ideal I of C(X, R), construct the set of points for which every function in the
ideal vanishes on the complement.
The open set set_of_ideal I realized as a term of opens X.
Equations
An auxiliary lemma used in the proof of ideal_of_set_of_ideal_eq_closure which may be useful
on its own.
The Galois insertion continuous_map.opens_of_ideal : ideal C(X, 𝕜) → opens X and
λ s, continuous_map.ideal_of_set ↑s.
Equations
- continuous_map.ideal_opens_gi X 𝕜 = {choice := λ (I : ideal C(X, 𝕜)) (hI : continuous_map.ideal_of_set 𝕜 ↑(continuous_map.opens_of_ideal I) ≤ I), continuous_map.opens_of_ideal I.closure, gc := _, le_l_u := _, choice_eq := _}
The natural continuous map from a locally compact topological space X to the
character_space 𝕜 C(X, 𝕜) which sends x : X to point evaluation at x.
This is the natural homeomorphism between a compact Hausdorff space X and the
character_space 𝕜 C(X, 𝕜).