src/HOL/Word/Bool_List_Representation.thy
changeset 57514 bdc2c6b40bf2
parent 57492 74bf65a1910a
child 58410 6d46ad54a2ab
--- a/src/HOL/Word/Bool_List_Representation.thy	Sat Jul 05 10:09:01 2014 +0200
+++ b/src/HOL/Word/Bool_List_Representation.thy	Sat Jul 05 11:01:53 2014 +0200
@@ -783,7 +783,7 @@
   apply (case_tac binb rule: bin_exhaust)
   apply (case_tac b)
    apply (case_tac [!] "ba")
-     apply (auto simp: rbl_succ bin_to_bl_aux_alt Let_def add_ac)
+     apply (auto simp: rbl_succ bin_to_bl_aux_alt Let_def ac_simps)
   done
 
 lemma rbl_add_app2: 
@@ -1021,7 +1021,7 @@
    apply (erule allE)
    apply (erule (1) impE)
    apply (drule bin_nth_split, erule conjE, erule allE,
-          erule trans, simp add : add_ac)+
+          erule trans, simp add : ac_simps)+
   done
 
 lemma bin_rsplit_all: