Documentation

Mathlib.MeasureTheory.Constructions.BorelSpace.Basic

Borel (measurable) space #

Main definitions #

Main statements #

MeasurableSpace structure generated by TopologicalSpace.

Equations
Instances For
    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) :
    • borel_le : borel α h

      Borel-measurable sets are measurable.

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

    Instances
      • measurable_eq : inst✝ = borel α

        The measurable sets are exactly the Borel-measurable sets.

      A space with MeasurableSpace and TopologicalSpace structures such that the σ-algebra of measurable sets is exactly the σ-algebra generated by open 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.
        Instances For

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

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

            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.
            Instances For

              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.
              Instances For
                theorem MeasurableSet.induction_on_open {α : Type u_1} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] {C : Set αProp} (h_open : (U : Set α) → IsOpen UC U) (h_compl : (t : Set α) → MeasurableSet tC tC t) (h_union : (f : Set α) → Pairwise (Disjoint on f)(∀ (i : ), MeasurableSet (f i)) → ((i : ) → C (f i)) → C (⋃ (i : ), f i)) ⦃t : Set α :
                MeasurableSet tC t
                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_is_closed' {γ : Type u_3} {δ : Type u_5} [TopologicalSpace γ] [MeasurableSpace γ] [BorelSpace γ] [MeasurableSpace δ] {f : δγ} (hf : ∀ (s : Set γ), IsClosed sSet.Nonempty ss 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} {π : ιType u_7} [Countable ι] [t' : (i : ι) → TopologicalSpace (π i)] [(i : ι) → MeasurableSpace (π i)] [∀ (i : ι), TopologicalSpace.SecondCountableTopology (π i)] [∀ (i : ι), OpensMeasurableSpace (π i)] :
                OpensMeasurableSpace ((i : ι) → π i)
                Equations

                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.

                  Equations
                  theorem measure_interior_of_null_frontier {α' : Type u_6} [TopologicalSpace α'] [MeasurableSpace α'] {μ : MeasureTheory.Measure α'} {s : Set α'} (h : μ (frontier s) = 0) :
                  μ (interior s) = μ s
                  theorem measure_closure_of_null_frontier {α' : Type u_6} [TopologicalSpace α'] [MeasurableSpace α'] {μ : MeasureTheory.Measure α'} {s : Set α'} (h : μ (frontier s) = 0) :
                  μ (closure s) = μ s
                  @[simp]
                  theorem measurableSet_le {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace δ] [PartialOrder α] [OrderClosedTopology α] [TopologicalSpace.SecondCountableTopology α] {f : δα} {g : δα} (hf : Measurable f) (hg : Measurable g) :
                  MeasurableSet {a | f a g a}
                  theorem measurableSet_lt {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderClosedTopology α] [TopologicalSpace.SecondCountableTopology α] {f : δα} {g : δα} (hf : Measurable f) (hg : Measurable g) :
                  MeasurableSet {a | f a < g a}
                  theorem generateFrom_Ico_mem_le_borel {α : Type u_7} [TopologicalSpace α] [LinearOrder α] [OrderClosedTopology α] (s : Set α) (t : Set α) :
                  MeasurableSpace.generateFrom {S | l, l s u, u t l < u Set.Ico l u = S} borel α
                  theorem Dense.borel_eq_generateFrom_Ico_mem_aux {α : Type u_7} [TopologicalSpace α] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {s : Set α} (hd : Dense s) (hbot : ∀ (x : α), IsBot xx s) (hIoo : ∀ (x y : α), x < ySet.Ioo x y = y s) :
                  borel α = MeasurableSpace.generateFrom {S | l, l s u, u s l < u Set.Ico l u = S}
                  theorem Dense.borel_eq_generateFrom_Ioc_mem_aux {α : Type u_7} [TopologicalSpace α] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {s : Set α} (hd : Dense s) (hbot : ∀ (x : α), IsTop xx s) (hIoo : ∀ (x y : α), x < ySet.Ioo x y = x s) :
                  borel α = MeasurableSpace.generateFrom {S | l, l s u, u s l < u Set.Ioc l u = S}
                  theorem MeasureTheory.Measure.ext_of_Ico_finite {α : Type u_7} [TopologicalSpace α] {m : MeasurableSpace α} [TopologicalSpace.SecondCountableTopology α] [LinearOrder α] [OrderTopology α] [BorelSpace α] (μ : MeasureTheory.Measure α) (ν : MeasureTheory.Measure α) [MeasureTheory.IsFiniteMeasure μ] (hμν : μ Set.univ = ν Set.univ) (h : ∀ ⦃a b : α⦄, a < bμ (Set.Ico a b) = ν (Set.Ico a b)) :
                  μ = ν

                  Two finite measures on a Borel space are equal if they agree on all closed-open intervals. If α is a conditionally complete linear order with no top element, MeasureTheory.Measure.ext_of_Ico is an extensionality lemma with weaker assumptions on μ and ν.

                  theorem MeasureTheory.Measure.ext_of_Ioc_finite {α : Type u_7} [TopologicalSpace α] {m : MeasurableSpace α} [TopologicalSpace.SecondCountableTopology α] [LinearOrder α] [OrderTopology α] [BorelSpace α] (μ : MeasureTheory.Measure α) (ν : MeasureTheory.Measure α) [MeasureTheory.IsFiniteMeasure μ] (hμν : μ Set.univ = ν Set.univ) (h : ∀ ⦃a b : α⦄, a < bμ (Set.Ioc a b) = ν (Set.Ioc a b)) :
                  μ = ν

                  Two finite measures on a Borel space are equal if they agree on all open-closed intervals. If α is a conditionally complete linear order with no top element, MeasureTheory.Measure.ext_of_Ioc is an extensionality lemma with weaker assumptions on μ and ν.

                  theorem MeasureTheory.Measure.ext_of_Ico' {α : Type u_7} [TopologicalSpace α] {m : MeasurableSpace α} [TopologicalSpace.SecondCountableTopology α] [LinearOrder α] [OrderTopology α] [BorelSpace α] [NoMaxOrder α] (μ : MeasureTheory.Measure α) (ν : MeasureTheory.Measure α) (hμ : ∀ ⦃a b : α⦄, a < bμ (Set.Ico a b) ) (h : ∀ ⦃a b : α⦄, a < bμ (Set.Ico a b) = ν (Set.Ico a b)) :
                  μ = ν

                  Two measures which are finite on closed-open intervals are equal if the agree on all closed-open intervals.

                  theorem MeasureTheory.Measure.ext_of_Ioc' {α : Type u_7} [TopologicalSpace α] {m : MeasurableSpace α} [TopologicalSpace.SecondCountableTopology α] [LinearOrder α] [OrderTopology α] [BorelSpace α] [NoMinOrder α] (μ : MeasureTheory.Measure α) (ν : MeasureTheory.Measure α) (hμ : ∀ ⦃a b : α⦄, a < bμ (Set.Ioc a b) ) (h : ∀ ⦃a b : α⦄, a < bμ (Set.Ioc a b) = ν (Set.Ioc a b)) :
                  μ = ν

                  Two measures which are finite on closed-open intervals are equal if the agree on all open-closed intervals.

                  Two measures which are finite on closed-open intervals are equal if the agree on all closed-open intervals.

                  Two measures which are finite on closed-open intervals are equal if the agree on all open-closed intervals.

                  Two finite measures on a Borel space are equal if they agree on all left-infinite right-closed intervals.

                  Two finite measures on a Borel space are equal if they agree on all left-closed right-infinite intervals.

                  theorem Measurable.max {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderClosedTopology α] [TopologicalSpace.SecondCountableTopology α] {f : δα} {g : δα} (hf : Measurable f) (hg : Measurable g) :
                  Measurable fun a => max (f a) (g a)
                  theorem AEMeasurable.max {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderClosedTopology α] [TopologicalSpace.SecondCountableTopology α] {f : δα} {g : δα} {μ : MeasureTheory.Measure δ} (hf : AEMeasurable f) (hg : AEMeasurable g) :
                  AEMeasurable fun a => max (f a) (g a)
                  theorem Measurable.min {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderClosedTopology α] [TopologicalSpace.SecondCountableTopology α] {f : δα} {g : δα} (hf : Measurable f) (hg : Measurable g) :
                  Measurable fun a => min (f a) (g a)
                  theorem AEMeasurable.min {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderClosedTopology α] [TopologicalSpace.SecondCountableTopology α] {f : δα} {g : δα} {μ : MeasureTheory.Measure δ} (hf : AEMeasurable f) (hg : AEMeasurable g) :
                  AEMeasurable fun a => min (f a) (g a)
                  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.

                  A continuous function from an OpensMeasurableSpace to a BorelSpace is ae-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.

                  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
                  Instances For
                    @[simp]
                    theorem Homeomorph.toMeasurableEquiv_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.fst p.snd) (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.fst p.snd) (hf : AEMeasurable f) (hg : AEMeasurable g) :
                    AEMeasurable fun a => c (f a) (g a)
                    theorem pi_le_borel_pi {ι : Type u_6} {π : ιType u_7} [(i : ι) → TopologicalSpace (π i)] [(i : ι) → MeasurableSpace (π i)] [∀ (i : ι), BorelSpace (π i)] :
                    MeasurableSpace.pi borel ((i : ι) → π i)
                    theorem prod_le_borel_prod {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [TopologicalSpace β] [MeasurableSpace β] [BorelSpace β] :
                    Prod.instMeasurableSpace borel (α × β)
                    instance Pi.borelSpace {ι : Type u_6} {π : ιType u_7} [Countable ι] [(i : ι) → TopologicalSpace (π i)] [(i : ι) → MeasurableSpace (π i)] [∀ (i : ι), TopologicalSpace.SecondCountableTopology (π i)] [∀ (i : ι), BorelSpace (π i)] :
                    BorelSpace ((i : ι) → π i)
                    Equations
                    theorem Measurable.isLUB {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} [Countable ι] {f : ιδα} {g : δα} (hf : ∀ (i : ι), Measurable (f i)) (hg : ∀ (b : δ), IsLUB {a | i, f i b = a} (g b)) :

                    If a function is the least upper bound of countably many measurable functions, then it is measurable.

                    theorem Measurable.isLUB_of_mem {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} [Countable ι] {f : ιδα} {g : δα} {g' : δα} (hf : ∀ (i : ι), Measurable (f i)) {s : Set δ} (hs : MeasurableSet s) (hg : ∀ (b : δ), b sIsLUB {a | i, f i b = a} (g b)) (hg' : Set.EqOn g g' s) (g'_meas : Measurable g') :

                    If a function is the least upper bound of countably many measurable functions on a measurable set s, and coincides with a measurable function outside of s, then it is measurable.

                    theorem AEMeasurable.isLUB {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} {μ : MeasureTheory.Measure δ} [Countable ι] {f : ιδα} {g : δα} (hf : ∀ (i : ι), AEMeasurable (f i)) (hg : ∀ᵐ (b : δ) ∂μ, IsLUB {a | i, f i b = a} (g b)) :
                    theorem Measurable.isGLB {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} [Countable ι] {f : ιδα} {g : δα} (hf : ∀ (i : ι), Measurable (f i)) (hg : ∀ (b : δ), IsGLB {a | i, f i b = a} (g b)) :

                    If a function is the greatest lower bound of countably many measurable functions, then it is measurable.

                    theorem Measurable.isGLB_of_mem {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} [Countable ι] {f : ιδα} {g : δα} {g' : δα} (hf : ∀ (i : ι), Measurable (f i)) {s : Set δ} (hs : MeasurableSet s) (hg : ∀ (b : δ), b sIsGLB {a | i, f i b = a} (g b)) (hg' : Set.EqOn g g' s) (g'_meas : Measurable g') :

                    If a function is the greatest lower bound of countably many measurable functions on a measurable set s, and coincides with a measurable function outside of s, then it is measurable.

                    theorem AEMeasurable.isGLB {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} {μ : MeasureTheory.Measure δ} [Countable ι] {f : ιδα} {g : δα} (hf : ∀ (i : ι), AEMeasurable (f i)) (hg : ∀ᵐ (b : δ) ∂μ, IsGLB {a | i, f i b = a} (g b)) :
                    theorem measurableSet_of_mem_nhdsWithin_Ioi_aux {α : Type u_1} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {s : Set α} (h : ∀ (x : α), x ss nhdsWithin x (Set.Ioi x)) (h' : ∀ (x : α), x sy, x < y) :

                    If a set is a right-neighborhood of all of its points, then it is measurable.

                    theorem measurableSet_bddAbove_range {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} [Countable ι] {f : ιδα} (hf : ∀ (i : ι), Measurable (f i)) :
                    MeasurableSet {b | BddAbove (Set.range fun i => f i b)}
                    theorem measurableSet_bddBelow_range {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [LinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} [Countable ι] {f : ιδα} (hf : ∀ (i : ι), Measurable (f i)) :
                    MeasurableSet {b | BddBelow (Set.range fun i => f i b)}
                    theorem Measurable.iSup_Prop {δ : Type u_5} [MeasurableSpace δ] {α : Type u_6} [MeasurableSpace α] [ConditionallyCompleteLattice α] (p : Prop) {f : δα} (hf : Measurable f) :
                    Measurable fun b => ⨆ (x : p), f b
                    theorem Measurable.iInf_Prop {δ : Type u_5} [MeasurableSpace δ] {α : Type u_6} [MeasurableSpace α] [ConditionallyCompleteLattice α] (p : Prop) {f : δα} (hf : Measurable f) :
                    Measurable fun b => ⨅ (x : p), f b
                    theorem measurable_iSup {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} [Countable ι] {f : ιδα} (hf : ∀ (i : ι), Measurable (f i)) :
                    Measurable fun b => ⨆ (i : ι), f i b
                    theorem aemeasurable_iSup {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} {μ : MeasureTheory.Measure δ} [Countable ι] {f : ιδα} (hf : ∀ (i : ι), AEMeasurable (f i)) :
                    AEMeasurable fun b => ⨆ (i : ι), f i b
                    theorem measurable_iInf {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} [Countable ι] {f : ιδα} (hf : ∀ (i : ι), Measurable (f i)) :
                    Measurable fun b => ⨅ (i : ι), f i b
                    theorem aemeasurable_iInf {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Sort u_6} {μ : MeasureTheory.Measure δ} [Countable ι] {f : ιδα} (hf : ∀ (i : ι), AEMeasurable (f i)) :
                    AEMeasurable fun b => ⨅ (i : ι), f i b
                    theorem measurable_sSup {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Type u_6} {f : ιδα} {s : Set ι} (hs : Set.Countable s) (hf : ∀ (i : ι), i sMeasurable (f i)) :
                    Measurable fun x => sSup ((fun i => f i x) '' s)
                    theorem measurable_sInf {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Type u_6} {f : ιδα} {s : Set ι} (hs : Set.Countable s) (hf : ∀ (i : ι), i sMeasurable (f i)) :
                    Measurable fun x => sInf ((fun i => f i x) '' s)
                    theorem measurable_biSup {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Type u_6} (s : Set ι) {f : ιδα} (hs : Set.Countable s) (hf : ∀ (i : ι), i sMeasurable (f i)) :
                    Measurable fun b => ⨆ (i : ι) (_ : i s), f i b
                    theorem aemeasurable_biSup {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Type u_6} {μ : MeasureTheory.Measure δ} (s : Set ι) {f : ιδα} (hs : Set.Countable s) (hf : ∀ (i : ι), i sAEMeasurable (f i)) :
                    AEMeasurable fun b => ⨆ (i : ι) (_ : i s), f i b
                    theorem measurable_biInf {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Type u_6} (s : Set ι) {f : ιδα} (hs : Set.Countable s) (hf : ∀ (i : ι), i sMeasurable (f i)) :
                    Measurable fun b => ⨅ (i : ι) (_ : i s), f i b
                    theorem aemeasurable_biInf {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Type u_6} {μ : MeasureTheory.Measure δ} (s : Set ι) {f : ιδα} (hs : Set.Countable s) (hf : ∀ (i : ι), i sAEMeasurable (f i)) :
                    AEMeasurable fun b => ⨅ (i : ι) (_ : i s), f i b
                    theorem measurable_liminf' {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Type u_6} {ι' : Type u_7} {f : ιδα} {v : Filter ι} (hf : ∀ (i : ι), Measurable (f i)) {p : ι'Prop} {s : ι'Set ι} (hv : Filter.HasCountableBasis v p s) (hs : ∀ (j : ι'), Set.Countable (s j)) :
                    Measurable fun x => Filter.liminf (fun i => f i x) v

                    liminf over a general filter is measurable. See measurable_liminf for the version over .

                    theorem measurable_limsup' {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {ι : Type u_6} {ι' : Type u_7} {f : ιδα} {u : Filter ι} (hf : ∀ (i : ι), Measurable (f i)) {p : ι'Prop} {s : ι'Set ι} (hu : Filter.HasCountableBasis u p s) (hs : ∀ (i : ι'), Set.Countable (s i)) :
                    Measurable fun x => Filter.limsup (fun i => f i x) u

                    limsup over a general filter is measurable. See measurable_limsup for the version over .

                    theorem measurable_liminf {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {f : δα} (hf : ∀ (i : ), Measurable (f i)) :
                    Measurable fun x => Filter.liminf (fun i => f i x) Filter.atTop

                    liminf over is measurable. See measurable_liminf' for a version with a general filter.

                    theorem measurable_limsup {α : Type u_1} {δ : Type u_5} [TopologicalSpace α] [MeasurableSpace α] [BorelSpace α] [MeasurableSpace δ] [ConditionallyCompleteLinearOrder α] [OrderTopology α] [TopologicalSpace.SecondCountableTopology α] {f : δα} (hf : ∀ (i : ), Measurable (f i)) :
                    Measurable fun x => Filter.limsup (fun i => f i x) Filter.atTop

                    limsup over is measurable. See measurable_limsup' for a version with a general filter.

                    Convert a Homeomorph to a MeasurableEquiv.

                    Equations
                    Instances For
                      Equations
                      theorem measure_eq_measure_preimage_add_measure_tsum_Ico_zpow {α : Type u_1} [MeasurableSpace α] (μ : MeasureTheory.Measure α) {f : αENNReal} (hf : Measurable f) {s : Set α} (hs : MeasurableSet s) {t : NNReal} (ht : 1 < t) :
                      μ s = μ (s f ⁻¹' {0}) + μ (s f ⁻¹' {}) + ∑' (n : ), μ (s f ⁻¹' Set.Ico (t ^ n) (t ^ (n + 1)))

                      One can cut out ℝ≥0∞ into the sets {0}, Ico (t^n) (t^(n+1)) for n : ℤ and {∞}. This gives a way to compute the measure of a set in terms of sets on which a given function f does not fluctuate by more than t.

                      theorem Measurable.infDist {α : Type u_1} {β : Type u_2} [PseudoMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} (hf : Measurable f) {s : Set α} :
                      Measurable fun x => Metric.infDist (f x) s
                      theorem Measurable.infNndist {α : Type u_1} {β : Type u_2} [PseudoMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} (hf : Measurable f) {s : Set α} :
                      Measurable fun x => Metric.infNndist (f x) s
                      theorem Measurable.dist {α : Type u_1} {β : Type u_2} [PseudoMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace β] [TopologicalSpace.SecondCountableTopology α] {f : βα} {g : βα} (hf : Measurable f) (hg : Measurable g) :
                      Measurable fun b => dist (f b) (g b)
                      theorem Measurable.nndist {α : Type u_1} {β : Type u_2} [PseudoMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace β] [TopologicalSpace.SecondCountableTopology α] {f : βα} {g : βα} (hf : Measurable f) (hg : Measurable g) :
                      Measurable fun b => nndist (f b) (g b)
                      theorem Measurable.infEdist {α : Type u_1} {β : Type u_2} [PseudoEMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} (hf : Measurable f) {s : Set α} :
                      Measurable fun x => EMetric.infEdist (f x) s
                      theorem tendsto_measure_cthickening {α : Type u_1} [PseudoEMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] {μ : MeasureTheory.Measure α} {s : Set α} (hs : R, R > 0 μ (Metric.cthickening R s) ) :
                      Filter.Tendsto (fun r => μ (Metric.cthickening r s)) (nhds 0) (nhds (μ (closure s)))

                      If a set has a closed thickening with finite measure, then the measure of its r-closed thickenings converges to the measure of its closure as r tends to 0.

                      theorem tendsto_measure_cthickening_of_isClosed {α : Type u_1} [PseudoEMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] {μ : MeasureTheory.Measure α} {s : Set α} (hs : R, R > 0 μ (Metric.cthickening R s) ) (h's : IsClosed s) :
                      Filter.Tendsto (fun r => μ (Metric.cthickening r s)) (nhds 0) (nhds (μ s))

                      If a closed set has a closed thickening with finite measure, then the measure of its closed r-thickenings converge to its measure as r tends to 0.

                      theorem tendsto_measure_thickening {α : Type u_1} [PseudoEMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] {μ : MeasureTheory.Measure α} {s : Set α} (hs : R, R > 0 μ (Metric.thickening R s) ) :
                      Filter.Tendsto (fun r => μ (Metric.thickening r s)) (nhdsWithin 0 (Set.Ioi 0)) (nhds (μ (closure s)))

                      If a set has a thickening with finite measure, then the measures of its r-thickenings converge to the measure of its closure as r > 0 tends to 0.

                      theorem tendsto_measure_thickening_of_isClosed {α : Type u_1} [PseudoEMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] {μ : MeasureTheory.Measure α} {s : Set α} (hs : R, R > 0 μ (Metric.thickening R s) ) (h's : IsClosed s) :
                      Filter.Tendsto (fun r => μ (Metric.thickening r s)) (nhdsWithin 0 (Set.Ioi 0)) (nhds (μ s))

                      If a closed set has a thickening with finite measure, then the measure of its r-thickenings converge to its measure as r > 0 tends to 0.

                      theorem Measurable.edist {α : Type u_1} {β : Type u_2} [PseudoEMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace β] [TopologicalSpace.SecondCountableTopology α] {f : βα} {g : βα} (hf : Measurable f) (hg : Measurable g) :
                      Measurable fun b => edist (f b) (g b)
                      theorem AEMeasurable.edist {α : Type u_1} {β : Type u_2} [PseudoEMetricSpace α] [MeasurableSpace α] [OpensMeasurableSpace α] [MeasurableSpace β] [TopologicalSpace.SecondCountableTopology α] {f : βα} {g : βα} {μ : MeasureTheory.Measure β} (hf : AEMeasurable f) (hg : AEMeasurable g) :
                      AEMeasurable fun a => edist (f a) (g a)

                      Given a compact set in a proper space, the measure of its r-closed thickenings converges to its measure as r tends to 0.

                      theorem Real.isPiSystem_Ioo_rat :
                      IsPiSystem (⋃ (a : ) (b : ) (_ : a < b), {Set.Ioo a b})

                      The intervals (-(n + 1), (n + 1)) form a finite spanning sets in the set of open intervals with rational endpoints for a locally finite measure μ on .

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        theorem Real.measure_ext_Ioo_rat {μ : MeasureTheory.Measure } {ν : MeasureTheory.Measure } [MeasureTheory.IsLocallyFiniteMeasure μ] (h : ∀ (a b : ), μ (Set.Ioo a b) = ν (Set.Ioo a b)) :
                        μ = ν
                        theorem Measurable.real_toNNReal {α : Type u_1} [MeasurableSpace α] {f : α} (hf : Measurable f) :
                        Measurable fun x => Real.toNNReal (f x)
                        theorem AEMeasurable.real_toNNReal {α : Type u_1} [MeasurableSpace α] {f : α} {μ : MeasureTheory.Measure α} (hf : AEMeasurable f) :
                        theorem Measurable.coe_nnreal_real {α : Type u_1} [MeasurableSpace α] {f : αNNReal} (hf : Measurable f) :
                        Measurable fun x => ↑(f x)
                        theorem AEMeasurable.coe_nnreal_real {α : Type u_1} [MeasurableSpace α] {f : αNNReal} {μ : MeasureTheory.Measure α} (hf : AEMeasurable f) :
                        AEMeasurable fun x => ↑(f x)
                        theorem Measurable.coe_nnreal_ennreal {α : Type u_1} [MeasurableSpace α] {f : αNNReal} (hf : Measurable f) :
                        Measurable fun x => ↑(f x)
                        theorem AEMeasurable.coe_nnreal_ennreal {α : Type u_1} [MeasurableSpace α] {f : αNNReal} {μ : MeasureTheory.Measure α} (hf : AEMeasurable f) :
                        AEMeasurable fun x => ↑(f x)
                        theorem Measurable.ennreal_ofReal {α : Type u_1} [MeasurableSpace α] {f : α} (hf : Measurable f) :
                        Measurable fun x => ENNReal.ofReal (f x)
                        @[simp]
                        theorem measurable_coe_nnreal_real_iff {α : Type u_1} [MeasurableSpace α] {f : αNNReal} :
                        (Measurable fun x => ↑(f x)) Measurable f
                        @[simp]
                        theorem aEMeasurable_coe_nnreal_real_iff {α : Type u_1} [MeasurableSpace α] {f : αNNReal} {μ : MeasureTheory.Measure α} :
                        (AEMeasurable fun x => ↑(f x)) AEMeasurable f
                        theorem ENNReal.measurable_of_measurable_nnreal {α : Type u_1} [MeasurableSpace α] {f : ENNRealα} (h : Measurable fun p => f p) :

                        ℝ≥0∞ is MeasurableEquiv to ℝ≥0 ⊕ Unit.

                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          theorem ENNReal.measurable_of_measurable_nnreal_prod {β : Type u_2} {γ : Type u_3} [MeasurableSpace β] [MeasurableSpace γ] {f : ENNReal × βγ} (H₁ : Measurable fun p => f (p.fst, p.snd)) (H₂ : Measurable fun x => f (, x)) :
                          theorem ENNReal.measurable_of_measurable_nnreal_nnreal {β : Type u_2} [MeasurableSpace β] {f : ENNReal × ENNRealβ} (h₁ : Measurable fun p => f (p.fst, p.snd)) (h₂ : Measurable fun r => f (, r)) (h₃ : Measurable fun r => f (r, )) :
                          theorem Measurable.ennreal_toNNReal {α : Type u_1} [MeasurableSpace α] {f : αENNReal} (hf : Measurable f) :
                          @[simp]
                          theorem measurable_coe_nnreal_ennreal_iff {α : Type u_1} [MeasurableSpace α] {f : αNNReal} :
                          (Measurable fun x => ↑(f x)) Measurable f
                          @[simp]
                          theorem aemeasurable_coe_nnreal_ennreal_iff {α : Type u_1} [MeasurableSpace α] {f : αNNReal} {μ : MeasureTheory.Measure α} :
                          (AEMeasurable fun x => ↑(f x)) AEMeasurable f
                          theorem Measurable.ennreal_toReal {α : Type u_1} [MeasurableSpace α] {f : αENNReal} (hf : Measurable f) :
                          Measurable fun x => ENNReal.toReal (f x)
                          theorem AEMeasurable.ennreal_toReal {α : Type u_1} [MeasurableSpace α] {f : αENNReal} {μ : MeasureTheory.Measure α} (hf : AEMeasurable f) :
                          theorem Measurable.ennreal_tsum {α : Type u_1} [MeasurableSpace α] {ι : Type u_6} [Countable ι] {f : ιαENNReal} (h : ∀ (i : ι), Measurable (f i)) :
                          Measurable fun x => ∑' (i : ι), f i x

                          note: ℝ≥0∞ can probably be generalized in a future version of this lemma.

                          theorem Measurable.ennreal_tsum' {α : Type u_1} [MeasurableSpace α] {ι : Type u_6} [Countable ι] {f : ιαENNReal} (h : ∀ (i : ι), Measurable (f i)) :
                          Measurable (∑' (i : ι), f i)
                          theorem Measurable.nnreal_tsum {α : Type u_1} [MeasurableSpace α] {ι : Type u_6} [Countable ι] {f : ιαNNReal} (h : ∀ (i : ι), Measurable (f i)) :
                          Measurable fun x => ∑' (i : ι), f i x
                          theorem AEMeasurable.ennreal_tsum {α : Type u_1} [MeasurableSpace α] {ι : Type u_6} [Countable ι] {f : ιαENNReal} {μ : MeasureTheory.Measure α} (h : ∀ (i : ι), AEMeasurable (f i)) :
                          AEMeasurable fun x => ∑' (i : ι), f i x
                          theorem AEMeasurable.nnreal_tsum {α : Type u_6} [MeasurableSpace α] {ι : Type u_7} [Countable ι] {f : ιαNNReal} {μ : MeasureTheory.Measure α} (h : ∀ (i : ι), AEMeasurable (f i)) :
                          AEMeasurable fun x => ∑' (i : ι), f i x
                          theorem Measurable.coe_real_ereal {α : Type u_1} [MeasurableSpace α] {f : α} (hf : Measurable f) :
                          Measurable fun x => ↑(f x)
                          theorem AEMeasurable.coe_real_ereal {α : Type u_1} [MeasurableSpace α] {f : α} {μ : MeasureTheory.Measure α} (hf : AEMeasurable f) :
                          AEMeasurable fun x => ↑(f x)
                          theorem EReal.measurable_of_measurable_real {α : Type u_1} [MeasurableSpace α] {f : ERealα} (h : Measurable fun p => f p) :
                          theorem Measurable.ereal_toReal {α : Type u_1} [MeasurableSpace α] {f : αEReal} (hf : Measurable f) :
                          Measurable fun x => EReal.toReal (f x)
                          theorem AEMeasurable.ereal_toReal {α : Type u_1} [MeasurableSpace α] {f : αEReal} {μ : MeasureTheory.Measure α} (hf : AEMeasurable f) :
                          AEMeasurable fun x => EReal.toReal (f x)
                          theorem Measurable.coe_ereal_ennreal {α : Type u_1} [MeasurableSpace α] {f : αENNReal} (hf : Measurable f) :
                          Measurable fun x => ↑(f x)
                          theorem AEMeasurable.coe_ereal_ennreal {α : Type u_1} [MeasurableSpace α] {f : αENNReal} {μ : MeasureTheory.Measure α} (hf : AEMeasurable f) :
                          AEMeasurable fun x => ↑(f x)
                          theorem Measurable.norm {α : Type u_1} {β : Type u_2} [MeasurableSpace α] [NormedAddCommGroup α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} (hf : Measurable f) :
                          Measurable fun a => f a
                          theorem AEMeasurable.norm {α : Type u_1} {β : Type u_2} [MeasurableSpace α] [NormedAddCommGroup α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} {μ : MeasureTheory.Measure β} (hf : AEMeasurable f) :
                          AEMeasurable fun a => f a
                          theorem Measurable.nnnorm {α : Type u_1} {β : Type u_2} [MeasurableSpace α] [NormedAddCommGroup α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} (hf : Measurable f) :
                          Measurable fun a => f a‖₊
                          theorem AEMeasurable.nnnorm {α : Type u_1} {β : Type u_2} [MeasurableSpace α] [NormedAddCommGroup α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} {μ : MeasureTheory.Measure β} (hf : AEMeasurable f) :
                          theorem Measurable.ennnorm {α : Type u_1} {β : Type u_2} [MeasurableSpace α] [NormedAddCommGroup α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} (hf : Measurable f) :
                          Measurable fun a => f a‖₊
                          theorem AEMeasurable.ennnorm {α : Type u_1} {β : Type u_2} [MeasurableSpace α] [NormedAddCommGroup α] [OpensMeasurableSpace α] [MeasurableSpace β] {f : βα} {μ : MeasureTheory.Measure β} (hf : AEMeasurable f) :
                          AEMeasurable fun a => f a‖₊