src/HOLCF/Pcpo.thy
changeset 2640 ee4dfce170a0
parent 2394 91d8abf108be
child 3326 930c9bed5a09
--- a/src/HOLCF/Pcpo.thy	Sat Feb 15 18:24:05 1997 +0100
+++ b/src/HOLCF/Pcpo.thy	Mon Feb 17 10:57:11 1997 +0100
@@ -1,22 +1,31 @@
+(*  Title:      HOLCF/Pcpo.thy
+    ID:         $Id$
+    Author:     Franz Regensburger
+    Copyright   1993 Technische Universitaet Muenchen
+
+introduction of the classes cpo and pcpo 
+*)
 Pcpo = Porder +
 
-classes pcpo < po
+(* The class cpo of chain complete partial orders *)
+(* ********************************************** *)
+axclass cpo < po
+        (* class axiom: *)
+  cpo   "is_chain S ==> ? x. range(S) <<| (x::'a::po)" 
 
-arities void :: pcpo
+(* The class pcpo of pointed cpos *)
+(* ****************************** *)
+axclass pcpo < cpo
+
+  least         "? x.!y.x<<y"
 
 consts
-
-  UU		:: "'a::pcpo"        
+  UU            :: "'a::pcpo"        
 
 syntax (symbols)
-
-  UU		:: "'a::pcpo"				("\\<bottom>")
-
-rules
+  UU            :: "'a::pcpo"                           ("\\<bottom>")
 
-  minimal	"UU << x"       
-  cpo		"is_chain S ==> ? x. range(S) <<| (x::'a::pcpo)" 
-
-inst_void_pcpo  "(UU::void) = UU_void"
+defs
+  UU_def        "UU == @x.!y.x<<y"       
 
 end