src/HOL/HOLCF/LowerPD.thy
changeset 41430 1aa23e9f2c87
parent 41402 b647212cee03
child 41479 655f583840d0
--- a/src/HOL/HOLCF/LowerPD.thy	Tue Jan 04 15:03:27 2011 -0800
+++ b/src/HOL/HOLCF/LowerPD.thy	Tue Jan 04 15:32:56 2011 -0800
@@ -116,7 +116,7 @@
 by intro_classes (fast intro: lower_pd_minimal)
 
 lemma inst_lower_pd_pcpo: "\<bottom> = lower_principal (PDUnit compact_bot)"
-by (rule lower_pd_minimal [THEN UU_I, symmetric])
+by (rule lower_pd_minimal [THEN bottomI, symmetric])
 
 
 subsection {* Monadic unit and plus *}
@@ -240,8 +240,8 @@
 lemma lower_plus_bottom_iff [simp]:
   "xs \<union>\<flat> ys = \<bottom> \<longleftrightarrow> xs = \<bottom> \<and> ys = \<bottom>"
 apply safe
-apply (rule UU_I, erule subst, rule lower_plus_below1)
-apply (rule UU_I, erule subst, rule lower_plus_below2)
+apply (rule bottomI, erule subst, rule lower_plus_below1)
+apply (rule bottomI, erule subst, rule lower_plus_below2)
 apply (rule lower_plus_absorb)
 done