src/Doc/Codegen/Foundations.thy
changeset 61076 bdc1e2f0a86a
parent 59377 056945909f60
child 61781 e1e6bb36b27a
equal deleted inserted replaced
61075:f6b0d827240e 61076:bdc1e2f0a86a
   142   or \emph{@{attribute code_post}} respectively.
   142   or \emph{@{attribute code_post}} respectively.
   143 
   143 
   144   \emph{Function transformers} provide a very general
   144   \emph{Function transformers} provide a very general
   145   interface, transforming a list of function theorems to another list
   145   interface, transforming a list of function theorems to another list
   146   of function theorems, provided that neither the heading constant nor
   146   of function theorems, provided that neither the heading constant nor
   147   its type change.  The @{term "0\<Colon>nat"} / @{const Suc} pattern
   147   its type change.  The @{term "0::nat"} / @{const Suc} pattern
   148   used in theory @{text Code_Abstract_Nat} (see \secref{abstract_nat})
   148   used in theory @{text Code_Abstract_Nat} (see \secref{abstract_nat})
   149   uses this interface.
   149   uses this interface.
   150 
   150 
   151   \noindent The current setup of the pre- and postprocessor may be inspected
   151   \noindent The current setup of the pre- and postprocessor may be inspected
   152   using the @{command_def print_codeproc} command.  @{command_def
   152   using the @{command_def print_codeproc} command.  @{command_def