src/FOL/IFOL.thy
changeset 12662 a9bbba3473f3
parent 12368 2af9ad81ea56
child 12875 bda60442bf02
--- a/src/FOL/IFOL.thy	Tue Jan 08 00:03:10 2002 +0100
+++ b/src/FOL/IFOL.thy	Tue Jan 08 00:03:42 2002 +0100
@@ -43,7 +43,7 @@
 
 
 syntax
-  "~="          :: "['a, 'a] => o"              (infixl 50)
+  "_not_equal"  :: "['a, 'a] => o"              (infixl "~=" 50)
 translations
   "x ~= y"      == "~ (x = y)"
 
@@ -54,7 +54,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)
   "op -->"      :: "[o, o] => o"                (infixr "\<longrightarrow>" 25)
   "op <->"      :: "[o, o] => o"                (infixr "\<longleftrightarrow>" 25)