src/HOL/HOLCF/Deflation.thy
changeset 46868 6c250adbe101
parent 42151 4da4fc77664b
child 58880 0baae4311a9f
--- a/src/HOL/HOLCF/Deflation.thy	Sun Mar 11 13:39:16 2012 +0100
+++ b/src/HOL/HOLCF/Deflation.thy	Sun Mar 11 13:54:08 2012 +0100
@@ -379,9 +379,9 @@
     by simp
 qed
 
-locale pcpo_ep_pair = ep_pair +
-  constrains e :: "'a::pcpo \<rightarrow> 'b::pcpo"
-  constrains p :: "'b::pcpo \<rightarrow> 'a::pcpo"
+locale pcpo_ep_pair = ep_pair e p
+  for e :: "'a::pcpo \<rightarrow> 'b::pcpo"
+  and p :: "'b::pcpo \<rightarrow> 'a::pcpo"
 begin
 
 lemma e_strict [simp]: "e\<cdot>\<bottom> = \<bottom>"