src/FOL/IFOL.thy
changeset 19656 09be06943252
parent 19380 b808efaa5828
child 19683 3620e494cef2
--- a/src/FOL/IFOL.thy	Tue May 16 21:32:56 2006 +0200
+++ b/src/FOL/IFOL.thy	Tue May 16 21:33:01 2006 +0200
@@ -49,13 +49,11 @@
   not_equal     :: "['a, 'a] => o"              (infixl "~=" 50)
   "x ~= y == ~ (x = y)"
 
-abbreviation (xsymbols)
-  not_equal1  (infixl "\<noteq>" 50)
-  "x \<noteq> y == ~ (x = y)"
+const_syntax (xsymbols)
+  not_equal  (infixl "\<noteq>" 50)
 
-abbreviation (HTML output)
-  not_equal2  (infixl "\<noteq>" 50)
-  "not_equal2 == not_equal"
+const_syntax (HTML output)
+  not_equal  (infixl "\<noteq>" 50)
 
 syntax (xsymbols)
   Not           :: "o => o"                     ("\<not> _" [40] 40)