src/HOL/HOLCF/Pcpo.thy
changeset 54863 82acc20ded73
parent 42151 4da4fc77664b
child 58880 0baae4311a9f
--- a/src/HOL/HOLCF/Pcpo.thy	Wed Dec 25 17:39:06 2013 +0100
+++ b/src/HOL/HOLCF/Pcpo.thy	Wed Dec 25 17:39:06 2013 +0100
@@ -118,8 +118,8 @@
     apply (rule lub_below [OF 2])
     apply (rule below_lub [OF 3])
     apply (rule below_trans)
-    apply (rule chain_mono [OF 1 le_maxI1])
-    apply (rule chain_mono [OF 2 le_maxI2])
+    apply (rule chain_mono [OF 1 max.cobounded1])
+    apply (rule chain_mono [OF 2 max.cobounded2])
     done
   show "(\<Squnion>i. Y i i) \<sqsubseteq> (\<Squnion>i. \<Squnion>j. Y i j)"
     apply (rule lub_mono [OF 3 4])