src/HOL/Lim.thy
changeset 45031 9583f2b56f85
parent 44571 bd91b77c4cd6
child 50331 4b6dc5077e98
--- a/src/HOL/Lim.thy	Tue Sep 20 15:23:17 2011 +0200
+++ b/src/HOL/Lim.thy	Tue Sep 20 10:52:08 2011 -0700
@@ -422,8 +422,7 @@
   assumes "\<forall>f. (\<forall>n. f n \<noteq> a) \<and> f ----> a \<longrightarrow>
     eventually (\<lambda>n. P (f n)) sequentially"
   shows "eventually P (at a)"
-  using assms sequentially_imp_eventually_within [where s=UNIV]
-  unfolding within_UNIV by simp
+  using assms sequentially_imp_eventually_within [where s=UNIV] by simp
 
 lemma LIMSEQ_SEQ_conv1:
   fixes f :: "'a::topological_space \<Rightarrow> 'b::topological_space"