mathlib3 documentation

measure_theory.function.simple_func

Simple functions #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

A function f from a measurable space to any type is called simple, if every preimage f ⁻¹' {x} is measurable, and the range is finite. In this file, we define simple functions and establish their basic properties; and we construct a sequence of simple functions approximating an arbitrary Borel measurable function f : α → ℝ≥0∞.

The theorem measurable.ennreal_induction shows that in order to prove something for an arbitrary measurable function into ℝ≥0∞, it is sufficient to show that the property holds for (multiples of) characteristic functions and is closed under addition and supremum of increasing sequences of functions.

structure measure_theory.simple_func (α : Type u) [measurable_space α] (β : Type v) :
Type (max u v)

A function f from a measurable space to any type is called simple, if every preimage f ⁻¹' {x} is measurable, and the range is finite. This structure bundles a function with these properties.

Instances for measure_theory.simple_func
theorem measure_theory.simple_func.coe_injective {α : Type u_1} {β : Type u_2} [measurable_space α] ⦃f g : measure_theory.simple_func α β⦄ (H : f = g) :
f = g
@[ext]
theorem measure_theory.simple_func.ext {α : Type u_1} {β : Type u_2} [measurable_space α] {f g : measure_theory.simple_func α β} (H : (a : α), f a = g a) :
f = g
@[simp]
theorem measure_theory.simple_func.apply_mk {α : Type u_1} {β : Type u_2} [measurable_space α] (f : α β) (h : (x : β), measurable_set (f ⁻¹' {x})) (h' : (set.range f).finite) (x : α) :

Simple function defined on the empty type.

Equations
@[protected]
noncomputable def measure_theory.simple_func.range {α : Type u_1} {β : Type u_2} [measurable_space α] (f : measure_theory.simple_func α β) :

Range of a simple function α →ₛ β as a finset β.

Equations
@[simp]
theorem measure_theory.simple_func.mem_range {α : Type u_1} {β : Type u_2} [measurable_space α] {f : measure_theory.simple_func α β} {b : β} :
theorem measure_theory.simple_func.mem_range_self {α : Type u_1} {β : Type u_2} [measurable_space α] (f : measure_theory.simple_func α β) (x : α) :
theorem measure_theory.simple_func.mem_range_of_measure_ne_zero {α : Type u_1} {β : Type u_2} [measurable_space α] {f : measure_theory.simple_func α β} {x : β} {μ : measure_theory.measure α} (H : μ (f ⁻¹' {x}) 0) :
theorem measure_theory.simple_func.forall_range_iff {α : Type u_1} {β : Type u_2} [measurable_space α] {f : measure_theory.simple_func α β} {p : β Prop} :
( (y : β), y f.range p y) (x : α), p (f x)
theorem measure_theory.simple_func.exists_range_iff {α : Type u_1} {β : Type u_2} [measurable_space α] {f : measure_theory.simple_func α β} {p : β Prop} :
( (y : β) (H : y f.range), p y) (x : α), p (f x)
theorem measure_theory.simple_func.exists_forall_le {α : Type u_1} {β : Type u_2} [measurable_space α] [nonempty β] [preorder β] [is_directed β has_le.le] (f : measure_theory.simple_func α β) :
(C : β), (x : α), f x C
def measure_theory.simple_func.const (α : Type u_1) {β : Type u_2} [measurable_space α] (b : β) :

Constant function as a simple_func.

Equations
theorem measure_theory.simple_func.const_apply {α : Type u_1} {β : Type u_2} [measurable_space α] (a : α) (b : β) :
@[simp]
theorem measure_theory.simple_func.range_const {β : Type u_2} (α : Type u_1) [measurable_space α] [nonempty α] (b : β) :
theorem measure_theory.simple_func.simple_func_bot {β : Type u_2} {α : Type u_1} (f : measure_theory.simple_func α β) [nonempty β] :
(c : β), (x : α), f x = c
theorem measure_theory.simple_func.measurable_set_cut {α : Type u_1} {β : Type u_2} [measurable_space α] (r : α β Prop) (f : measure_theory.simple_func α β) (h : (b : β), measurable_set {a : α | r a b}) :
measurable_set {a : α | r a (f a)}
@[measurability]
@[protected, measurability]

A simple function is measurable

@[protected, measurability]
@[protected]
theorem measure_theory.simple_func.sum_measure_preimage_singleton {α : Type u_1} {β : Type u_2} [measurable_space α] (f : measure_theory.simple_func α β) {μ : measure_theory.measure α} (s : finset β) :
s.sum (λ (y : β), μ (f ⁻¹' {y})) = μ (f ⁻¹' s)
noncomputable def measure_theory.simple_func.piecewise {α : Type u_1} {β : Type u_2} [measurable_space α] (s : set α) (hs : measurable_set s) (f g : measure_theory.simple_func α β) :

If-then-else as a simple_func.

Equations
theorem measure_theory.simple_func.piecewise_apply {α : Type u_1} {β : Type u_2} [measurable_space α] {s : set α} (hs : measurable_set s) (f g : measure_theory.simple_func α β) (a : α) :
theorem measure_theory.simple_func.range_indicator {α : Type u_1} {β : Type u_2} [measurable_space α] {s : set α} (hs : measurable_set s) (hs_nonempty : s.nonempty) (hs_ne_univ : s set.univ) (x y : β) :
theorem measure_theory.simple_func.measurable_bind {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space γ] (f : measure_theory.simple_func α β) (g : β α γ) (hg : (b : β), measurable (g b)) :
measurable (λ (a : α), g (f a) a)

If f : α →ₛ β is a simple function and g : β → α →ₛ γ is a family of simple functions, then f.bind g binds the first argument of g to f. In other words, f.bind g a = g (f a) a.

Equations
@[simp]
theorem measure_theory.simple_func.bind_apply {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (f : measure_theory.simple_func α β) (g : β measure_theory.simple_func α γ) (a : α) :
(f.bind g) a = (g (f a)) a
def measure_theory.simple_func.map {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (g : β γ) (f : measure_theory.simple_func α β) :

Given a function g : β → γ and a simple function f : α →ₛ β, f.map g return the simple function g ∘ f : α →ₛ γ

Equations
theorem measure_theory.simple_func.map_apply {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (g : β γ) (f : measure_theory.simple_func α β) (a : α) :
@[simp]
theorem measure_theory.simple_func.coe_map {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (g : β γ) (f : measure_theory.simple_func α β) :
@[simp]
theorem measure_theory.simple_func.map_preimage {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (f : measure_theory.simple_func α β) (g : β γ) (s : set γ) :
theorem measure_theory.simple_func.map_preimage_singleton {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (f : measure_theory.simple_func α β) (g : β γ) (c : γ) :
def measure_theory.simple_func.comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space β] (f : measure_theory.simple_func β γ) (g : α β) (hgm : measurable g) :

Composition of a simple_fun and a measurable function is a simple_func.

Equations
@[simp]
theorem measure_theory.simple_func.coe_comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space β] (f : measure_theory.simple_func β γ) {g : α β} (hgm : measurable g) :
(f.comp g hgm) = f g
theorem measure_theory.simple_func.range_comp_subset_range {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space β] (f : measure_theory.simple_func β γ) {g : α β} (hgm : measurable g) :
(f.comp g hgm).range f.range
noncomputable def measure_theory.simple_func.extend {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space β] (f₁ : measure_theory.simple_func α γ) (g : α β) (hg : measurable_embedding g) (f₂ : measure_theory.simple_func β γ) :

Extend a simple_func along a measurable embedding: f₁.extend g hg f₂ is the function F : β →ₛ γ such that F ∘ g = f₁ and F y = f₂ y whenever y ∉ range g.

Equations
@[simp]
theorem measure_theory.simple_func.extend_apply {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space β] (f₁ : measure_theory.simple_func α γ) {g : α β} (hg : measurable_embedding g) (f₂ : measure_theory.simple_func β γ) (x : α) :
(f₁.extend g hg f₂) (g x) = f₁ x
@[simp]
theorem measure_theory.simple_func.extend_apply' {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space β] (f₁ : measure_theory.simple_func α γ) {g : α β} (hg : measurable_embedding g) (f₂ : measure_theory.simple_func β γ) {y : β} (h : ¬ (x : α), g x = y) :
(f₁.extend g hg f₂) y = f₂ y
@[simp]
theorem measure_theory.simple_func.extend_comp_eq' {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space β] (f₁ : measure_theory.simple_func α γ) {g : α β} (hg : measurable_embedding g) (f₂ : measure_theory.simple_func β γ) :
(f₁.extend g hg f₂) g = f₁
@[simp]
theorem measure_theory.simple_func.extend_comp_eq {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [measurable_space β] (f₁ : measure_theory.simple_func α γ) {g : α β} (hg : measurable_embedding g) (f₂ : measure_theory.simple_func β γ) :
(f₁.extend g hg f₂).comp g _ = f₁

If f is a simple function taking values in β → γ and g is another simple function with the same domain and codomain β, then f.seq g = f a (g a).

Equations
@[simp]
theorem measure_theory.simple_func.seq_apply {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (f : measure_theory.simple_func α γ)) (g : measure_theory.simple_func α β) (a : α) :
(f.seq g) a = f a (g a)

Combine two simple functions f : α →ₛ β and g : α →ₛ β into λ a, (f a, g a).

Equations
@[simp]
theorem measure_theory.simple_func.pair_apply {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (f : measure_theory.simple_func α β) (g : measure_theory.simple_func α γ) (a : α) :
(f.pair g) a = (f a, g a)
theorem measure_theory.simple_func.pair_preimage {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (f : measure_theory.simple_func α β) (g : measure_theory.simple_func α γ) (s : set β) (t : set γ) :
theorem measure_theory.simple_func.pair_preimage_singleton {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] (f : measure_theory.simple_func α β) (g : measure_theory.simple_func α γ) (b : β) (c : γ) :
(f.pair g) ⁻¹' {(b, c)} = f ⁻¹' {b} g ⁻¹' {c}
@[protected, instance]
Equations
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_one {α : Type u_1} {β : Type u_2} [measurable_space α] [has_one β] :
1 = 1
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_zero {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] :
0 = 0
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_mul {α : Type u_1} {β : Type u_2} [measurable_space α] [has_mul β] (f g : measure_theory.simple_func α β) :
(f * g) = f * g
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_add {α : Type u_1} {β : Type u_2} [measurable_space α] [has_add β] (f g : measure_theory.simple_func α β) :
(f + g) = f + g
@[simp, norm_cast]
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_neg {α : Type u_1} {β : Type u_2} [measurable_space α] [has_neg β] (f : measure_theory.simple_func α β) :
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_div {α : Type u_1} {β : Type u_2} [measurable_space α] [has_div β] (f g : measure_theory.simple_func α β) :
(f / g) = f / g
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_sub {α : Type u_1} {β : Type u_2} [measurable_space α] [has_sub β] (f g : measure_theory.simple_func α β) :
(f - g) = f - g
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_le {α : Type u_1} {β : Type u_2} [measurable_space α] [preorder β] {f g : measure_theory.simple_func α β} :
f g f g
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_sup {α : Type u_1} {β : Type u_2} [measurable_space α] [has_sup β] (f g : measure_theory.simple_func α β) :
(f g) = f g
@[simp, norm_cast]
theorem measure_theory.simple_func.coe_inf {α : Type u_1} {β : Type u_2} [measurable_space α] [has_inf β] (f g : measure_theory.simple_func α β) :
(f g) = f g
theorem measure_theory.simple_func.add_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_add β] (f g : measure_theory.simple_func α β) (a : α) :
(f + g) a = f a + g a
theorem measure_theory.simple_func.mul_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_mul β] (f g : measure_theory.simple_func α β) (a : α) :
(f * g) a = f a * g a
theorem measure_theory.simple_func.div_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_div β] (f g : measure_theory.simple_func α β) (x : α) :
(f / g) x = f x / g x
theorem measure_theory.simple_func.sub_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_sub β] (f g : measure_theory.simple_func α β) (x : α) :
(f - g) x = f x - g x
theorem measure_theory.simple_func.neg_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_neg β] (f : measure_theory.simple_func α β) (x : α) :
(-f) x = -f x
theorem measure_theory.simple_func.inv_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_inv β] (f : measure_theory.simple_func α β) (x : α) :
theorem measure_theory.simple_func.sup_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_sup β] (f g : measure_theory.simple_func α β) (a : α) :
(f g) a = f a g a
theorem measure_theory.simple_func.inf_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_inf β] (f g : measure_theory.simple_func α β) (a : α) :
(f g) a = f a g a
@[simp]
theorem measure_theory.simple_func.range_one {α : Type u_1} {β : Type u_2} [measurable_space α] [nonempty α] [has_one β] :
1.range = {1}
@[simp]
theorem measure_theory.simple_func.range_zero {α : Type u_1} {β : Type u_2} [measurable_space α] [nonempty α] [has_zero β] :
0.range = {0}
theorem measure_theory.simple_func.eq_zero_of_mem_range_zero {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] {y : β} :
y 0.range y = 0
theorem measure_theory.simple_func.add_eq_map₂ {α : Type u_1} {β : Type u_2} [measurable_space α] [has_add β] (f g : measure_theory.simple_func α β) :
f + g = measure_theory.simple_func.map (λ (p : β × β), p.fst + p.snd) (f.pair g)
theorem measure_theory.simple_func.mul_eq_map₂ {α : Type u_1} {β : Type u_2} [measurable_space α] [has_mul β] (f g : measure_theory.simple_func α β) :
f * g = measure_theory.simple_func.map (λ (p : β × β), p.fst * p.snd) (f.pair g)
theorem measure_theory.simple_func.sup_eq_map₂ {α : Type u_1} {β : Type u_2} [measurable_space α] [has_sup β] (f g : measure_theory.simple_func α β) :
f g = measure_theory.simple_func.map (λ (p : β × β), p.fst p.snd) (f.pair g)
theorem measure_theory.simple_func.map_add {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [has_add β] [has_add γ] {g : β γ} (hg : (x y : β), g (x + y) = g x + g y) (f₁ f₂ : measure_theory.simple_func α β) :
theorem measure_theory.simple_func.map_mul {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [has_mul β] [has_mul γ] {g : β γ} (hg : (x y : β), g (x * y) = g x * g y) (f₁ f₂ : measure_theory.simple_func α β) :
@[simp]
theorem measure_theory.simple_func.coe_smul {α : Type u_1} {β : Type u_2} [measurable_space α] {K : Type u_5} [has_smul K β] (c : K) (f : measure_theory.simple_func α β) :
(c f) = c f
theorem measure_theory.simple_func.smul_apply {α : Type u_1} {β : Type u_2} [measurable_space α] {K : Type u_5} [has_smul K β] (k : K) (f : measure_theory.simple_func α β) (a : α) :
(k f) a = k f a
@[protected, instance]
Equations
@[simp]
theorem measure_theory.simple_func.coe_pow {α : Type u_1} {β : Type u_2} [measurable_space α] [monoid β] (f : measure_theory.simple_func α β) (n : ) :
(f ^ n) = f ^ n
theorem measure_theory.simple_func.pow_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [monoid β] (n : ) (f : measure_theory.simple_func α β) (a : α) :
(f ^ n) a = f a ^ n
@[simp]
theorem measure_theory.simple_func.coe_zpow {α : Type u_1} {β : Type u_2} [measurable_space α] [div_inv_monoid β] (f : measure_theory.simple_func α β) (z : ) :
(f ^ z) = f ^ z
theorem measure_theory.simple_func.zpow_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [div_inv_monoid β] (z : ) (f : measure_theory.simple_func α β) (a : α) :
(f ^ z) a = f a ^ z
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
theorem measure_theory.simple_func.finset_sup_apply {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [semilattice_sup β] [order_bot β] {f : γ measure_theory.simple_func α β} (s : finset γ) (a : α) :
(s.sup f) a = s.sup (λ (c : γ), (f c) a)
noncomputable def measure_theory.simple_func.restrict {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] (f : measure_theory.simple_func α β) (s : set α) :

Restrict a simple function f : α →ₛ β to a set s. If s is measurable, then f.restrict s a = if a ∈ s then f a else 0, otherwise f.restrict s = const α 0.

Equations
@[simp]
theorem measure_theory.simple_func.coe_restrict {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] (f : measure_theory.simple_func α β) {s : set α} (hs : measurable_set s) :
@[simp]
theorem measure_theory.simple_func.map_restrict_of_zero {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [has_zero β] [has_zero γ] {g : β γ} (hg : g 0 = 0) (f : measure_theory.simple_func α β) (s : set α) :
theorem measure_theory.simple_func.restrict_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] (f : measure_theory.simple_func α β) {s : set α} (hs : measurable_set s) (a : α) :
(f.restrict s) a = s.indicator f a
theorem measure_theory.simple_func.restrict_preimage {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] (f : measure_theory.simple_func α β) {s : set α} (hs : measurable_set s) {t : set β} (ht : 0 t) :
theorem measure_theory.simple_func.restrict_preimage_singleton {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] (f : measure_theory.simple_func α β) {s : set α} (hs : measurable_set s) {r : β} (hr : r 0) :
(f.restrict s) ⁻¹' {r} = s f ⁻¹' {r}
theorem measure_theory.simple_func.mem_restrict_range {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] {r : β} {s : set α} {f : measure_theory.simple_func α β} (hs : measurable_set s) :
r (f.restrict s).range r = 0 s set.univ r f '' s
theorem measure_theory.simple_func.mem_image_of_mem_range_restrict {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] {r : β} {s : set α} {f : measure_theory.simple_func α β} (hr : r (f.restrict s).range) (h0 : r 0) :
r f '' s
theorem measure_theory.simple_func.restrict_mono {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] [preorder β] (s : set α) {f g : measure_theory.simple_func α β} (H : f g) :
noncomputable def measure_theory.simple_func.approx {α : Type u_1} {β : Type u_2} [measurable_space α] [semilattice_sup β] [order_bot β] [has_zero β] (i : β) (f : α β) (n : ) :

Fix a sequence i : ℕ → β. Given a function α → β, its n-th approximation by simple functions is defined so that in case β = ℝ≥0∞ it sends each a to the supremum of the set {i k | k ≤ n ∧ i k ≤ f a}, see approx_apply and supr_approx_apply for details.

Equations
theorem measure_theory.simple_func.approx_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [semilattice_sup β] [order_bot β] [has_zero β] [topological_space β] [order_closed_topology β] [measurable_space β] [opens_measurable_space β] {i : β} {f : α β} {n : } (a : α) (hf : measurable f) :
(measure_theory.simple_func.approx i f n) a = (finset.range n).sup (λ (k : ), ite (i k f a) (i k) 0)
theorem measure_theory.simple_func.approx_comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} [measurable_space α] [semilattice_sup β] [order_bot β] [has_zero β] [topological_space β] [order_closed_topology β] [measurable_space β] [opens_measurable_space β] [measurable_space γ] {i : β} {f : γ β} {g : α γ} {n : } (a : α) (hf : measurable f) (hg : measurable g) :
theorem measure_theory.simple_func.supr_approx_apply {α : Type u_1} {β : Type u_2} [measurable_space α] [topological_space β] [complete_lattice β] [order_closed_topology β] [has_zero β] [measurable_space β] [opens_measurable_space β] (i : β) (f : α β) (a : α) (hf : measurable f) (h_zero : 0 = ) :
( (n : ), (measure_theory.simple_func.approx i f n) a) = (k : ) (h : i k f a), i k

A sequence of ℝ≥0∞s such that its range is the set of non-negative rational numbers.

Equations

Integral of a simple function whose codomain is ℝ≥0∞.

Equations
theorem measure_theory.simple_func.lintegral_eq_of_subset {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} (f : measure_theory.simple_func α ennreal) {s : finset ennreal} (hs : (x : α), f x 0 μ (f ⁻¹' {f x}) 0 f x s) :
f.lintegral μ = s.sum (λ (x : ennreal), x * μ (f ⁻¹' {x}))
theorem measure_theory.simple_func.map_lintegral {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} (g : β ennreal) (f : measure_theory.simple_func α β) :
(measure_theory.simple_func.map g f).lintegral μ = f.range.sum (λ (x : β), g x * μ (f ⁻¹' {x}))

Calculate the integral of (g ∘ f), where g : β → ℝ≥0∞ and f : α →ₛ β.

Integral of a simple function α →ₛ ℝ≥0∞ as a bilinear map.

Equations
theorem measure_theory.simple_func.lintegral_mono {α : Type u_1} {m : measurable_space α} {μ ν : measure_theory.measure α} {f g : measure_theory.simple_func α ennreal} (hfg : f g) (hμν : μ ν) :

simple_func.lintegral is monotone both in function and in measure.

simple_func.lintegral depends only on the measures of f ⁻¹' {y}.

If two simple functions are equal a.e., then their lintegrals are equal.

theorem measure_theory.simple_func.lintegral_map' {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_2} [measurable_space β] {μ' : measure_theory.measure β} (f : measure_theory.simple_func α ennreal) (g : measure_theory.simple_func β ennreal) (m' : α β) (eq : (a : α), f a = g (m' a)) (h : (s : set β), measurable_set s μ' s = μ (m' ⁻¹' s)) :
f.lintegral μ = g.lintegral μ'
theorem measure_theory.simple_func.support_eq {α : Type u_1} {β : Type u_2} [measurable_space α] [has_zero β] (f : measure_theory.simple_func α β) :
function.support f = (y : β) (H : y finset.filter (λ (y : β), y 0) f.range), f ⁻¹' {y}
@[protected]

A simple_func has finite measure support if it is equal to 0 outside of a set of finite measure.

Equations
theorem measure_theory.simple_func.fin_meas_supp_iff {α : Type u_1} {β : Type u_2} {m : measurable_space α} [has_zero β] {μ : measure_theory.measure α} {f : measure_theory.simple_func α β} :
f.fin_meas_supp μ (y : β), y 0 μ (f ⁻¹' {y}) <
@[protected]
theorem measure_theory.simple_func.fin_meas_supp.map {α : Type u_1} {β : Type u_2} {γ : Type u_3} {m : measurable_space α} [has_zero β] [has_zero γ] {μ : measure_theory.measure α} {f : measure_theory.simple_func α β} {g : β γ} (hf : f.fin_meas_supp μ) (hg : g 0 = 0) :
theorem measure_theory.simple_func.fin_meas_supp.of_map {α : Type u_1} {β : Type u_2} {γ : Type u_3} {m : measurable_space α} [has_zero β] [has_zero γ] {μ : measure_theory.measure α} {f : measure_theory.simple_func α β} {g : β γ} (h : (measure_theory.simple_func.map g f).fin_meas_supp μ) (hg : (b : β), g b = 0 b = 0) :
theorem measure_theory.simple_func.fin_meas_supp.map_iff {α : Type u_1} {β : Type u_2} {γ : Type u_3} {m : measurable_space α} [has_zero β] [has_zero γ] {μ : measure_theory.measure α} {f : measure_theory.simple_func α β} {g : β γ} (hg : {b : β}, g b = 0 b = 0) :
@[protected]
theorem measure_theory.simple_func.fin_meas_supp.pair {α : Type u_1} {β : Type u_2} {γ : Type u_3} {m : measurable_space α} [has_zero β] [has_zero γ] {μ : measure_theory.measure α} {f : measure_theory.simple_func α β} {g : measure_theory.simple_func α γ} (hf : f.fin_meas_supp μ) (hg : g.fin_meas_supp μ) :
@[protected]
theorem measure_theory.simple_func.fin_meas_supp.map₂ {α : Type u_1} {β : Type u_2} {γ : Type u_3} {δ : Type u_4} {m : measurable_space α} [has_zero β] [has_zero γ] {μ : measure_theory.measure α} {f : measure_theory.simple_func α β} [has_zero δ] (hf : f.fin_meas_supp μ) {g : measure_theory.simple_func α γ} (hg : g.fin_meas_supp μ) {op : β γ δ} (H : op 0 0 = 0) :
@[protected]
theorem measure_theory.simple_func.fin_meas_supp.add {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_2} [add_monoid β] {f g : measure_theory.simple_func α β} (hf : f.fin_meas_supp μ) (hg : g.fin_meas_supp μ) :
(f + g).fin_meas_supp μ
@[protected]
theorem measure_theory.simple_func.fin_meas_supp.mul {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_2} [monoid_with_zero β] {f g : measure_theory.simple_func α β} (hf : f.fin_meas_supp μ) (hg : g.fin_meas_supp μ) :
(f * g).fin_meas_supp μ
@[protected]

To prove something for an arbitrary simple function, it suffices to show that the property holds for (multiples of) characteristic functions and is closed under addition (of functions with disjoint support).

It is possible to make the hypotheses in h_add a bit stronger, and such conditions can be added once we need them (for example it is only necessary to consider the case where g is a multiple of a characteristic function, and that this multiple doesn't appear in the image of f)

theorem measurable.ennreal_induction {α : Type u_1} [measurable_space α] {P : ennreal) Prop} (h_ind : (c : ennreal) ⦃s : set α⦄, measurable_set s P (s.indicator (λ (_x : α), c))) (h_add : ⦃f g : α ennreal⦄, disjoint (function.support f) (function.support g) measurable f measurable g P f P g P (f + g)) (h_supr : ⦃f : α ennreal⦄, ( (n : ), measurable (f n)) monotone f ( (n : ), P (f n)) P (λ (x : α), (n : ), f n x)) ⦃f : α ennreal (hf : measurable f) :
P f

To prove something for an arbitrary measurable function into ℝ≥0∞, it suffices to show that the property holds for (multiples of) characteristic functions and is closed under addition and supremum of increasing sequences of functions.

It is possible to make the hypotheses in the induction steps a bit stronger, and such conditions can be added once we need them (for example in h_add it is only necessary to consider the sum of a simple function with a multiple of a characteristic function and that the intersection of their images is a subset of {0}.