author | haftmann |
Sun, 14 Sep 2008 21:50:35 +0200 | |
changeset 28213 | b52f9205a02d |
child 28419 | f65e8b318581 |
permissions | -rw-r--r-- |
theory Introduction imports Setup begin chapter {* Code generation from @{text "Isabelle/HOL"} theories *} section {* Introduction and Overview *} text {* This tutorial introduces a generic code generator for the Isabelle system \cite{isa-tutorial}. *} subsection {* Code generation via shallow embedding *} text {* example *} subsection {* Code generator architecture *} text {* foundation, forward references for yet unexplained things *} end