Skip to content

Commit b1ccddb

Browse files
committed
replace a failing grind with norm_num; it's been minimized and reported elsewhere
1 parent a9faeaa commit b1ccddb

File tree

1 file changed

+6
-1
lines changed

1 file changed

+6
-1
lines changed

Mathlib/Analysis/Normed/Module/Convex.lean

Lines changed: 6 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -77,7 +77,12 @@ theorem convexHull_sphere_eq_closedBall [Nontrivial F] (x : F) {r : ℝ} (hr : 0
7777
refine subset_antisymm (convexHull_min sphere_subset_closedBall (convex_closedBall 0 r))
7878
(fun x h ↦ mem_convexHull_iff.mpr fun U hU_sub hU ↦ ?_)
7979
have zero_mem : (0 : F) ∈ U := by
80-
have _ : Invertible (2 : ℝ) := by use 2⁻¹ <;> grind
80+
#adaptation_note
81+
/--
82+
This `norm_num` was `grind` until nightly-2025-11-26.
83+
The problem has been minmized as https://github.com/leanprover/lean4/pull/11410
84+
-/
85+
have _ : Invertible (2 : ℝ) := by use 2⁻¹ <;> norm_num
8186
obtain ⟨z, hz⟩ := NormedSpace.sphere_nonempty (E := F).mpr hr
8287
rw [← midpoint_self_neg (R := ℝ) (x := z)]
8388
exact Convex.midpoint_mem hU (hU_sub hz) <| hU_sub (by simp_all)

0 commit comments

Comments
 (0)