src/HOLCF/Pcpo.thy
changeset 29634 2baf1b2f6655
parent 29614 1f7b1b0df292
child 31024 0fdf666e08bf
--- a/src/HOLCF/Pcpo.thy	Mon Jan 26 22:14:51 2009 +0100
+++ b/src/HOLCF/Pcpo.thy	Mon Jan 26 22:15:35 2009 +0100
@@ -14,7 +14,7 @@
 
 class cpo = po +
         -- {* class axiom: *}
-  assumes cpo:   "chain S \<Longrightarrow> \<exists>x. range S <<| x"
+  assumes cpo:   "chain S \<Longrightarrow> \<exists>x :: 'a::po. range S <<| x"
 
 text {* in cpo's everthing equal to THE lub has lub properties for every chain *}
 
@@ -257,10 +257,10 @@
 class finite_po = finite + po
 
 class chfin = po +
-  assumes chfin: "chain Y \<Longrightarrow> \<exists>n. max_in_chain n Y"
+  assumes chfin: "chain Y \<Longrightarrow> \<exists>n. max_in_chain n (Y :: nat => 'a::po)"
 
 class flat = pcpo +
-  assumes ax_flat: "x \<sqsubseteq> y \<Longrightarrow> (x = \<bottom>) \<or> (x = y)"
+  assumes ax_flat: "(x :: 'a::pcpo) \<sqsubseteq> y \<Longrightarrow> x = \<bottom> \<or> x = y"
 
 text {* finite partial orders are chain-finite *}