src/HOLCF/LowerPD.thy
changeset 36635 080b755377c0
parent 35901 12f09bf2c77f
child 37770 cddb3106adb8
--- a/src/HOLCF/LowerPD.thy	Tue May 04 08:55:39 2010 +0200
+++ b/src/HOLCF/LowerPD.thy	Tue May 04 08:55:43 2010 +0200
@@ -393,7 +393,7 @@
     (\<lambda>x y. \<Lambda> f. x\<cdot>f +\<flat> y\<cdot>f)"
 
 lemma ACI_lower_bind:
-  "ab_semigroup_idem_mult (\<lambda>x y. \<Lambda> f. x\<cdot>f +\<flat> y\<cdot>f)"
+  "class.ab_semigroup_idem_mult (\<lambda>x y. \<Lambda> f. x\<cdot>f +\<flat> y\<cdot>f)"
 apply unfold_locales
 apply (simp add: lower_plus_assoc)
 apply (simp add: lower_plus_commute)