src/HOL/Fun.thy
changeset 19656 09be06943252
parent 19536 1a3a3cf8b4fa
child 20044 92cc2f4c7335
--- a/src/HOL/Fun.thy	Tue May 16 21:32:56 2006 +0200
+++ b/src/HOL/Fun.thy	Tue May 16 21:33:01 2006 +0200
@@ -48,17 +48,15 @@
   comp :: "['b => 'c, 'a => 'b, 'a] => 'c"   (infixl "o" 55)
   "f o g == %x. f(g(x))"
 
+const_syntax (xsymbols)
+  comp  (infixl "\<circ>" 55)
+
+const_syntax (HTML output)
+  comp  (infixl "\<circ>" 55)
+
 text{*compatibility*}
 lemmas o_def = comp_def
 
-abbreviation (xsymbols)
-  comp1  (infixl "\<circ>" 55)
-  "comp1 == comp"
-
-abbreviation (HTML output)
-  comp2  (infixl "\<circ>" 55)
-  "comp2 == comp"
-
 constdefs
   inj_on :: "['a => 'b, 'a set] => bool"         (*injective*)
   "inj_on f A == ! x:A. ! y:A. f(x)=f(y) --> x=y"