Documentation

Mathlib.Topology.Baire.BaireMeasurable

Baire category and Baire measurable sets #

This file defines some of the basic notions of Baire category and Baire measurable sets.

Main definitions #

First, we define the notation =ᵇ. This denotes eventual equality with respect to the filter of residual sets in a topological space.

A set s in a topological space α is called a BaireMeasurableSet or said to have the property of Baire if it satisfies either of the following equivalent conditions:

Notation for =ᶠ[residual _]. That is, eventual equality with respect to the filter of residual sets.

Equations
Instances For

    Pretty printer defined by notation3 command.

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

      Notation to say that a property of points in a topological space holds almost everywhere in the sense of Baire category. That is, on a residual set.

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

        Pretty printer defined by notation3 command.

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

          Notation to say that a property of points in a topological space holds on a non meager set.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def BaireMeasurableSet {α : Type u_1} [TopologicalSpace α] (s : Set α) :

            We say a set is a BaireMeasurableSet if it differs from some Borel set by a meager set. This forms a σ-algebra.

            It is equivalent, and a more standard definition, to say that the set differs from some open set by a meager set. See BaireMeasurableSet.iff_residualEq_isOpen

            Equations
            Instances For
              theorem BaireMeasurableSet.iUnion {α : Type u_1} [TopologicalSpace α] {ι : Sort u_3} [Countable ι] {s : ιSet α} (h : ∀ (i : ι), BaireMeasurableSet (s i)) :
              BaireMeasurableSet (⋃ (i : ι), s i)
              theorem BaireMeasurableSet.biUnion {α : Type u_1} [TopologicalSpace α] {ι : Type u_3} {s : ιSet α} {t : Set ι} (ht : t.Countable) (h : it, BaireMeasurableSet (s i)) :
              BaireMeasurableSet (⋃ it, s i)
              theorem BaireMeasurableSet.sUnion {α : Type u_1} [TopologicalSpace α] {s : Set (Set α)} (hs : s.Countable) (h : ts, BaireMeasurableSet t) :
              theorem BaireMeasurableSet.iInter {α : Type u_1} [TopologicalSpace α] {ι : Sort u_3} [Countable ι] {s : ιSet α} (h : ∀ (i : ι), BaireMeasurableSet (s i)) :
              BaireMeasurableSet (⋂ (i : ι), s i)
              theorem BaireMeasurableSet.biInter {α : Type u_1} [TopologicalSpace α] {ι : Type u_3} {s : ιSet α} {t : Set ι} (ht : t.Countable) (h : it, BaireMeasurableSet (s i)) :
              BaireMeasurableSet (⋂ it, s i)
              theorem BaireMeasurableSet.sInter {α : Type u_1} [TopologicalSpace α] {s : Set (Set α)} (hs : s.Countable) (h : ts, BaireMeasurableSet t) :
              theorem BaireMeasurableSet.diff {α : Type u_1} [TopologicalSpace α] {s : Set α} {t : Set α} (hs : BaireMeasurableSet s) (ht : BaireMeasurableSet t) :
              theorem BaireMeasurableSet.congr {α : Type u_1} [TopologicalSpace α] {s : Set α} {t : Set α} (hs : BaireMeasurableSet s) (h : s =ᶠ[residual α] t) :
              theorem MeasurableSet.residualEq_isOpen {α : Type u_1} [TopologicalSpace α] {s : Set α} [MeasurableSpace α] [BorelSpace α] (h : MeasurableSet s) :
              ∃ (u : Set α), IsOpen u s =ᶠ[residual α] u

              Any Borel set differs from some open set by a meager set.

              theorem BaireMeasurableSet.residualEq_isOpen {α : Type u_1} [TopologicalSpace α] {s : Set α} (h : BaireMeasurableSet s) :
              ∃ (u : Set α), IsOpen u s =ᶠ[residual α] u

              Any BaireMeasurableSet differs from some open set by a meager set.

              A set is Baire measurable if and only if it differs from some open set by a meager set.

              theorem tendsto_residual_of_isOpenMap {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} (hc : Continuous f) (ho : IsOpenMap f) :
              theorem IsMeagre.preimage_of_isOpenMap {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} (hc : Continuous f) (ho : IsOpenMap f) {s : Set β} (h : IsMeagre s) :

              The preimage of a meager set under a continuous open map is meager.

              theorem BaireMeasurableSet.preimage {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} (hc : Continuous f) (ho : IsOpenMap f) {s : Set β} (h : BaireMeasurableSet s) :

              The preimage of a BaireMeasurableSet under a continuous open map is Baire measurable.

              theorem Homeomorph.residual_map_eq {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] (h : α ≃ₜ β) :
              Filter.map (⇑h) (residual α) = residual β