src/FOL/IFOL.thy
changeset 21524 7843e2fd14a9
parent 21404 eb85850d3eb7
child 21539 c5cf9243ad62
--- a/src/FOL/IFOL.thy	Fri Nov 24 22:05:19 2006 +0100
+++ b/src/FOL/IFOL.thy	Sun Nov 26 18:07:16 2006 +0100
@@ -54,24 +54,23 @@
 notation (HTML output)
   not_equal  (infixl "\<noteq>" 50)
 
-syntax (xsymbols)
-  Not           :: "o => o"                     ("\<not> _" [40] 40)
-  "op &"        :: "[o, o] => o"                (infixr "\<and>" 35)
-  "op |"        :: "[o, o] => o"                (infixr "\<or>" 30)
-  "ALL "        :: "[idts, o] => o"             ("(3\<forall>_./ _)" [0, 10] 10)
-  "EX "         :: "[idts, o] => o"             ("(3\<exists>_./ _)" [0, 10] 10)
-  "EX! "        :: "[idts, o] => o"             ("(3\<exists>!_./ _)" [0, 10] 10)
-  "op -->"      :: "[o, o] => o"                (infixr "\<longrightarrow>" 25)
-  "op <->"      :: "[o, o] => o"                (infixr "\<longleftrightarrow>" 25)
+notation (xsymbols)
+  Not  ("\<not> _" [40] 40) and
+  "op &"  (infixr "\<and>" 35) and
+  "op |"  (infixr "\<or>" 30) and
+  All  (binder "\<forall>" 10) and
+  Ex  (binder "\<exists>" 10) and
+  Ex1  (binder "\<exists>!" 10) and
+  "op -->"  (infixr "\<longrightarrow>" 25) and
+  "op <->"  (infixr "\<longleftrightarrow>" 25)
 
-syntax (HTML output)
-  Not           :: "o => o"                     ("\<not> _" [40] 40)
-  "op &"        :: "[o, o] => o"                (infixr "\<and>" 35)
-  "op |"        :: "[o, o] => o"                (infixr "\<or>" 30)
-  "ALL "        :: "[idts, o] => o"             ("(3\<forall>_./ _)" [0, 10] 10)
-  "EX "         :: "[idts, o] => o"             ("(3\<exists>_./ _)" [0, 10] 10)
-  "EX! "        :: "[idts, o] => o"             ("(3\<exists>!_./ _)" [0, 10] 10)
-
+notation (HTML output)
+  Not  ("\<not> _" [40] 40) and
+  "op &"  (infixr "\<and>" 35) and
+  "op |"  (infixr "\<or>" 30) and
+  All  (binder "\<forall>" 10) and
+  Ex  (binder "\<exists>" 10) and
+  Ex1  (binder "\<exists>!" 10)
 
 local