src/HOL/HOL.thy
changeset 20741 c8fdad2dc6e6
parent 20713 823967ef47f1
child 20766 9913d3bc3d17
--- a/src/HOL/HOL.thy	Wed Sep 27 21:44:38 2006 +0200
+++ b/src/HOL/HOL.thy	Wed Sep 27 21:49:34 2006 +0200
@@ -229,13 +229,13 @@
 end;
 *} -- {* show types that are presumably too general *}
 
-syntax
-  uminus :: "'a\<Colon>minus \<Rightarrow> 'a" ("- _" [81] 80)
+const_syntax
+  uminus  ("- _" [81] 80)
 
-syntax (xsymbols)
-  abs :: "'a::minus => 'a"    ("\<bar>_\<bar>")
-syntax (HTML output)
-  abs :: "'a::minus => 'a"    ("\<bar>_\<bar>")
+const_syntax (xsymbols)
+  abs  ("\<bar>_\<bar>")
+const_syntax (HTML output)
+  abs  ("\<bar>_\<bar>")
 
 
 subsection {*Equality*}