src/Sequents/LK0.thy
changeset 12662 a9bbba3473f3
parent 12116 4027b15377a5
child 14565 c6dc17aab88a
--- a/src/Sequents/LK0.thy	Tue Jan 08 00:03:10 2002 +0100
+++ b/src/Sequents/LK0.thy	Tue Jan 08 00:03:42 2002 +0100
@@ -35,7 +35,7 @@
   Ex           :: ('a => o) => o     (binder "EX " 10)
 
 syntax
-  "~="          :: ['a, 'a] => o                (infixl 50)
+  "_not_equal" :: ['a, 'a] => o                (infixl "~=" 50)
 
 translations
   "x ~= y"      == "~ (x = y)"
@@ -49,7 +49,7 @@
   "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 ~="       :: ['a, 'a] => o        (infixl "\\<noteq>" 50)
+  "_not_equal"  :: ['a, 'a] => o        (infixl "\\<noteq>" 50)
 
 syntax (HTML output)
   Not           :: o => o               ("\\<not> _" [40] 40)