src/HOLCF/Product_Cpo.thy
changeset 29533 7f4a32134447
parent 29531 2eb29775b0b6
child 29535 08824fad8879
--- a/src/HOLCF/Product_Cpo.thy	Wed Jan 14 18:05:05 2009 -0800
+++ b/src/HOLCF/Product_Cpo.thy	Wed Jan 14 18:18:48 2009 -0800
@@ -5,7 +5,7 @@
 header {* The cpo of cartesian products *}
 
 theory Product_Cpo
-imports Ffun
+imports Cont
 begin
 
 defaultsort cpo
@@ -192,12 +192,13 @@
   assumes f: "cont (\<lambda>x. f x)"
   assumes g: "cont (\<lambda>x. g x)"
   shows "cont (\<lambda>x. (f x, g x))"
-apply (rule cont2cont_app2 [OF cont2cont_lambda cont_pair2 g])
-apply (rule cont2cont_app2 [OF cont_const cont_pair1 f])
+apply (rule cont2cont_apply [OF _ cont_pair1 f])
+apply (rule cont2cont_apply [OF _ cont_pair2 g])
+apply (rule cont_const)
 done
 
-lemmas cont2cont_fst [cont2cont] = cont2cont_app3 [OF cont_fst]
+lemmas cont2cont_fst [cont2cont] = cont2cont_compose [OF cont_fst]
 
-lemmas cont2cont_snd [cont2cont] = cont2cont_app3 [OF cont_snd]
+lemmas cont2cont_snd [cont2cont] = cont2cont_compose [OF cont_snd]
 
 end