src/HOL/Code_Setup.thy
changeset 25916 d957d9982241
parent 25885 6fbc3f54f819
child 25962 13b6c0b31005
--- a/src/HOL/Code_Setup.thy	Tue Jan 15 02:38:13 2008 +0100
+++ b/src/HOL/Code_Setup.thy	Tue Jan 15 16:19:19 2008 +0100
@@ -86,7 +86,7 @@
 
 text {* type bool *}
 
-lemmas [code unfold] = imp_conv_disj
+lemmas [code func, code unfold] = imp_conv_disj
 
 code_type bool
   (SML "bool")