add code lemmas for word operations
authorhuffman
Thu, 19 Apr 2012 19:32:30 +0200
changeset 47611 e3c699a1fae6
parent 47610 261f9de35b18
child 47612 bc9c7b5c26fd
add code lemmas for word operations
src/HOL/Word/Word.thy
--- a/src/HOL/Word/Word.thy	Thu Apr 19 19:18:47 2012 +0200
+++ b/src/HOL/Word/Word.thy	Thu Apr 19 19:32:30 2012 +0200
@@ -294,7 +294,7 @@
 
 text {* Legacy theorems: *}
 
-lemma word_arith_wis: shows
+lemma word_arith_wis [code]: shows
   word_add_def: "a + b = word_of_int (uint a + uint b)" and
   word_sub_wi: "a - b = word_of_int (uint a - uint b)" and
   word_mult_def: "a * b = word_of_int (uint a * uint b)" and
@@ -416,7 +416,7 @@
 
 end
 
-lemma shows
+lemma [code]: shows
   word_not_def: "NOT (a::'a::len0 word) = word_of_int (NOT (uint a))" and
   word_and_def: "(a::'a word) AND b = word_of_int (uint a AND uint b)" and
   word_or_def: "(a::'a word) OR b = word_of_int (uint a OR uint b)" and