src/HOL/HOL.thy
changeset 5305 513925de8962
parent 5186 439e292b5b87
child 5492 d9fc3457554e
--- a/src/HOL/HOL.thy	Wed Aug 12 16:21:18 1998 +0200
+++ b/src/HOL/HOL.thy	Wed Aug 12 16:23:25 1998 +0200
@@ -47,7 +47,6 @@
 
   (* Infixes *)
 
-  o             :: ['b => 'c, 'a => 'b, 'a] => 'c   (infixl 55)
   "="           :: ['a, 'a] => bool                 (infixl 50)
   "&"           :: [bool, bool] => bool             (infixr 35)
   "|"           :: [bool, bool] => bool             (infixr 30)
@@ -180,7 +179,6 @@
 defs
   (*misc definitions*)
   Let_def       "Let s f == f(s)"
-  o_def         "(f::'b=>'c) o g == (%(x::'a). f(g(x)))"
   if_def        "If P x y == @z::'a. (P=True --> z=x) & (P=False --> z=y)"
 
   (*arbitrary is completely unspecified, but is made to appear as a