src/HOLCF/Bifinite.thy
changeset 29614 1f7b1b0df292
parent 29252 ea97aa6aeba2
child 30729 461ee3e49ad3
--- a/src/HOLCF/Bifinite.thy	Thu Jan 22 09:04:45 2009 +0100
+++ b/src/HOLCF/Bifinite.thy	Thu Jan 22 09:04:46 2009 +0100
@@ -10,7 +10,7 @@
 
 subsection {* Omega-profinite and bifinite domains *}
 
-class profinite = cpo +
+class profinite =
   fixes approx :: "nat \<Rightarrow> 'a \<rightarrow> 'a"
   assumes chain_approx [simp]: "chain approx"
   assumes lub_approx_app [simp]: "(\<Squnion>i. approx i\<cdot>x) = x"