Documentation

Mathlib.MeasureTheory.Constructions.Polish

The Borel sigma-algebra on Polish spaces #

We discuss several results pertaining to the relationship between the topology and the Borel structure on Polish spaces.

Main definitions and results #

First, we define the class of analytic sets and establish its basic properties.

Then, we show Lusin's theorem that two disjoint analytic sets can be separated by Borel sets.

We then prove the Lusin-Souslin theorem that a continuous injective image of a Borel subset of a Polish space is Borel. The proof of this nontrivial result relies on the above results on analytic sets.

We use this to prove several versions of the Borel isomorphism theorem.

Analytic sets #

@[irreducible]

An analytic set is a set which is the continuous image of some Polish space. There are several equivalent characterizations of this definition. For the definition, we pick one that avoids universe issues: a set is analytic if and only if it is a continuous image of ℕ → ℕ (or if it is empty). The above more usual characterization is given in analyticSet_iff_exists_polishSpace_range.

Warning: these are analytic sets in the context of descriptive set theory (which is why they are registered in the namespace MeasureTheory). They have nothing to do with analytic sets in the context of complex analysis.

Instances For
    theorem IsOpen.analyticSet_image {α : Type u_1} [TopologicalSpace α] {β : Type u_3} [TopologicalSpace β] [PolishSpace β] {s : Set β} (hs : IsOpen s) {f : βα} (f_cont : Continuous f) :

    The image of an open set under a continuous map is analytic.

    A set is analytic if and only if it is the continuous image of some Polish space.

    The continuous image of an analytic set is analytic

    theorem MeasureTheory.AnalyticSet.iInter {α : Type u_1} [TopologicalSpace α] {ι : Type u_2} [hι : Nonempty ι] [Countable ι] [T2Space α] {s : ιSet α} (hs : ∀ (n : ι), MeasureTheory.AnalyticSet (s n)) :
    MeasureTheory.AnalyticSet (⋂ (n : ι), s n)

    A countable intersection of analytic sets is analytic.

    theorem MeasureTheory.AnalyticSet.iUnion {α : Type u_1} [TopologicalSpace α] {ι : Type u_2} [Countable ι] {s : ιSet α} (hs : ∀ (n : ι), MeasureTheory.AnalyticSet (s n)) :
    MeasureTheory.AnalyticSet (⋃ (n : ι), s n)

    A countable union of analytic sets is analytic.

    Given a Borel-measurable set in a Polish space, there exists a finer Polish topology making it clopen. This is in fact an equivalence, see isClopenable_iff_measurableSet.

    Given a Borel-measurable function from a Polish space to a second-countable space, there exists a finer Polish topology on the source space for which the function is continuous.

    The image of a measurable set in a Polish space under a measurable map is an analytic set.

    Separating sets with measurable sets #

    def MeasureTheory.MeasurablySeparable {α : Type u_3} [MeasurableSpace α] (s : Set α) (t : Set α) :

    Two sets u and v in a measurable space are measurably separable if there exists a measurable set containing u and disjoint from v. This is mostly interesting for Borel-separable sets.

    Instances For
      theorem MeasureTheory.MeasurablySeparable.iUnion {ι : Type u_2} [Countable ι] {α : Type u_3} [MeasurableSpace α] {s : ιSet α} {t : ιSet α} (h : ∀ (m n : ι), MeasureTheory.MeasurablySeparable (s m) (t n)) :
      MeasureTheory.MeasurablySeparable (⋃ (n : ι), s n) (⋃ (m : ι), t m)

      The hard part of the Lusin separation theorem saying that two disjoint analytic sets are contained in disjoint Borel sets (see the full statement in AnalyticSet.measurablySeparable). Here, we prove this when our analytic sets are the ranges of functions from ℕ → ℕ.

      The Lusin separation theorem: if two analytic sets are disjoint, then they are contained in disjoint Borel sets.

      Suslin's Theorem: in a Hausdorff topological space, an analytic set with an analytic complement is measurable.

      Measurability of preimages under measurable maps #

      If f : X → Y is a surjective Borel measurable map from a Polish space to a topological space with second countable topology, then the preimage of a set s is measurable if and only if the set is measurable. One implication is the definition of measurability, the other one heavily relies on X being a Polish space.

      If f : X → Y is a Borel measurable map from a Polish space to a topological space with second countable topology, then the preimage of a set s is measurable if and only if the set is measurable in Set.range f.

      If f : X → Y is a Borel measurable map from a Polish space to a topological space with second countable topology and the range of f is measurable, then the preimage of a set s is measurable if and only if the intesection with Set.range f is measurable.

      If f : X → Y is a Borel measurable map from a Polish space to a topological space with second countable topology, then for any measurable space β and g : Y → β, the composition g ∘ f is measurable if and only if the restriction of g to the range of f is measurable.

      If f : X → Y is a surjective Borel measurable map from a Polish space to a topological space with second countable topology, then for any measurable space α and g : Y → α, the composition g ∘ f is measurable if and only if g is measurable.

      Injective images of Borel sets #

      The Lusin-Souslin theorem: the range of a continuous injective function defined on a Polish space is Borel-measurable.

      theorem IsClosed.measurableSet_image_of_continuousOn_injOn {γ : Type u_3} [tγ : TopologicalSpace γ] [PolishSpace γ] {β : Type u_4} [TopologicalSpace β] [T2Space β] [MeasurableSpace β] [BorelSpace β] {s : Set γ} (hs : IsClosed s) {f : γβ} (f_cont : ContinuousOn f s) (f_inj : Set.InjOn f s) :
      theorem MeasurableSet.image_of_continuousOn_injOn {γ : Type u_3} [tγ : TopologicalSpace γ] [PolishSpace γ] [MeasurableSpace γ] [hγb : BorelSpace γ] {β : Type u_4} [tβ : TopologicalSpace β] [T2Space β] [MeasurableSpace β] [BorelSpace β] {s : Set γ} {f : γβ} (hs : MeasurableSet s) (f_cont : ContinuousOn f s) (f_inj : Set.InjOn f s) :

      The Lusin-Souslin theorem: if s is Borel-measurable in a Polish space, then its image under a continuous injective map is also Borel-measurable.

      theorem MeasurableSet.image_of_measurable_injOn {γ : Type u_3} [tγ : TopologicalSpace γ] [PolishSpace γ] [MeasurableSpace γ] [hγb : BorelSpace γ] {β : Type u_4} [tβ : TopologicalSpace β] [T2Space β] [MeasurableSpace β] [BorelSpace β] {s : Set γ} {f : γβ} [TopologicalSpace.SecondCountableTopology β] (hs : MeasurableSet s) (f_meas : Measurable f) (f_inj : Set.InjOn f s) :

      The Lusin-Souslin theorem: if s is Borel-measurable in a Polish space, then its image under a measurable injective map taking values in a second-countable topological space is also Borel-measurable.

      theorem Continuous.measurableEmbedding {γ : Type u_3} [tγ : TopologicalSpace γ] [PolishSpace γ] [MeasurableSpace γ] [hγb : BorelSpace γ] {β : Type u_4} [tβ : TopologicalSpace β] [T2Space β] [MeasurableSpace β] [BorelSpace β] {f : γβ} (f_cont : Continuous f) (f_inj : Function.Injective f) :

      An injective continuous function on a Polish space is a measurable embedding.

      theorem ContinuousOn.measurableEmbedding {γ : Type u_3} [tγ : TopologicalSpace γ] [PolishSpace γ] [MeasurableSpace γ] [hγb : BorelSpace γ] {β : Type u_4} [tβ : TopologicalSpace β] [T2Space β] [MeasurableSpace β] [BorelSpace β] {s : Set γ} {f : γβ} (hs : MeasurableSet s) (f_cont : ContinuousOn f s) (f_inj : Set.InjOn f s) :

      If s is Borel-measurable in a Polish space and f is continuous injective on s, then the restriction of f to s is a measurable embedding.

      theorem Measurable.measurableEmbedding {γ : Type u_3} [tγ : TopologicalSpace γ] [PolishSpace γ] [MeasurableSpace γ] [hγb : BorelSpace γ] {β : Type u_4} [tβ : TopologicalSpace β] [T2Space β] [MeasurableSpace β] [BorelSpace β] {f : γβ} [TopologicalSpace.SecondCountableTopology β] (f_meas : Measurable f) (f_inj : Function.Injective f) :

      An injective measurable function from a Polish space to a second-countable topological space is a measurable embedding.

      In a Polish space, a set is clopenable if and only if it is Borel-measurable.

      theorem MeasureTheory.measurableSet_exists_tendsto {ι : Type u_2} {γ : Type u_3} [tγ : TopologicalSpace γ] [PolishSpace γ] [MeasurableSpace γ] {β : Type u_4} [MeasurableSpace β] [hγ : OpensMeasurableSpace γ] [Countable ι] {l : Filter ι} [Filter.IsCountablyGenerated l] {f : ιβγ} (hf : ∀ (i : ι), Measurable (f i)) :
      MeasurableSet {x | c, Filter.Tendsto (fun n => f n x) l (nhds c)}

      The set of points for which a measurable sequence of functions converges is measurable.

      The Borel Isomorphism Theorem #

      noncomputable def PolishSpace.borelSchroederBernstein {α : Type u_1} [TopologicalSpace α] {β : Type u_3} [TopologicalSpace β] [PolishSpace α] [PolishSpace β] [MeasurableSpace α] [MeasurableSpace β] [BorelSpace α] [BorelSpace β] {f : αβ} {g : βα} (fmeas : Measurable f) (finj : Function.Injective f) (gmeas : Measurable g) (ginj : Function.Injective g) :
      α ≃ᵐ β

      If two Polish spaces admit Borel measurable injections to one another, then they are Borel isomorphic.

      Instances For

        Any uncountable Polish space is Borel isomorphic to the Cantor space ℕ → Bool.

        Instances For
          noncomputable def PolishSpace.measurableEquivOfNotCountable {α : Type u_1} [TopologicalSpace α] {β : Type u_3} [TopologicalSpace β] [PolishSpace α] [PolishSpace β] [MeasurableSpace α] [MeasurableSpace β] [BorelSpace α] [BorelSpace β] (hα : ¬Countable α) (hβ : ¬Countable β) :
          α ≃ᵐ β

          The Borel Isomorphism Theorem: Any two uncountable Polish spaces are Borel isomorphic.

          Instances For
            noncomputable def PolishSpace.Equiv.measurableEquiv {α : Type u_1} [TopologicalSpace α] {β : Type u_3} [TopologicalSpace β] [PolishSpace α] [PolishSpace β] [MeasurableSpace α] [MeasurableSpace β] [BorelSpace α] [BorelSpace β] (e : α β) :
            α ≃ᵐ β

            The Borel Isomorphism Theorem: If two Polish spaces have the same cardinality, they are Borel isomorphic.

            Instances For

              Any Polish Borel space is measurably equivalent to a subset of the reals.

              Any Polish Borel space embeds measurably into the reals.