src/HOL/Lim.thy
changeset 31336 e17f13cd1280
parent 31017 2c227493ea56
child 31338 d41a8ba25b67
--- a/src/HOL/Lim.thy	Thu May 28 22:54:57 2009 -0700
+++ b/src/HOL/Lim.thy	Thu May 28 22:57:17 2009 -0700
@@ -700,7 +700,7 @@
     }
     then have "(\<forall>no. \<exists>n. no \<le> n \<and> norm (X (?F n) - L) \<ge> r)" by simp
     with rdef have "\<exists>e>0. (\<forall>no. \<exists>n. no \<le> n \<and> norm (X (?F n) - L) \<ge> e)" by auto
-    thus ?thesis by (unfold LIMSEQ_def, auto simp add: linorder_not_less)
+    thus ?thesis by (unfold LIMSEQ_iff, auto simp add: linorder_not_less)
   qed
   ultimately show False by simp
 qed