mathlib documentation

measure_theory.​borel_space

measure_theory.​borel_space

Borel (measurable) space

Main definitions

Main statements

def borel (α : Type u) [topological_space α] :

measurable_space structure generated by topological_space.

Equations
theorem borel_eq_top_of_encodable {α : Type u} [topological_space α] [t1_space α] [encodable α] :

theorem borel_comap {α : Type u} {β : Type v} {f : α → β} {t : topological_space β} :

theorem continuous.​borel_measurable {α : Type u} {β : Type v} [topological_space α] [topological_space β] {f : α → β} :

@[class]
structure opens_measurable_space (α : Type u_1) [topological_space α] [h : measurable_space α] :
Prop

A space with measurable_space and topological_space structures such that all open sets are measurable.

Instances
@[class]
structure borel_space (α : Type u_1) [topological_space α] [measurable_space α] :
Prop
  • measurable_eq : _inst_2 = borel α

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

Instances
@[instance]

In a borel_space all open sets are measurable.

Equations
@[instance]
def subtype.​borel_space {α : Type u_1} [topological_space α] [measurable_space α] [hα : borel_space α] (s : set α) :

Equations
  • _ = _
@[instance]

Equations
  • _ = _
@[instance]

Equations
  • _ = _

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 : is_measurable s.

theorem continuous.​measurable {α : Type u} {γ : Type w} [topological_space α] [measurable_space α] [opens_measurable_space α] [topological_space γ] [measurable_space γ] [borel_space γ] {f : α → γ} :

A continuous function from an opens_measurable_space to a borel_space is measurable.

A homeomorphism between two Borel spaces is a measurable equivalence.

Equations
theorem measurable_of_continuous_on_compl_singleton {α : Type u} {γ : Type w} [topological_space α] [measurable_space α] [opens_measurable_space α] [topological_space γ] [measurable_space γ] [borel_space γ] [t1_space α] {f : α → γ} (a : α) :
continuous_on f {x : α | x a}measurable f

theorem continuous.​measurable2 {α : Type u} {β : Type v} {γ : Type w} {δ : Type x} [topological_space α] [measurable_space α] [opens_measurable_space α] [topological_space β] [measurable_space β] [opens_measurable_space β] [topological_space γ] [measurable_space γ] [borel_space γ] [measurable_space δ] [topological_space.second_countable_topology α] [topological_space.second_countable_topology β] {f : δ → α} {g : δ → β} {c : α → β → γ} :
continuous (λ (p : α × β), c p.fst p.snd)measurable fmeasurable gmeasurable (λ (a : δ), c (f a) (g a))

theorem measurable.​smul {α : Type u} {γ : Type w} {δ : Type x} [topological_space α] [measurable_space α] [opens_measurable_space α] [topological_space γ] [measurable_space γ] [borel_space γ] [measurable_space δ] [semiring α] [topological_space.second_countable_topology α] [add_comm_monoid γ] [topological_space.second_countable_topology γ] [semimodule α γ] [topological_semimodule α γ] {f : δ → α} {g : δ → γ} :
measurable fmeasurable gmeasurable (λ (c : δ), f c g c)

theorem measurable.​const_smul {γ : Type w} {δ : Type x} [topological_space γ] [measurable_space γ] [borel_space γ] [measurable_space δ] {α : Type u_1} [topological_space α] [semiring α] [add_comm_monoid γ] [semimodule α γ] [topological_semimodule α γ] {f : δ → γ} (hf : measurable f) (c : α) :
measurable (λ (x : δ), c f x)

theorem measurable_const_smul_iff {γ : Type w} {δ : Type x} [topological_space γ] [measurable_space γ] [borel_space γ] [measurable_space δ] {α : Type u_1} [topological_space α] [division_ring α] [add_comm_monoid γ] [semimodule α γ] [topological_semimodule α γ] {f : δ → γ} {c : α} :
c 0(measurable (λ (x : δ), c f x) measurable f)

