doc-src/Codegen/Thy/Foundations.thy
changeset 45211 3dd426ae6bea
parent 43410 957617fe0765
child 46521 addcdf0dd283
equal deleted inserted replaced
45210:b416573f1807 45211:3dd426ae6bea
   123   \noindent The current setup of the preprocessor may be inspected
   123   \noindent The current setup of the preprocessor may be inspected
   124   using the @{command_def print_codeproc} command.  @{command_def
   124   using the @{command_def print_codeproc} command.  @{command_def
   125   code_thms} (see \secref{sec:equations}) provides a convenient
   125   code_thms} (see \secref{sec:equations}) provides a convenient
   126   mechanism to inspect the impact of a preprocessor setup on code
   126   mechanism to inspect the impact of a preprocessor setup on code
   127   equations.
   127   equations.
   128 
       
   129   \begin{warn}
       
   130     Attribute @{attribute code_unfold} also applies to the
       
   131     preprocessor of the ancient @{text "SML code generator"}; in case
       
   132     this is not what you intend, use @{attribute code_inline} instead.
       
   133   \end{warn}
       
   134 *}
   128 *}
   135 
   129 
   136 
   130 
   137 subsection {* Understanding code equations \label{sec:equations} *}
   131 subsection {* Understanding code equations \label{sec:equations} *}
   138 
   132