remove unused lemmas
authorhuffman
Thu, 23 Feb 2012 14:43:01 +0100
changeset 46606 7a5c05b5f945
parent 46605 b2563f7cf844
child 46607 6ae8121448af
remove unused lemmas
src/HOL/Word/Bit_Representation.thy
--- a/src/HOL/Word/Bit_Representation.thy	Thu Feb 23 14:29:29 2012 +0100
+++ b/src/HOL/Word/Bit_Representation.thy	Thu Feb 23 14:43:01 2012 +0100
@@ -111,12 +111,6 @@
   apply (simp add: z1pmod2)
   done
 
-lemma B1_mod_2 [simp]: "(Int.Bit1 w) mod 2 = 1"
-  unfolding numeral_simps number_of_is_id by (simp add: z1pmod2)
-
-lemma B0_mod_2 [simp]: "(Int.Bit0 w) mod 2 = 0"
-  unfolding numeral_simps number_of_is_id by simp
-
 lemma neB1E [elim!]:
   assumes ne: "y \<noteq> (1::bit)"
   assumes y: "y = (0::bit) \<Longrightarrow> P"