src/HOLCF/LowerPD.thy
changeset 29672 07f3da9fd2a0
parent 29511 7071b017cb35
child 29990 b11793ea15a3
--- a/src/HOLCF/LowerPD.thy	Wed Jan 28 17:12:25 2009 +0100
+++ b/src/HOLCF/LowerPD.thy	Thu Jan 29 10:07:43 2009 +0100
@@ -258,9 +258,9 @@
 
 lemma lower_plus_left_absorb: "xs +\<flat> (xs +\<flat> ys) = xs +\<flat> ys"
 by (rule aci_lower_plus.mult_left_idem)
-
+(*
 lemmas lower_plus_aci = aci_lower_plus.mult_ac_idem
-
+*)
 lemma lower_plus_less1: "xs \<sqsubseteq> xs +\<flat> ys"
 apply (induct xs ys rule: lower_pd.principal_induct2, simp, simp)
 apply (simp add: PDPlus_lower_less)