src/HOL/Word/Bit_Int.thy
changeset 46608 37e383cc7831
parent 46605 b2563f7cf844
child 46609 5cb607cb7651
--- a/src/HOL/Word/Bit_Int.thy	Thu Feb 23 15:04:51 2012 +0100
+++ b/src/HOL/Word/Bit_Int.thy	Thu Feb 23 15:15:48 2012 +0100
@@ -403,11 +403,11 @@
    apply (auto simp: le_Bits)
   done
 
-lemma bin_sc_FP [simp]: "bin_sc n 0 Int.Pls = Int.Pls"
-  by (induct n) (auto simp: BIT_simps)
+lemma bin_sc_FP [simp]: "bin_sc n 0 0 = 0"
+  by (induct n) auto
 
-lemma bin_sc_TM [simp]: "bin_sc n 1 Int.Min = Int.Min"
-  by (induct n) (auto simp: BIT_simps)
+lemma bin_sc_TM [simp]: "bin_sc n 1 -1 = -1"
+  by (induct n) auto
   
 lemmas bin_sc_simps = bin_sc.Z bin_sc.Suc bin_sc_TM bin_sc_FP