src/Doc/Codegen/Inductive_Predicate.thy
changeset 76987 4c275405faae
parent 72184 881bd98bddee
equal deleted inserted replaced
76986:1e31ddcab458 76987:4c275405faae
    21 text \<open>
    21 text \<open>
    22   The \<open>predicate compiler\<close> is an extension of the code generator
    22   The \<open>predicate compiler\<close> is an extension of the code generator
    23   which turns inductive specifications into equational ones, from
    23   which turns inductive specifications into equational ones, from
    24   which in turn executable code can be generated.  The mechanisms of
    24   which in turn executable code can be generated.  The mechanisms of
    25   this compiler are described in detail in
    25   this compiler are described in detail in
    26   @{cite "Berghofer-Bulwahn-Haftmann:2009:TPHOL"}.
    26   \<^cite>\<open>"Berghofer-Bulwahn-Haftmann:2009:TPHOL"\<close>.
    27 
    27 
    28   Consider the simple predicate \<^const>\<open>append\<close> given by these two
    28   Consider the simple predicate \<^const>\<open>append\<close> given by these two
    29   introduction rules:
    29   introduction rules:
    30 \<close>
    30 \<close>
    31 
    31