src/HOL/Word/Bool_List_Representation.thy
changeset 46645 573aff6b9b0a
parent 46617 8c5d10d41391
child 46652 bec50f8b3727
--- a/src/HOL/Word/Bool_List_Representation.thy	Fri Feb 24 11:23:36 2012 +0100
+++ b/src/HOL/Word/Bool_List_Representation.thy	Fri Feb 24 13:25:21 2012 +0100
@@ -681,13 +681,13 @@
   by (simp add : bl_to_bin_app_cat)
 
 lemma mask_lem: "(bl_to_bin (True # replicate n False)) = 
-    Int.succ (bl_to_bin (replicate n True))"
+    (bl_to_bin (replicate n True)) + 1"
   apply (unfold bl_to_bin_def)
   apply (induct n)
-   apply (simp add: Int.succ_def)
+   apply simp
   apply (simp only: Suc_eq_plus1 replicate_add
                     append_Cons [symmetric] bl_to_bin_aux_append)
-  apply (simp add: BIT_simps)
+  apply (simp add: Bit_B0_2t Bit_B1_2t)
   done
 
 (* function bl_of_nth *)