avoid using Int.succ_def in proofs
authorhuffman
Fri, 24 Feb 2012 16:59:20 +0100
changeset 46655 be76913ec1a4
parent 46654 134b74908a8e
child 46656 5ba230f8232f
avoid using Int.succ_def in proofs
src/HOL/Word/Bool_List_Representation.thy
--- a/src/HOL/Word/Bool_List_Representation.thy	Fri Feb 24 16:55:29 2012 +0100
+++ b/src/HOL/Word/Bool_List_Representation.thy	Fri Feb 24 16:59:20 2012 +0100
@@ -790,7 +790,7 @@
   apply (case_tac binb rule: bin_exhaust)
   apply (case_tac b)
    apply (case_tac [!] "ba")
-     apply (auto simp: rbl_succ succ_def bin_to_bl_aux_alt Let_def add_ac)
+     apply (auto simp: rbl_succ bin_to_bl_aux_alt Let_def add_ac)
   done
 
 lemma rbl_add_app2: