changeset 46172 | c06e868dc339 |
parent 46136 | a3d4cf5203f5 |
child 46173 | 5cc700033194 |
--- a/src/HOL/Word/Word.thy Tue Jan 10 10:48:39 2012 +0100 +++ b/src/HOL/Word/Word.thy Tue Jan 10 14:48:42 2012 +0100 @@ -2155,6 +2155,9 @@ n < len_of TYPE('a) \<and> bin_nth (number_of w) n" unfolding word_number_of_alt test_bit_wi .. +lemma test_bit_1 [simp]: "(1::'a::len word) !! n \<longleftrightarrow> n = 0" + unfolding word_1_wi test_bit_wi by auto + lemma nth_0 [simp]: "~ (0::'a::len0 word) !! n" unfolding word_test_bit_def by simp