src/HOLCF/Cfun1.thy
changeset 6382 8b0c9205da75
parent 5291 5706f0ef1d43
child 10834 a7897aebbffc
--- a/src/HOLCF/Cfun1.thy	Wed Mar 17 13:47:04 1999 +0100
+++ b/src/HOLCF/Cfun1.thy	Wed Mar 17 13:47:34 1999 +0100
@@ -1,9 +1,9 @@
-(*  Title:      HOLCF/cfun1.thy
+(*  Title:      HOLCF/Cfun1.thy
     ID:         $Id$
     Author:     Franz Regensburger
     Copyright   1993 Technische Universitaet Muenchen
 
-Definition of the type ->  of continuous functions
+Definition of the type ->  of continuous functions.
 
 *)
 
@@ -11,7 +11,7 @@
 
 default cpo
 
-typedef (CFun)  ('a, 'b) "->" (infixr 0) = "{f. cont f}" (CfunI)
+typedef (CFun)  ('a, 'b) "->" (infixr 0) = "{f::'a => 'b. cont f}" (CfunI)
 
 (* to make << defineable *)
 instance "->"  :: (cpo,cpo)sq_ord