Skip to content

Commit

Permalink
chore(analysis/mean_inequalities_pow): weaken assumptions on rpow_add…
Browse files Browse the repository at this point in the history
…_le_rpow (#15823)
  • Loading branch information
ericrbg committed Aug 4, 2022
1 parent 20f68fc commit 7eaf341
Show file tree
Hide file tree
Showing 3 changed files with 11 additions and 4 deletions.
11 changes: 9 additions & 2 deletions src/analysis/mean_inequalities_pow.lean
Original file line number Diff line number Diff line change
Expand Up @@ -172,9 +172,11 @@ begin
rwa one_div_div at h_rpow_add_rpow_le_add,
end

lemma rpow_add_le_add_rpow {p : ℝ} (a b : ℝ≥0) (hp_pos : 0 < p) (hp1 : p ≤ 1) :
lemma rpow_add_le_add_rpow {p : ℝ} (a b : ℝ≥0) (hp : 0 p) (hp1 : p ≤ 1) :
(a + b) ^ p ≤ a ^ p + b ^ p :=
begin
rcases hp.eq_or_lt with rfl|hp_pos,
{ simp },
have h := rpow_add_rpow_le a b hp_pos hp1,
rw one_div_one at h,
repeat { rw nnreal.rpow_one at h },
Expand Down Expand Up @@ -286,9 +288,14 @@ begin
rwa one_div_div at h_rpow_add_rpow_le_add,
end

lemma rpow_add_le_add_rpow {p : ℝ} (a b : ℝ≥0∞) (hp_pos : 0 < p) (hp1 : p ≤ 1) :
lemma rpow_add_le_add_rpow {p : ℝ} (a b : ℝ≥0∞) (hp : 0 p) (hp1 : p ≤ 1) :
(a + b) ^ p ≤ a ^ p + b ^ p :=
begin
rcases hp.eq_or_lt with rfl|hp_pos,
{ suffices : (1 : ℝ≥0∞) ≤ 1 + 1,
{ simpa using this },
norm_cast,
norm_num },
have h := rpow_add_rpow_le a b hp_pos hp1,
rw one_div_one at h,
repeat { rw ennreal.rpow_one at h },
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/lp_space.lean
Original file line number Diff line number Diff line change
Expand Up @@ -229,7 +229,7 @@ begin
{ refine (real.rpow_le_rpow (norm_nonneg _) (norm_add_le _ _) hp.le).trans _,
dsimp [C],
split_ifs with h h,
{ simpa using nnreal.coe_le_coe.2 (nnreal.rpow_add_le_add_rpow (∥f i∥₊) (∥g i∥₊) hp h.le) },
{ simpa using nnreal.coe_le_coe.2 (nnreal.rpow_add_le_add_rpow (∥f i∥₊) (∥g i∥₊) hp.le h.le) },
{ let F : fin 2 → ℝ≥0 := ![∥f i∥₊, ∥g i∥₊],
have : ∀ i, (0:ℝ) ≤ F i := λ i, (F i).coe_nonneg,
simp only [not_lt] at h,
Expand Down
2 changes: 1 addition & 1 deletion src/measure_theory/function/lp_space.lean
Original file line number Diff line number Diff line change
Expand Up @@ -760,7 +760,7 @@ end
... ≤ (∫⁻ a, (∥f a∥₊ : ℝ≥0∞) ^ q + (∥g a∥₊ : ℝ≥0∞) ^ q ∂μ) ^ (1 / q) :
begin
refine ennreal.rpow_le_rpow (lintegral_mono (λ a, _)) (by simp [hq_pos.le] : 01 / q),
exact ennreal.rpow_add_le_add_rpow _ _ hq_pos hq1,
exact ennreal.rpow_add_le_add_rpow _ _ hq_pos.le hq1,
end
... < ∞ :
begin
Expand Down

0 comments on commit 7eaf341

Please sign in to comment.