Documentation

Mathlib.MeasureTheory.Measure.Support

Support of a Measure #

This file develops the theory of the support of a measure μ on a topological measurable space. The support is defined as the set of points whose every open neighborhood has positive measure. We give equivalent characterizations, prove basic measure-theoretic properties, and study interactions with sums, restrictions, and absolute continuity. Under various Lindelöf conditions, the support is conull, and various descriptions of the complement of the support are provided.

Main definitions #

Main results #

Tags #

measure, support, Lindelöf

A point x is in the support of μ if any open neighborhood of x has positive measure. We provide the definition in terms of the filter-theoretic equivalent ∃ᶠ u in (𝓝 x).smallSets, 0 < μ u.

Equations
Instances For
    theorem Filter.HasBasis.mem_measureSupport {X : Type u_1} [TopologicalSpace X] [MeasurableSpace X] {μ : MeasureTheory.Measure X} {ι : Sort u_2} {p : ιProp} {s : ιSet X} {x : X} (hl : (nhds x).HasBasis p s) :
    x μ.support ∀ (i : ι), p i0 < μ (s i)
    theorem MeasureTheory.Measure.mem_support_iff {X : Type u_1} [TopologicalSpace X] [MeasurableSpace X] {μ : Measure X} {x : X} :
    x μ.support ∃ᶠ (u : Set X) in (nhds x).smallSets, 0 < μ u

    A point x is in the support of measure μ iff any neighborhood of x contains a subset with positive measure.

    theorem MeasureTheory.Measure.mem_support_iff_forall {X : Type u_1} [TopologicalSpace X] [MeasurableSpace X] {μ : Measure X} (x : X) :
    x μ.support Unhds x, 0 < μ U

    A point x is in the support of measure μ iff every neighborhood of x has positive measure.

    theorem MeasureTheory.Measure.notMem_support_iff {X : Type u_1} [TopologicalSpace X] [MeasurableSpace X] {μ : Measure X} {x : X} :
    xμ.support ∀ᶠ (u : Set X) in (nhds x).smallSets, μ u = 0

    A point x lies outside the support of μ iff all of the subsets of one of its neighborhoods have measure zero.

    theorem Filter.HasBasis.notMem_measureSupport {X : Type u_1} [TopologicalSpace X] [MeasurableSpace X] {μ : MeasureTheory.Measure X} {ι : Sort u_2} {p : ιProp} {s : ιSet X} {x : X} (hl : (nhds x).HasBasis p s) :
    xμ.support ∃ (i : ι), p i μ (s i) = 0

    The support of the sum of two measures is the union of the supports.

    theorem MeasureTheory.Measure.notMem_support_iff_exists {X : Type u_1} [TopologicalSpace X] [MeasurableSpace X] {μ : Measure X} {x : X} :
    xμ.support Unhds x, μ U = 0

    A point x lies outside the support of μ iff some neighborhood of x has measure zero.

    theorem MeasureTheory.Measure.support_eq_forall_isOpen {X : Type u_1} [TopologicalSpace X] [MeasurableSpace X] {μ : Measure X} :
    μ.support = {x : X | ∀ (u : Set X), x uIsOpen u0 < μ u}

    The support of a measure equals the set of points whose open neighborhoods all have positive measure.

    If the complement of the support is Lindelöf, then the support of a measure is conull.

    In a hereditarily Lindelöf space, the support of a measure is conull.

    Under the assumption OpensMeasurableSpace, this is redundant because the complement of the support is open, and therefore measurable.

    Under the assumption OpensMeasurableSpace, this is redundant because the support is closed, and therefore measurable.