equal
deleted
inserted
replaced
220 |
220 |
221 \item The scope and quality of generated code can be increased |
221 \item The scope and quality of generated code can be increased |
222 dramatically by applying refinement techniques, which are |
222 dramatically by applying refinement techniques, which are |
223 introduced in \secref{sec:refinement}. |
223 introduced in \secref{sec:refinement}. |
224 |
224 |
|
225 \item How to define partial functions such that code can be generated |
|
226 is explained in \secref{sec:partial}. |
|
227 |
225 \item Inductive predicates can be turned executable using an |
228 \item Inductive predicates can be turned executable using an |
226 extension of the code generator \secref{sec:inductive}. |
229 extension of the code generator \secref{sec:inductive}. |
227 |
230 |
228 \item If you want to utilize code generation to obtain fast |
231 \item If you want to utilize code generation to obtain fast |
229 evaluators e.g.~for decision procedures, have a look at |
232 evaluators e.g.~for decision procedures, have a look at |