Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 930ae46

Browse files
committed
chore(analysis/special_functions/pow): remove duplicate lemmas concerning monotonicity of rpow (#10794)
The lemmas `rpow_left_monotone_of_nonneg` and `rpow_left_strict_mono_of_pos` were duplicates of `monotone_rpow_of_nonneg` and `strict_mono_rpow_of_pos`, respectively. The duplicates are removed as well as references to them in mathlib in `measure_theory/function/{continuous_function_dense, lp_space}`
1 parent 61949af commit 930ae46

File tree

3 files changed

+4
-10
lines changed

3 files changed

+4
-10
lines changed

src/analysis/special_functions/pow.lean

Lines changed: 0 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -1471,12 +1471,6 @@ lemma rpow_left_bijective {x : ℝ} (hx : x ≠ 0) :
14711471
function.bijective (λ y : ℝ≥0∞, y^x) :=
14721472
⟨rpow_left_injective hx, rpow_left_surjective hx⟩
14731473

1474-
lemma rpow_left_monotone_of_nonneg {x : ℝ} (hx : 0 ≤ x) : monotone (λ y : ℝ≥0∞, y^x) :=
1475-
λ y z hyz, rpow_le_rpow hyz hx
1476-
1477-
lemma rpow_left_strict_mono_of_pos {x : ℝ} (hx : 0 < x) : strict_mono (λ y : ℝ≥0∞, y^x) :=
1478-
λ y z hyz, rpow_lt_rpow hyz hx
1479-
14801474
theorem tendsto_rpow_at_top {y : ℝ} (hy : 0 < y) :
14811475
tendsto (λ (x : ℝ≥0∞), x ^ y) (𝓝 ⊤) (𝓝 ⊤) :=
14821476
begin

src/measure_theory/function/continuous_map_dense.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -143,7 +143,7 @@ begin
143143
{ refine (snorm_mono_ae (filter.eventually_of_forall gc_bd)).trans _,
144144
rw snorm_indicator_const (u_open.sdiff F_closed).measurable_set hp₀.ne' hp,
145145
push_cast [← ennreal.coe_rpow_of_nonneg _ hp₀'],
146-
exact ennreal.mul_left_mono (ennreal.rpow_left_monotone_of_nonneg hp₀' h_μ_sdiff) },
146+
exact ennreal.mul_left_mono (ennreal.monotone_rpow_of_nonneg hp₀' h_μ_sdiff) },
147147
have gc_cont : continuous (λ x, g x • c) := g.continuous.smul continuous_const,
148148
have gc_mem_ℒp : mem_ℒp (λ x, g x • c) p μ,
149149
{ have : mem_ℒp ((λ x, g x • c) - s.indicator (λ x, c)) p μ :=

src/measure_theory/function/lp_space.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -477,7 +477,7 @@ begin
477477
push_cast,
478478
rw real.norm_rpow_of_nonneg (norm_nonneg _), },
479479
rw h_rpow,
480-
have h_rpow_mono := ennreal.rpow_left_strict_mono_of_pos hq_pos,
480+
have h_rpow_mono := ennreal.strict_mono_rpow_of_pos hq_pos,
481481
have h_rpow_surj := (ennreal.rpow_left_bijective hq_pos.ne.symm).2,
482482
let iso := h_rpow_mono.order_iso_of_surjective _ h_rpow_surj,
483483
exact (iso.ess_sup_apply (λ x, ((nnnorm (f x)) : ℝ≥0∞)) μ).symm, },
@@ -2034,7 +2034,7 @@ begin
20342034
refine (lintegral_liminf_le' (λ m, ((hf m).ennnorm.pow_const _))).trans_eq _,
20352035
have h_pow_liminf : at_top.liminf (λ n, snorm' (f n) p μ) ^ p
20362036
= at_top.liminf (λ n, (snorm' (f n) p μ) ^ p),
2037-
{ have h_rpow_mono := ennreal.rpow_left_strict_mono_of_pos hp_pos,
2037+
{ have h_rpow_mono := ennreal.strict_mono_rpow_of_pos hp_pos,
20382038
have h_rpow_surj := (ennreal.rpow_left_bijective hp_pos.ne.symm).2,
20392039
refine (h_rpow_mono.order_iso_of_surjective _ h_rpow_surj).liminf_apply _ _ _ _,
20402040
all_goals { is_bounded_default }, },
@@ -2232,7 +2232,7 @@ begin
22322232
(nnnorm (f (i + 1) a - f i a)))^p ∂μ
22332233
= ∫⁻ a, at_top.liminf (λ n, (∑ i in finset.range (n + 1), (nnnorm (f (i + 1) a - f i a)))^p) ∂μ,
22342234
{ refine lintegral_congr (λ x, _),
2235-
have h_rpow_mono := ennreal.rpow_left_strict_mono_of_pos (zero_lt_one.trans_le hp1),
2235+
have h_rpow_mono := ennreal.strict_mono_rpow_of_pos (zero_lt_one.trans_le hp1),
22362236
have h_rpow_surj := (ennreal.rpow_left_bijective hp_pos.ne.symm).2,
22372237
refine (h_rpow_mono.order_iso_of_surjective _ h_rpow_surj).liminf_apply _ _ _ _,
22382238
all_goals { is_bounded_default }, },

0 commit comments

Comments
 (0)