removed unused lemmas
authorhuffman
Tue, 27 Dec 2011 12:49:03 +0100
changeset 45999 cce7e6197a46
parent 45998 d7cc533ae60d
child 46000 871bdab23f5c
removed unused lemmas
src/HOL/Word/Bit_Representation.thy
--- a/src/HOL/Word/Bit_Representation.thy	Tue Dec 27 12:37:11 2011 +0100
+++ b/src/HOL/Word/Bit_Representation.thy	Tue Dec 27 12:49:03 2011 +0100
@@ -561,11 +561,6 @@
 lemmas bintrunc_Min_minus_I = bmsts(2)
 lemmas bintrunc_BIT_minus_I = bmsts(3)
 
-lemma bintrunc_0_Min: "bintrunc 0 Int.Min = Int.Pls"
-  by (fact bintrunc.Z) (* FIXME: delete *)
-lemma bintrunc_0_BIT: "bintrunc 0 (w BIT b) = Int.Pls"
-  by (fact bintrunc.Z) (* FIXME: delete *)
-
 lemma bintrunc_Suc_lem:
   "bintrunc (Suc n) x = y ==> m = Suc n ==> bintrunc m x = y"
   by auto