src/HOLCF/Cfun.thy
changeset 40003 427106657e04
parent 40002 c5b5f7a3a3b1
child 40005 3e3611136a13
--- a/src/HOLCF/Cfun.thy	Mon Oct 11 21:35:31 2010 -0700
+++ b/src/HOLCF/Cfun.thy	Tue Oct 12 05:25:21 2010 -0700
@@ -600,10 +600,10 @@
 using f
 proof (rule cont2cont_Let)
   fix x show "cont (\<lambda>y. g x y)"
-    using g by (rule cont_fst_snd_D2)
+    using g by (simp add: prod_cont_iff)
 next
   fix y show "cont (\<lambda>x. g x y)"
-    using g by (rule cont_fst_snd_D1)
+    using g by (simp add: prod_cont_iff)
 qed
 
 text {* The simple version (suggested by Joachim Breitner) is needed if