src/HOL/Analysis/Lipschitz.thy
changeset 68240 fa63bde6d659
parent 67979 53323937ee25
child 68838 5e013478bced
equal deleted inserted replaced
68239:0764ee22a4d1 68240:fa63bde6d659
   812   have lipschitz: "B-lipschitz_on (cball x (min u v) \<inter> X) (f s)" if s: "s \<in> cball t v" for s
   812   have lipschitz: "B-lipschitz_on (cball x (min u v) \<inter> X) (f s)" if s: "s \<in> cball t v" for s
   813   proof -
   813   proof -
   814     note s
   814     note s
   815     also note \<open>cball t v \<subseteq> T\<close>
   815     also note \<open>cball t v \<subseteq> T\<close>
   816     finally
   816     finally
   817     have deriv: "\<forall>y\<in>cball x u. (f s has_derivative blinfun_apply (f' (s, y))) (at y within cball x u)"
   817     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)"
   818       using \<open>_ \<subseteq> X\<close>
   818       using \<open>_ \<subseteq> X\<close>
   819       by (auto intro!: has_derivative_at_withinI[OF f'])
   819       by (auto intro!: has_derivative_at_withinI[OF f'])
   820     have "norm (f s y - f s z) \<le> B * norm (y - z)"
   820     have "norm (f s y - f s z) \<le> B * norm (y - z)"
   821       if "y \<in> cball x u" "z \<in> cball x u"
   821       if "y \<in> cball x u" "z \<in> cball x u"
   822       for y z
   822       for y z