We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 4481ab6 commit 42c6ec6Copy full SHA for 42c6ec6
Mathlib/Analysis/Normed/Operator/Banach.lean
@@ -130,7 +130,13 @@ theorem exists_approx_preimage_norm_le (surj : Surjective f) :
130
simp only [x, f.map_sub]
131
abel
132
_ ≤ ‖f x₁ - (a + d • y)‖ + ‖f x₂ - a‖ := norm_sub_le _ _
133
- _ ≤ 2 * δ := by grind [dist_eq_norm']
+ #adaptation_note
134
+ /--
135
+ These next two steps were `_ ≤ 2 * δ := by grind [dist_eq_norm']` until nightly-2025-11-28.
136
+ The problem is https://github.com/leanprover/lean4/pull/11410
137
+ -/
138
+ _ ≤ δ + δ := by rw [dist_eq_norm'] at h₁ h₂; gcongr
139
+ _ = 2 * δ := (two_mul _).symm
140
have J : ‖f (σ' d⁻¹ • x) - y‖ ≤ 1 / 2 * ‖y‖ :=
141
calc
142
‖f (σ' d⁻¹ • x) - y‖ = ‖d⁻¹ • f x - (d⁻¹ * d) • y‖ := by
0 commit comments