src/HOL/IMP/ACom.thy
changeset 57512 cc97b347b301
parent 54941 6d99745afe34
child 58249 180f1b3508ed
--- a/src/HOL/IMP/ACom.thy	Fri Jul 04 20:07:08 2014 +0200
+++ b/src/HOL/IMP/ACom.thy	Fri Jul 04 20:18:47 2014 +0200
@@ -104,7 +104,7 @@
 apply(induction c arbitrary: f p)
 apply (auto simp: anno_def nth_append nth_Cons numeral_eq_Suc shift_def
             split: nat.split)
-  apply (metis add_Suc_right add_diff_inverse nat_add_commute)
+  apply (metis add_Suc_right add_diff_inverse add.commute)
  apply(rule_tac f=f in arg_cong)
  apply arith
 apply (metis less_Suc_eq)