src/HOL/Filter.thy
changeset 61378 3e04c9ca001a
parent 61245 b77bf45efe21
child 61531 ab2e862263e7
--- a/src/HOL/Filter.thy	Fri Oct 09 19:51:20 2015 +0200
+++ b/src/HOL/Filter.thy	Fri Oct 09 20:26:03 2015 +0200
@@ -698,10 +698,6 @@
   Inf_many  (binder "\<exists>\<^sub>\<infinity>" 10) and
   Alm_all  (binder "\<forall>\<^sub>\<infinity>" 10)
 
-notation (HTML output)
-  Inf_many  (binder "\<exists>\<^sub>\<infinity>" 10) and
-  Alm_all  (binder "\<forall>\<^sub>\<infinity>" 10)
-
 lemma eventually_cofinite: "eventually P cofinite \<longleftrightarrow> finite {x. \<not> P x}"
   unfolding cofinite_def
 proof (rule eventually_Abs_filter, rule is_filter.intro)