one last fix
authorpaulson <lp15@cam.ac.uk>
Sun, 20 May 2018 20:14:30 +0100
changeset 68240 fa63bde6d659
parent 68239 0764ee22a4d1
child 68241 39a311f50344
one last fix
src/HOL/Analysis/Lipschitz.thy
--- a/src/HOL/Analysis/Lipschitz.thy	Sun May 20 18:37:34 2018 +0100
+++ b/src/HOL/Analysis/Lipschitz.thy	Sun May 20 20:14:30 2018 +0100
@@ -814,7 +814,7 @@
     note s
     also note \<open>cball t v \<subseteq> T\<close>
     finally
-    have deriv: "\<forall>y\<in>cball x u. (f s has_derivative blinfun_apply (f' (s, y))) (at y within cball x u)"
+    have deriv: "\<And>y. y \<in> cball x u \<Longrightarrow> (f s has_derivative blinfun_apply (f' (s, y))) (at y within cball x u)"
       using \<open>_ \<subseteq> X\<close>
       by (auto intro!: has_derivative_at_withinI[OF f'])
     have "norm (f s y - f s z) \<le> B * norm (y - z)"