src/HOL/Word/Word.thy
changeset 46602 c71f3e9367bb
parent 46440 d4994e2e7364
child 46603 83a5160e6b4d
--- a/src/HOL/Word/Word.thy	Thu Feb 23 12:08:59 2012 +0100
+++ b/src/HOL/Word/Word.thy	Thu Feb 23 12:24:34 2012 +0100
@@ -790,14 +790,6 @@
   shows "bl_to_bin (bin_to_bl (len_of TYPE('a)) (uint x)) = uint x"
   by (rule trans [OF bin_bl_bin word_ubin.norm_Rep])
 
-(* FIXME: the next two lemmas should be unnecessary, because the lhs
-terms should never occur in practice *)
-lemma num_AB_u [simp]: "number_of (uint x) = x"
-  unfolding word_number_of_def by (rule word_uint.Rep_inverse)
-
-lemma num_AB_s [simp]: "number_of (sint x) = x"
-  unfolding word_number_of_def by (rule word_sint.Rep_inverse)
-
 (* naturals *)
 lemma uints_unats: "uints n = int ` unats n"
   apply (unfold unats_def uints_num)