src/HOL/Infinite_Set.thy
changeset 14565 c6dc17aab88a
parent 14485 ea2707645af8
child 14766 c0401da7726d
--- a/src/HOL/Infinite_Set.thy	Wed Apr 14 13:28:46 2004 +0200
+++ b/src/HOL/Infinite_Set.thy	Wed Apr 14 14:13:05 2004 +0200
@@ -359,6 +359,10 @@
   "MOST " :: "[idts, bool] \<Rightarrow> bool"       ("(3\<forall>\<^sub>\<infinity>_./ _)" [0,10] 10)
   "INF "    :: "[idts, bool] \<Rightarrow> bool"     ("(3\<exists>\<^sub>\<infinity>_./ _)" [0,10] 10)
 
+syntax (HTML output)
+  "MOST " :: "[idts, bool] \<Rightarrow> bool"       ("(3\<forall>\<^sub>\<infinity>_./ _)" [0,10] 10)
+  "INF "    :: "[idts, bool] \<Rightarrow> bool"     ("(3\<exists>\<^sub>\<infinity>_./ _)" [0,10] 10)
+
 lemma INF_EX:
   "(\<exists>\<^sub>\<infinity>x. P x) \<Longrightarrow> (\<exists>x. P x)"
 proof (unfold INF_def, rule ccontr)