doc-src/IsarAdvanced/Codegen/Thy/Further.thy
author haftmann
Sun, 14 Sep 2008 21:50:35 +0200
changeset 28213 b52f9205a02d
child 28419 f65e8b318581
permissions -rw-r--r--
New outline for codegen tutorial -- draft

theory Further
imports Setup
begin

section {* Further topics *}

subsection {* Serializer options *}

subsection {* Evaluation oracle *}

subsection {* Code antiquotation *}

subsection {* Creating new targets *}

text {* extending targets, adding targets *}

end