equal
deleted
inserted
replaced
115 text {* |
115 text {* |
116 \noindent \emph{Function transformers} provide a very general |
116 \noindent \emph{Function transformers} provide a very general |
117 interface, transforming a list of function theorems to another list |
117 interface, transforming a list of function theorems to another list |
118 of function theorems, provided that neither the heading constant nor |
118 of function theorems, provided that neither the heading constant nor |
119 its type change. The @{term "0\<Colon>nat"} / @{const Suc} pattern |
119 its type change. The @{term "0\<Colon>nat"} / @{const Suc} pattern |
120 elimination implemented in theory @{text Efficient_Nat} (see |
120 elimination implemented in theory @{text Code_Binary_Nat} (see |
121 \secref{eff_nat}) uses this interface. |
121 \secref{eff_nat}) uses this interface. |
122 |
122 |
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 |