Skip to content

Commit

Permalink
feat(measure_theory/function/uniform_integrable): Uniform integrabili…
Browse files Browse the repository at this point in the history
…ty and Vitali convergence theorem (#12408)

This PR defines uniform integrability (both in the measure theory sense as well as the probability theory sense) and proves the Vitali convergence theorem which establishes a relation between convergence in measure and uniform integrability with convergence in Lp.
  • Loading branch information
JasonKYi committed Mar 7, 2022
1 parent 1ee91a5 commit f28023e
Show file tree
Hide file tree
Showing 5 changed files with 748 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/analysis/special_functions/pow.lean
Expand Up @@ -1404,6 +1404,13 @@ begin
rw [rpow_mul, ←one_div, @rpow_lt_rpow_iff _ _ (1/z) (by simp [hz])],
end

lemma rpow_one_div_le_iff {x y : ℝ≥0∞} {z : ℝ} (hz : 0 < z) : x ^ (1 / z) ≤ y ↔ x ≤ y ^ z :=
begin
nth_rewrite 0 ← ennreal.rpow_one y,
nth_rewrite 1 ← @_root_.mul_inv_cancel _ _ z hz.ne.symm,
rw [ennreal.rpow_mul, ← one_div, ennreal.rpow_le_rpow_iff (one_div_pos.2 hz)],
end

lemma rpow_lt_rpow_of_exponent_lt {x : ℝ≥0∞} {y z : ℝ} (hx : 1 < x) (hx' : x ≠ ⊤) (hyz : y < z) :
x^y < x^z :=
begin
Expand Down
17 changes: 17 additions & 0 deletions src/measure_theory/function/lp_space.lean
Expand Up @@ -1807,6 +1807,23 @@ end

end indicator_const_Lp

lemma mem_ℒp.norm_rpow [opens_measurable_space E] {f : α → E}
(hf : mem_ℒp f p μ) (hp_ne_zero : p ≠ 0) (hp_ne_top : p ≠ ∞) :
mem_ℒp (λ (x : α), ∥f x∥ ^ p.to_real) 1 μ :=
begin
refine ⟨hf.1.norm.pow_const _, _⟩,
have := hf.snorm_ne_top,
rw snorm_eq_lintegral_rpow_nnnorm hp_ne_zero hp_ne_top at this,
rw snorm_one_eq_lintegral_nnnorm,
convert ennreal.rpow_lt_top_of_nonneg (@ennreal.to_real_nonneg p) this,
rw [← ennreal.rpow_mul, one_div_mul_cancel (ennreal.to_real_pos hp_ne_zero hp_ne_top).ne.symm,
ennreal.rpow_one],
congr,
ext1 x,
rw [ennreal.coe_rpow_of_nonneg _ ennreal.to_real_nonneg, real.nnnorm_of_nonneg],
congr
end

end measure_theory

open measure_theory
Expand Down

0 comments on commit f28023e

Please sign in to comment.