Documentation

Mathlib.MeasureTheory.Constructions.BorelSpace.Basic

Borel (measurable) space #

Main definitions #

Main statements #

theorem borel_anti {α : Type u_1} :
theorem borel_comap {α : Type u_1} {β : Type u_2} {f : αβ} {t : TopologicalSpace β} :
theorem Continuous.borel_measurable {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} (hf : Continuous f) :

A space with MeasurableSpace and TopologicalSpace structures such that all open sets are measurable.

  • borel_le : borel α h

    Borel-measurable sets are measurable.

Instances

    A space with MeasurableSpace and TopologicalSpace structures such that the σ-algebra of measurable sets is exactly the σ-algebra generated by open sets.

    • measurable_eq : inst✝ = borel α

      The measurable sets are exactly the Borel-measurable sets.

    Instances

      The behaviour of borelize α depends on the existing assumptions on α.

      Finally, borelize α β γ runs borelize α; borelize β; borelize γ.

      Equations
      • One or more equations did not get rendered due to their size.

      Add instances borel e : MeasurableSpace e and ⟨rfl⟩ : BorelSpace e.

      Equations
      • One or more equations did not get rendered due to their size.

      Given a type e, an assumption i : MeasurableSpace e, and an instance [BorelSpace e], replace i with borel e.

      Equations
      • One or more equations did not get rendered due to their size.

      Given a type $t, if there is an assumption [i : MeasurableSpace $t], then try to prove [BorelSpace $t] and replace i with borel $t. Otherwise, add instances borel $t : MeasurableSpace $t and ⟨rfl⟩ : BorelSpace $t.

      Equations
      • One or more equations did not get rendered due to their size.
      @[instance 100]
      @[instance 100]

      In a BorelSpace all open sets are measurable.

      instance Subtype.borelSpace {α : Type u_6} [TopologicalSpace α] [MeasurableSpace α] [ : BorelSpace α] (s : Set α) :
      theorem MeasurableSet.induction_on_open {γ : Type u_3} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] {C : (s : Set γ) → MeasurableSet sProp} (isOpen : ∀ (U : Set γ) (hU : IsOpen U), C U ) (compl : ∀ (t : Set γ) (ht : MeasurableSet t), C t htC t ) (iUnion : ∀ (f : Set γ), Pairwise (Function.onFun Disjoint f)∀ (hf : ∀ (i : ), MeasurableSet (f i)), (∀ (i : ), C (f i) )C (⋃ (i : ), f i) ) (t : Set γ) (ht : MeasurableSet t) :
      C t ht
      theorem Inseparable.mem_measurableSet_iff {γ : Type u_3} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] {x y : γ} (h : Inseparable x y) {s : Set γ} (hs : MeasurableSet s) :
      x s y s

      If two points are topologically inseparable, then they can't be separated by a Borel measurable set.

      theorem IsCompact.closure_subset_measurableSet {γ : Type u_3} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [R1Space γ] {K s : Set γ} (hK : IsCompact K) (hs : MeasurableSet s) (hKs : K s) :

      If K is a compact set in an R₁ space and s ⊇ K is a Borel measurable superset, then s includes the closure of K as well.

      theorem IsCompact.measure_closure {γ : Type u_3} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [R1Space γ] {K : Set γ} (hK : IsCompact K) (μ : MeasureTheory.Measure γ) :
      μ (closure K) = μ K

      In an R₁ topological space with Borel measure μ, the measure of the closure of a compact set K is equal to the measure of K.

      See also MeasureTheory.Measure.OuterRegular.measure_closure_eq_of_isCompact for a version that assumes μ to be outer regular but does not assume the σ-algebra to be Borel.

      theorem measurable_of_isOpen {γ : Type u_3} {δ : Type u_5} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [MeasurableSpace δ] {f : δγ} (hf : ∀ (s : Set γ), IsOpen sMeasurableSet (f ⁻¹' s)) :
      theorem measurable_of_isClosed {γ : Type u_3} {δ : Type u_5} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [MeasurableSpace δ] {f : δγ} (hf : ∀ (s : Set γ), IsClosed sMeasurableSet (f ⁻¹' s)) :
      theorem measurable_of_isClosed' {γ : Type u_3} {δ : Type u_5} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [MeasurableSpace δ] {f : δγ} (hf : ∀ (s : Set γ), IsClosed ss.Nonemptys Set.univMeasurableSet (f ⁻¹' s)) :

      If s is a measurable set, then 𝓝[s] a is a measurably generated filter for each a. This cannot be an instance because it depends on a non-instance hs : MeasurableSet s.

      instance Pi.opensMeasurableSpace {ι : Type u_6} {X : ιType u_7} [Countable ι] [t' : (i : ι) → TopologicalSpace (X i)] [(i : ι) → MeasurableSpace (X i)] [∀ (i : ι), SecondCountableTopology (X i)] [∀ (i : ι), OpensMeasurableSpace (X i)] :
      OpensMeasurableSpace ((i : ι) → X i)

      The typeclass SecondCountableTopologyEither α β registers the fact that at least one of the two spaces has second countable topology. This is the right assumption to ensure that continuous maps from α to β are strongly measurable.

      Instances

        If either α or β has second-countable topology, then the open sets in α × β belong to the product sigma-algebra.

        theorem interior_ae_eq_of_null_frontier {α' : Type u_6} [TopologicalSpace α'] [MeasurableSpace α'] {μ : MeasureTheory.Measure α'} {s : Set α'} (h : μ (frontier s) = 0) :
        theorem measure_interior_of_null_frontier {α' : Type u_6} [TopologicalSpace α'] [MeasurableSpace α'] {μ : MeasureTheory.Measure α'} {s : Set α'} (h : μ (frontier s) = 0) :
        μ (interior s) = μ s
        theorem closure_ae_eq_of_null_frontier {α' : Type u_6} [TopologicalSpace α'] [MeasurableSpace α'] {μ : MeasureTheory.Measure α'} {s : Set α'} (h : μ (frontier s) = 0) :
        theorem measure_closure_of_null_frontier {α' : Type u_6} [TopologicalSpace α'] [MeasurableSpace α'] {μ : MeasureTheory.Measure α'} {s : Set α'} (h : μ (frontier s) = 0) :
        μ (closure s) = μ s
        theorem Continuous.measurable {α : Type u_1} {γ : Type u_3} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] {f : αγ} (hf : Continuous f) :

        A continuous function from an OpensMeasurableSpace to a BorelSpace is measurable.

        theorem Continuous.aemeasurable {α : Type u_1} {γ : Type u_3} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] {f : αγ} (h : Continuous f) {μ : MeasureTheory.Measure α} :

        A continuous function from an OpensMeasurableSpace to a BorelSpace is ae-measurable.

        @[deprecated IsClosedEmbedding.measurable (since := "2024-10-20")]

        Alias of IsClosedEmbedding.measurable.

        theorem ContinuousOn.measurable_piecewise {α : Type u_1} {γ : Type u_3} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] {f g : αγ} {s : Set α} [(j : α) → Decidable (j s)] (hf : ContinuousOn f s) (hg : ContinuousOn g s) (hs : MeasurableSet s) :

        If a function is defined piecewise in terms of functions which are continuous on their respective pieces, then it is measurable.

        @[instance 100]
        @[instance 100]
        @[instance 100]
        @[instance 100]
        @[instance 100]
        def Homeomorph.toMeasurableEquiv {γ : Type u_3} {γ₂ : Type u_4} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [TopologicalSpace γ₂] [MeasurableSpace γ₂] [BorelSpace γ₂] (h : γ ≃ₜ γ₂) :
        γ ≃ᵐ γ₂

        A homeomorphism between two Borel spaces is a measurable equivalence.

        Equations
        theorem Homeomorph.measurableEmbedding {γ : Type u_3} {γ₂ : Type u_4} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [TopologicalSpace γ₂] [MeasurableSpace γ₂] [BorelSpace γ₂] (h : γ ≃ₜ γ₂) :
        @[simp]
        theorem Homeomorph.toMeasurableEquiv_coe {γ : Type u_3} {γ₂ : Type u_4} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [TopologicalSpace γ₂] [MeasurableSpace γ₂] [BorelSpace γ₂] (h : γ ≃ₜ γ₂) :
        @[simp]
        theorem Homeomorph.toMeasurableEquiv_symm_coe {γ : Type u_3} {γ₂ : Type u_4} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [TopologicalSpace γ₂] [MeasurableSpace γ₂] [BorelSpace γ₂] (h : γ ≃ₜ γ₂) :
        theorem Continuous.measurable2 {α : Type u_1} {β : Type u_2} {γ : Type u_3} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [TopologicalSpace β] [MeasurableSpace β] [OpensMeasurableSpace β] [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [MeasurableSpace δ] [SecondCountableTopologyEither α β] {f : δα} {g : δβ} {c : αβγ} (h : Continuous fun (p : α × β) => c p.1 p.2) (hf : Measurable f) (hg : Measurable g) :
        Measurable fun (a : δ) => c (f a) (g a)
        theorem Continuous.aemeasurable2 {α : Type u_1} {β : Type u_2} {γ : Type u_3} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [TopologicalSpace β] [MeasurableSpace β] [OpensMeasurableSpace β] [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [MeasurableSpace δ] [SecondCountableTopologyEither α β] {f : δα} {g : δβ} {c : αβγ} {μ : MeasureTheory.Measure δ} (h : Continuous fun (p : α × β) => c p.1 p.2) (hf : AEMeasurable f μ) (hg : AEMeasurable g μ) :
        AEMeasurable (fun (a : δ) => c (f a) (g a)) μ
        theorem pi_le_borel_pi {ι : Type u_6} {X : ιType u_7} [(i : ι) → TopologicalSpace (X i)] [(i : ι) → MeasurableSpace (X i)] [∀ (i : ι), BorelSpace (X i)] :
        MeasurableSpace.pi borel ((i : ι) → X i)
        instance Pi.borelSpace {ι : Type u_6} {X : ιType u_7} [Countable ι] [(i : ι) → TopologicalSpace (X i)] [(i : ι) → MeasurableSpace (X i)] [∀ (i : ι), SecondCountableTopology (X i)] [∀ (i : ι), BorelSpace (X i)] :
        BorelSpace ((i : ι) → X i)
        theorem MeasurableEmbedding.borelSpace {α : Type u_6} {β : Type u_7} [MeasurableSpace α] [TopologicalSpace α] [MeasurableSpace β] [TopologicalSpace β] [ : BorelSpace β] {e : αβ} (h'e : MeasurableEmbedding e) (h''e : Topology.IsInducing e) :

        Given a measurable embedding to a Borel space which is also a topological embedding, then the source space is also a Borel space.

        @[deprecated Topology.IsEmbedding.measurableEmbedding (since := "2024-10-26")]

        Alias of Topology.IsEmbedding.measurableEmbedding.

        @[deprecated Topology.IsClosedEmbedding.measurableEmbedding (since := "2024-10-20")]

        Alias of Topology.IsClosedEmbedding.measurableEmbedding.

        @[deprecated Topology.IsOpenEmbedding.measurableEmbedding (since := "2024-10-18")]

        Alias of Topology.IsOpenEmbedding.measurableEmbedding.