theorem measurable.​max {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [opens_measurable_space α] [measurable_space δ] [decidable_linear_order α] [order_closed_topology α] [topological_space.second_countable_topology α] {f g : δ → α} :
measurable fmeasurable gmeasurable (λ (a : δ), max (f a) (g a))

theorem measurable.​min {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [opens_measurable_space α] [measurable_space δ] [decidable_linear_order α] [order_closed_topology α] [topological_space.second_countable_topology α] {f g : δ → α} :
measurable fmeasurable gmeasurable (λ (a : δ), min (f a) (g a))

theorem measurable.​add {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [has_add α] [has_continuous_add α] [topological_space.second_countable_topology α] {f g : δ → α} :
measurable fmeasurable gmeasurable (λ (a : δ), f a + g a)

theorem measurable.​mul {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [has_mul α] [has_continuous_mul α] [topological_space.second_countable_topology α] {f g : δ → α} :
measurable fmeasurable gmeasurable (λ (a : δ), f a * g a)

theorem measurable_mul_left {α : Type u} [topological_space α] [measurable_space α] [borel_space α] [has_mul α] [has_continuous_mul α] (x : α) :
measurable (λ (y : α), x * y)

theorem measurable_add_left {α : Type u} [topological_space α] [measurable_space α] [borel_space α] [has_add α] [has_continuous_add α] (x : α) :
measurable (λ (y : α), x + y)

theorem measurable_mul_right {α : Type u} [topological_space α] [measurable_space α] [borel_space α] [has_mul α] [has_continuous_mul α] (x : α) :
measurable (λ (y : α), y * x)

theorem measurable_add_right {α : Type u} [topological_space α] [measurable_space α] [borel_space α] [has_add α] [has_continuous_add α] (x : α) :
measurable (λ (y : α), y + x)

theorem finset.​measurable_sum {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] {ι : Type u_1} [add_comm_monoid α] [has_continuous_add α] [topological_space.second_countable_topology α] {f : ι → δ → α} (s : finset ι) :
(∀ (i : ι), measurable (f i))measurable (λ (a : δ), s.sum (λ (i : ι), f i a))

theorem finset.​measurable_prod {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] {ι : Type u_1} [comm_monoid α] [has_continuous_mul α] [topological_space.second_countable_topology α] {f : ι → δ → α} (s : finset ι) :
(∀ (i : ι), measurable (f i))measurable (λ (a : δ), s.prod (λ (i : ι), f i a))

theorem measurable.​inv {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [group α] [topological_group α] {f : δ → α} :
measurable fmeasurable (λ (a : δ), (f a)⁻¹)

theorem measurable.​neg {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [add_group α] [topological_add_group α] {f : δ → α} :
measurable fmeasurable (λ (a : δ), -f a)

theorem measurable.​inv' {δ : Type x} [measurable_space δ] {α : Type u_1} [normed_field α] [measurable_space α] [borel_space α] {f : δ → α} :
measurable fmeasurable (λ (a : δ), (f a)⁻¹)

theorem measurable.​of_neg {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [add_group α] [topological_add_group α] {f : δ → α} :
measurable (λ (a : δ), -f a)measurable f

theorem measurable.​of_inv {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [group α] [topological_group α] {f : δ → α} :
measurable (λ (a : δ), (f a)⁻¹)measurable f

@[simp]
theorem measurable_inv_iff {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [group α] [topological_group α] {f : δ → α} :
measurable (λ (a : δ), (f a)⁻¹) measurable f

@[simp]
theorem measurable_neg_iff {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [add_group α] [topological_add_group α] {f : δ → α} :
measurable (λ (a : δ), -f a) measurable f

theorem measurable.​sub {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [add_group α] [topological_add_group α] [topological_space.second_countable_topology α] {f g : δ → α} :
measurable fmeasurable gmeasurable (λ (x : δ), f x - g x)

theorem measurable.​is_lub {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [linear_order α] [order_topology α] [topological_space.second_countable_topology α] {ι : Type u_1} [encodable ι] {f : ι → δ → α} {g : δ → α} :
(∀ (i : ι), measurable (f i))(∀ (b : δ), is_lub {a : α | ∃ (i : ι), f i b = a} (g b))measurable g

theorem measurable.​is_glb {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [linear_order α] [order_topology α] [topological_space.second_countable_topology α] {ι : Type u_1} [encodable ι] {f : ι → δ → α} {g : δ → α} :
(∀ (i : ι), measurable (f i))(∀ (b : δ), is_glb {a : α | ∃ (i : ι), f i b = a} (g b))measurable g

theorem measurable_supr {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [complete_linear_order α] [order_topology α] [topological_space.second_countable_topology α] {ι : Type u_1} [encodable ι] {f : ι → δ → α} :
(∀ (i : ι), measurable (f i))measurable (λ (b : δ), ⨆ (i : ι), f i b)

theorem measurable_infi {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [complete_linear_order α] [order_topology α] [topological_space.second_countable_topology α] {ι : Type u_1} [encodable ι] {f : ι → δ → α} :
(∀ (i : ι), measurable (f i))measurable (λ (b : δ), ⨅ (i : ι), f i b)

theorem measurable.​supr_Prop {δ : Type x} [measurable_space δ] {α : Type u_1} [measurable_space α] [complete_lattice α] (p : Prop) {f : δ → α} :
measurable fmeasurable (λ (b : δ), ⨆ (h : p), f b)

theorem measurable.​infi_Prop {δ : Type x} [measurable_space δ] {α : Type u_1} [measurable_space α] [complete_lattice α] (p : Prop) {f : δ → α} :
measurable fmeasurable (λ (b : δ), ⨅ (h : p), f b)

theorem measurable_bsupr {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [complete_linear_order α] [order_topology α] [topological_space.second_countable_topology α] {ι : Type u_1} [encodable ι] (p : ι → Prop) {f : ι → δ → α} :
(∀ (i : ι), measurable (f i))measurable (λ (b : δ), ⨆ (i : ι) (hi : p i), f i b)

theorem measurable_binfi {α : Type u} {δ : Type x} [topological_space α] [measurable_space α] [borel_space α] [measurable_space δ] [complete_linear_order α] [order_topology α] [topological_space.second_countable_topology α] {ι : Type u_1} [encodable ι] (p : ι → Prop) {f : ι → δ → α} :
(∀ (i : ι), measurable (f i))measurable (λ (b : δ), ⨅ (i : ι) (hi : p i), f i b)

@[instance]

Equations
@[instance]

Equations
@[instance]

Equations
@[instance]

Equations
@[instance]

Equations
@[instance]

Equations
theorem is_measurable_ball {α : Type u} [metric_space α] [measurable_space α] [opens_measurable_space α] {x : α} {ε : } :

theorem measurable.​dist {α : Type u} {β : Type v} [metric_space α] [measurable_space α] [opens_measurable_space α] [topological_space.second_countable_topology α] [measurable_space β] {f g : β → α} :
measurable fmeasurable gmeasurable (λ (b : β), has_dist.dist (f b) (g b))

theorem measurable.​nndist {α : Type u} {β : Type v} [metric_space α] [measurable_space α] [opens_measurable_space α] [topological_space.second_countable_topology α] [measurable_space β] {f g : β → α} :
measurable fmeasurable gmeasurable (λ (b : β), nndist (f b) (g b))

theorem is_measurable_eball {α : Type u} [emetric_space α] [measurable_space α] [opens_measurable_space α] {x : α} {ε : ennreal} :

theorem measurable.​edist {α : Type u} {β : Type v} [emetric_space α] [measurable_space α] [opens_measurable_space α] [topological_space.second_countable_topology α] [measurable_space β] {f g : β → α} :
measurable fmeasurable gmeasurable (λ (b : β), has_edist.edist (f b) (g b))

theorem measurable.​sub_nnreal {α : Type u} [measurable_space α] {f g : α → nnreal} :
measurable fmeasurable gmeasurable (λ (a : α), f a - g a)

theorem measurable.​nnreal_of_real {α : Type u} [measurable_space α] {f : α → } :
measurable fmeasurable (λ (x : α), nnreal.of_real (f x))

theorem measurable.​nnreal_coe {α : Type u} [measurable_space α] {f : α → nnreal} :
measurable fmeasurable (λ (x : α), (f x))

theorem measurable.​ennreal_coe {α : Type u} [measurable_space α] {f : α → nnreal} :
measurable fmeasurable (λ (x : α), (f x))

theorem measurable.​ennreal_of_real {α : Type u} [measurable_space α] {f : α → } :
measurable fmeasurable (λ (x : α), ennreal.of_real (f x))

theorem ennreal.​measurable_of_measurable_nnreal {α : Type u} [measurable_space α] {f : ennreal → α} :
measurable (λ (p : nnreal), f p)measurable f

ennreal is measurable_equiv to nnrealunit.

Equations
theorem ennreal.​measurable_of_measurable_nnreal_nnreal {α : Type u} {β : Type v} [measurable_space α] [measurable_space β] (f : ennrealennreal → β) {g h : α → ennreal} :
measurable (λ (p : nnreal × nnreal), f (p.fst) (p.snd))measurable (λ (r : nnreal), f r)measurable (λ (r : nnreal), f r )measurable gmeasurable hmeasurable (λ (a : α), f (g a) (h a))

theorem measurable.​ennreal_mul {α : Type u_1} [measurable_space α] {f g : α → ennreal} :
measurable fmeasurable gmeasurable (λ (a : α), f a * g a)

theorem measurable.​ennreal_add {α : Type u_1} [measurable_space α] {f g : α → ennreal} :
measurable fmeasurable gmeasurable (λ (a : α), f a + g a)

theorem measurable.​ennreal_sub {α : Type u_1} [measurable_space α] {f g : α → ennreal} :
measurable fmeasurable gmeasurable (λ (a : α), f a - g a)

theorem measurable.​norm {α : Type u} {β : Type v} [measurable_space α] [normed_group α] [opens_measurable_space α] [measurable_space β] {f : β → α} :
measurable fmeasurable (λ (a : β), f a)

theorem measurable.​nnnorm {α : Type u} {β : Type v} [measurable_space α] [normed_group α] [opens_measurable_space α] [measurable_space β] {f : β → α} :
measurable fmeasurable (λ (a : β), nnnorm (f a))

theorem measurable.​ennnorm {α : Type u} {β : Type v} [measurable_space α] [normed_group α] [opens_measurable_space α] [measurable_space β] {f : β → α} :
measurable fmeasurable (λ (a : β), (nnnorm (f a)))

A measure μ is regular if

  • it is finite on all compact sets;
  • it is outer regular: μ(A) = inf { μ(U) | A ⊆ U open } for A measurable;
  • it is inner regular: μ(U) = sup { μ(K) | K ⊆ U compact } for U open.
theorem measure_theory.​measure.​regular.​outer_regular_eq {α : Type u} [measurable_space α] [topological_space α] {μ : measure_theory.measure α} (hμ : μ.regular) ⦃A : set α⦄ :
is_measurable A(⨅ (U : set α) (h : is_open U) (h2 : A U), μ U) = μ A

theorem measure_theory.​measure.​regular.​inner_regular_eq {α : Type u} [measurable_space α] [topological_space α] {μ : measure_theory.measure α} (hμ : μ.regular) ⦃U : set α⦄ :
is_open U(⨆ (K : set α) (h : is_compact K) (h2 : K U), μ K) = μ U