src/HOL/Analysis/Derivative.thy
changeset 64287 d85d88722745
parent 64267 b9a1486e79be
child 64394 141e1ed8d5a0
--- a/src/HOL/Analysis/Derivative.thy	Tue Oct 18 12:01:54 2016 +0200
+++ b/src/HOL/Analysis/Derivative.thy	Tue Oct 18 15:55:53 2016 +0100
@@ -1922,7 +1922,7 @@
     using assms(1,2,3) by (rule has_derivative_sequence_lipschitz)
   have "\<exists>g. \<forall>x\<in>s. ((\<lambda>n. f n x) \<longlongrightarrow> g x) sequentially"
     apply (rule bchoice)
-    unfolding convergent_eq_cauchy
+    unfolding convergent_eq_Cauchy
   proof
     fix x
     assume "x \<in> s"