src/HOL/Word/Bit_Int.thy
changeset 46605 b2563f7cf844
parent 46604 9f9e85264e4d
child 46608 37e383cc7831
--- a/src/HOL/Word/Bit_Int.thy	Thu Feb 23 13:16:18 2012 +0100
+++ b/src/HOL/Word/Bit_Int.thy	Thu Feb 23 14:29:29 2012 +0100
@@ -375,18 +375,14 @@
   "bin_sc n 0 w <= w"
   apply (induct n arbitrary: w)
    apply (case_tac [!] w rule: bin_exhaust)
-   apply (auto simp del: BIT_simps)
-   apply (unfold Bit_def)
-   apply (simp_all add: bitval_def split: bit.split)
+   apply (auto simp: le_Bits)
   done
 
 lemma bin_set_ge:
   "bin_sc n 1 w >= w"
   apply (induct n arbitrary: w)
    apply (case_tac [!] w rule: bin_exhaust)
-   apply (auto simp del: BIT_simps)
-   apply (unfold Bit_def)
-   apply (simp_all add: bitval_def split: bit.split)
+   apply (auto simp: le_Bits)
   done
 
 lemma bintr_bin_clr_le:
@@ -395,9 +391,7 @@
    apply simp
   apply (case_tac w rule: bin_exhaust)
   apply (case_tac m)
-   apply (auto simp del: BIT_simps)
-   apply (unfold Bit_def)
-   apply (simp_all add: bitval_def split: bit.split)
+   apply (auto simp: le_Bits)
   done
 
 lemma bintr_bin_set_ge:
@@ -406,9 +400,7 @@
    apply simp
   apply (case_tac w rule: bin_exhaust)
   apply (case_tac m)
-   apply (auto simp del: BIT_simps)
-   apply (unfold Bit_def)
-   apply (simp_all add: bitval_def split: bit.split)
+   apply (auto simp: le_Bits)
   done
 
 lemma bin_sc_FP [simp]: "bin_sc n 0 Int.Pls = Int.Pls"