src/HOL/Datatype.thy
changeset 19347 e2e709f3f955
parent 19202 0b9eb4b0ad98
child 19564 d3e2f532459a
--- a/src/HOL/Datatype.thy	Thu Apr 06 16:10:46 2006 +0200
+++ b/src/HOL/Datatype.thy	Thu Apr 06 16:11:30 2006 +0200
@@ -222,31 +222,31 @@
 
 subsubsection {* Codegenerator setup *}
 
-lemma [code]:
+lemma [code fun]:
   "(\<not> True) = False" by (rule HOL.simp_thms)
 
-lemma [code]:
+lemma [code fun]:
   "(\<not> False) = True" by (rule HOL.simp_thms)
 
-lemma [code]:
+lemma [code fun]:
   shows "(False \<and> x) = False"
   and   "(True \<and> x) = x"
   and   "(x \<and> False) = False"
   and   "(x \<and> True) = x" by simp_all
 
-lemma [code]:
+lemma [code fun]:
   shows "(False \<or> x) = x"
   and   "(True \<or> x) = True"
   and   "(x \<or> False) = x"
   and   "(x \<or> True) = True" by simp_all
 
 declare
-  if_True [code]
-  if_False [code]
+  if_True [code fun]
+  if_False [code fun]
   fst_conv [code]
   snd_conv [code]
 
-lemma [code unfold]:
+lemma [code unfolt]:
   "1 == Suc 0" by simp
 
 code_generate True False Not "op &" "op |" If