tuned prefix of ac rules
authorhaftmann
Thu, 11 Mar 2010 15:52:35 +0100
changeset 35732 3b17dff14c4f
parent 35731 1bdaa24fb56d
child 35733 b57070d54cd5
tuned prefix of ac rules
src/HOL/ex/Summation.thy
--- a/src/HOL/ex/Summation.thy	Thu Mar 11 15:52:35 2010 +0100
+++ b/src/HOL/ex/Summation.thy	Thu Mar 11 15:52:35 2010 +0100
@@ -10,7 +10,7 @@
 
 lemma add_setsum_orient:
   "setsum f {k..<j} + setsum f {l..<k} = setsum f {l..<k} + setsum f {k..<j}"
-  by (fact plus.commute)
+  by (fact add.commute)
 
 lemma add_setsum_int:
   fixes j k l :: int