Skip to content

Commit 10c93ae

Browse files
committed
1 parent 45eb7f2 commit 10c93ae

File tree

3 files changed

+43
-17
lines changed

3 files changed

+43
-17
lines changed

Mathlib/Analysis/Calculus/FDeriv/Basic.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Jeremy Avigad, Sébastien Gouëzel, Yury Kudryashov
55
66
! This file was ported from Lean 3 source module analysis.calculus.fderiv.basic
7-
! leanprover-community/mathlib commit 3a69562db5a458db8322b190ec8d9a8bbd8a5b14
7+
! leanprover-community/mathlib commit 41bef4ae1254365bc190aee63b947674d2977f01
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/
@@ -763,8 +763,7 @@ set_option linter.uppercaseLean3 false in
763763
theorem HasFDerivAtFilter.isBigO_sub_rev (hf : HasFDerivAtFilter f f' x L) {C}
764764
(hf' : AntilipschitzWith C f') : (fun x' => x' - x) =O[L] fun x' => f x' - f x :=
765765
have : (fun x' => x' - x) =O[L] fun x' => f' (x' - x) :=
766-
isBigO_iff.2
767-
⟨C, eventually_of_forall fun _ => AddMonoidHomClass.bound_of_antilipschitz f' hf' _⟩
766+
isBigO_iff.2 ⟨C, eventually_of_forall fun _ => ZeroHomClass.bound_of_antilipschitz f' hf' _⟩
768767
(this.trans (hf.trans_isBigO this).right_isBigO_add).congr (fun _ => rfl) fun _ =>
769768
sub_add_cancel _ _
770769
set_option linter.uppercaseLean3 false in

Mathlib/Analysis/Normed/Group/Basic.lean

Lines changed: 39 additions & 12 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Patrick Massot, Johannes Hölzl, Yaël Dillies
55
66
! This file was ported from Lean 3 source module analysis.normed.group.basic
7-
! leanprover-community/mathlib commit 195fcd60ff2bfe392543bceb0ec2adcdb472db4c
7+
! leanprover-community/mathlib commit 41bef4ae1254365bc190aee63b947674d2977f01
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/
@@ -547,11 +547,11 @@ theorem norm_div_le_of_le {r₁ r₂ : ℝ} (H₁ : ‖a₁‖ ≤ r₁) (H₂ :
547547
#align norm_div_le_of_le norm_div_le_of_le
548548
#align norm_sub_le_of_le norm_sub_le_of_le
549549

550-
@[to_additive]
551-
theorem dist_le_norm_mul_norm (a b : E) : dist a b ≤ ‖a‖ + ‖b‖ := by
550+
@[to_additive dist_le_norm_add_norm]
551+
theorem dist_le_norm_add_norm' (a b : E) : dist a b ≤ ‖a‖ + ‖b‖ := by
552552
rw [dist_eq_norm_div]
553553
apply norm_div_le
554-
#align dist_le_norm_mul_norm dist_le_norm_mul_norm
554+
#align dist_le_norm_add_norm' dist_le_norm_add_norm'
555555
#align dist_le_norm_add_norm dist_le_norm_add_norm
556556

557557
@[to_additive abs_norm_sub_norm_le]
@@ -1010,12 +1010,39 @@ theorem MonoidHomClass.antilipschitz_of_bound [MonoidHomClass 𝓕 E F] (f :
10101010
#align monoid_hom_class.antilipschitz_of_bound MonoidHomClass.antilipschitz_of_bound
10111011
#align add_monoid_hom_class.antilipschitz_of_bound AddMonoidHomClass.antilipschitz_of_bound
10121012

1013-
@[to_additive]
1014-
theorem MonoidHomClass.bound_of_antilipschitz [MonoidHomClass 𝓕 E F] (f : 𝓕) {K : ℝ≥0}
1015-
(h : AntilipschitzWith K f) (x) : ‖x‖ ≤ K * ‖f x‖ := by
1016-
simpa only [dist_one_right, map_one] using h.le_mul_dist x 1
1017-
#align monoid_hom_class.bound_of_antilipschitz MonoidHomClass.bound_of_antilipschitz
1018-
#align add_monoid_hom_class.bound_of_antilipschitz AddMonoidHomClass.bound_of_antilipschitz
1013+
@[to_additive LipschitzWith.norm_le_mul]
1014+
theorem LipschitzWith.norm_le_mul' {f : E → F} {K : ℝ≥0} (h : LipschitzWith K f) (hf : f 1 = 1)
1015+
(x) : ‖f x‖ ≤ K * ‖x‖ := by simpa only [dist_one_right, hf] using h.dist_le_mul x 1
1016+
#align lipschitz_with.norm_le_mul' LipschitzWith.norm_le_mul'
1017+
#align lipschitz_with.norm_le_mul LipschitzWith.norm_le_mul
1018+
1019+
@[to_additive LipschitzWith.nnorm_le_mul]
1020+
theorem LipschitzWith.nnorm_le_mul' {f : E → F} {K : ℝ≥0} (h : LipschitzWith K f) (hf : f 1 = 1)
1021+
(x) : ‖f x‖₊ ≤ K * ‖x‖₊ :=
1022+
h.norm_le_mul' hf x
1023+
#align lipschitz_with.nnorm_le_mul' LipschitzWith.nnorm_le_mul'
1024+
#align lipschitz_with.nnorm_le_mul LipschitzWith.nnorm_le_mul
1025+
1026+
@[to_additive AntilipschitzWith.le_mul_norm]
1027+
theorem AntilipschitzWith.le_mul_norm' {f : E → F} {K : ℝ≥0} (h : AntilipschitzWith K f)
1028+
(hf : f 1 = 1) (x) : ‖x‖ ≤ K * ‖f x‖ := by
1029+
simpa only [dist_one_right, hf] using h.le_mul_dist x 1
1030+
#align antilipschitz_with.le_mul_norm' AntilipschitzWith.le_mul_norm'
1031+
#align antilipschitz_with.le_mul_norm AntilipschitzWith.le_mul_norm
1032+
1033+
@[to_additive AntilipschitzWith.le_mul_nnnorm]
1034+
theorem AntilipschitzWith.le_mul_nnnorm' {f : E → F} {K : ℝ≥0} (h : AntilipschitzWith K f)
1035+
(hf : f 1 = 1) (x) : ‖x‖₊ ≤ K * ‖f x‖₊ :=
1036+
h.le_mul_norm' hf x
1037+
#align antilipschitz_with.le_mul_nnnorm' AntilipschitzWith.le_mul_nnnorm'
1038+
#align antilipschitz_with.le_mul_nnnorm AntilipschitzWith.le_mul_nnnorm
1039+
1040+
@[to_additive]
1041+
theorem OneHomClass.bound_of_antilipschitz [OneHomClass 𝓕 E F] (f : 𝓕) {K : ℝ≥0}
1042+
(h : AntilipschitzWith K f) (x) : ‖x‖ ≤ K * ‖f x‖ :=
1043+
h.le_mul_nnnorm' (map_one f) x
1044+
#align one_hom_class.bound_of_antilipschitz OneHomClass.bound_of_antilipschitz
1045+
#align zero_hom_class.bound_of_antilipschitz ZeroHomClass.bound_of_antilipschitz
10191046

10201047
end NNNorm
10211048

@@ -1905,11 +1932,11 @@ theorem mul_div_lipschitzWith (hf : AntilipschitzWith Kf f) (hg : LipschitzWith
19051932
#align antilipschitz_with.mul_div_lipschitz_with AntilipschitzWith.mul_div_lipschitzWith
19061933
#align antilipschitz_with.add_sub_lipschitz_with AntilipschitzWith.add_sub_lipschitzWith
19071934

1908-
@[to_additive]
1935+
@[to_additive le_mul_norm_sub]
19091936
theorem le_mul_norm_div {f : E → F} (hf : AntilipschitzWith K f) (x y : E) :
19101937
‖x / y‖ ≤ K * ‖f x / f y‖ := by simp [← dist_eq_norm_div, hf.le_mul_dist x y]
19111938
#align antilipschitz_with.le_mul_norm_div AntilipschitzWith.le_mul_norm_div
1912-
#align antilipschitz_with.le_add_norm_sub AntilipschitzWith.le_add_norm_sub
1939+
#align antilipschitz_with.le_mul_norm_sub AntilipschitzWith.le_mul_norm_sub
19131940

19141941
end AntilipschitzWith
19151942

Mathlib/Analysis/NormedSpace/ContinuousLinearMap.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Jan-David Salchow, Sébastien Gouëzel, Jean Lo
55
66
! This file was ported from Lean 3 source module analysis.normed_space.continuous_linear_map
7-
! leanprover-community/mathlib commit 6285167a053ad0990fc88e56c48ccd9fae6550eb
7+
! leanprover-community/mathlib commit 41bef4ae1254365bc190aee63b947674d2977f01
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/
@@ -142,7 +142,7 @@ theorem antilipschitz_of_bound (f : E →SL[σ] F) {K : ℝ≥0} (h : ∀ x, ‖
142142

143143
theorem bound_of_antilipschitz (f : E →SL[σ] F) {K : ℝ≥0} (h : AntilipschitzWith K f) (x) :
144144
‖x‖ ≤ K * ‖f x‖ :=
145-
AddMonoidHomClass.bound_of_antilipschitz _ h x
145+
ZeroHomClass.bound_of_antilipschitz _ h x
146146
#align continuous_linear_map.bound_of_antilipschitz ContinuousLinearMap.bound_of_antilipschitz
147147

148148
end ContinuousLinearMap

0 commit comments

Comments
 (0)