src/HOL/Analysis/Abstract_Limits.thy
changeset 71172 575b3a818de5
parent 70337 48609a6af1a0
child 77934 01c88cf514fc
--- a/src/HOL/Analysis/Abstract_Limits.thy	Thu Nov 28 20:38:07 2019 +0100
+++ b/src/HOL/Analysis/Abstract_Limits.thy	Thu Nov 28 23:06:22 2019 +0100
@@ -79,16 +79,16 @@
     have "\<forall>\<^sub>F b in F. f b \<in> topspace X \<inter> S"
       by (metis (no_types) limitin_def openin_topspace topspace_subtopology)
     with L show ?rhs
-      apply (clarsimp simp add: limitin_def eventually_mono topspace_subtopology openin_subtopology_alt)
+      apply (clarsimp simp add: limitin_def eventually_mono openin_subtopology_alt)
       apply (drule_tac x="S \<inter> U" in spec, force simp: elim: eventually_mono)
       done
   next
     assume ?rhs
     then show ?lhs
       using eventually_elim2
-      by (fastforce simp add: limitin_def topspace_subtopology openin_subtopology_alt)
+      by (fastforce simp add: limitin_def openin_subtopology_alt)
   qed
-qed (auto simp: limitin_def topspace_subtopology)
+qed (auto simp: limitin_def)
 
 
 lemma limitin_canonical_iff_gen [simp]: