src/HOLCF/LowerPD.thy
changeset 37770 cddb3106adb8
parent 36635 080b755377c0
child 39970 9023b897e67a
--- a/src/HOLCF/LowerPD.thy	Mon Jul 12 11:21:56 2010 +0200
+++ b/src/HOLCF/LowerPD.thy	Mon Jul 12 11:39:27 2010 +0200
@@ -234,7 +234,7 @@
   "approx n\<cdot>(xs +\<flat> ys) = (approx n\<cdot>xs) +\<flat> (approx n\<cdot>ys)"
 by (induct xs ys rule: lower_pd.principal_induct2, simp, simp, simp)
 
-interpretation lower_add!: semilattice lower_add proof
+interpretation lower_add: semilattice lower_add proof
   fix xs ys zs :: "'a lower_pd"
   show "(xs +\<flat> ys) +\<flat> zs = xs +\<flat> (ys +\<flat> zs)"
     apply (induct xs ys arbitrary: zs rule: lower_pd.principal_induct2, simp, simp)