src/HOL/Code_Setup.thy
changeset 25860 844ab7ace3db
parent 25534 d0b74fdd6067
child 25866 263aaf988d44
     1.1 --- a/src/HOL/Code_Setup.thy	Mon Jan 07 11:40:20 2008 +0100
     1.2 +++ b/src/HOL/Code_Setup.thy	Tue Jan 08 10:24:34 2008 +0100
     1.3 @@ -84,7 +84,7 @@
     1.4  
     1.5  text {* type bool *}
     1.6  
     1.7 -lemmas [code] = imp_conv_disj
     1.8 +lemmas [code unfold] = imp_conv_disj
     1.9  
    1.10  code_type bool
    1.11    (SML "bool")