src/HOL/Library/Extended_Real.thy
changeset 61806 d2e62ae01cd8
parent 61738 c4f6031f1310
child 61810 3c5040d5694a
--- a/src/HOL/Library/Extended_Real.thy	Mon Dec 07 10:38:04 2015 +0100
+++ b/src/HOL/Library/Extended_Real.thy	Mon Dec 07 16:44:26 2015 +0000
@@ -2443,11 +2443,8 @@
   assume "open S" and "x \<in> S"
   then have S: "open S" "ereal x \<in> ereal ` S"
     by (simp_all add: inj_image_mem_iff)
-  have "\<forall>x. f x \<in> ereal ` S \<longrightarrow> real_of_ereal (f x) \<in> S"
-    by auto
-  from this lim[THEN topological_tendstoD, OF open_ereal, OF S]
   show "eventually (\<lambda>x. real_of_ereal (f x) \<in> S) net"
-    by (rule eventually_mono)
+    by (auto intro: eventually_mono' [OF lim[THEN topological_tendstoD, OF open_ereal, OF S]])
 qed
 
 lemma lim_ereal[simp]: "((\<lambda>n. ereal (f n)) ---> ereal x) net \<longleftrightarrow> (f ---> x) net"