doc-src/IsarAdvanced/Codegen/Thy/Program.thy
author haftmann
Thu, 25 Sep 2008 09:28:08 +0200
changeset 28350 715163ec93c0
parent 28213 b52f9205a02d
child 28419 f65e8b318581
permissions -rw-r--r--
non left-linear equations for nbe

theory Program
imports Setup
begin

section {* Turning Theories into Programs *}

subsection {* The @{text "Isabelle/HOL"} default setup *}

text {* Invoking the code generator *}

subsection {* Selecting code equations *}

text {* inspection by @{text "code_thms"} *}

subsection {* The preprocessor *}

subsection {* Datatypes *}

text {* example: @{text "rat"}, cases *}

subsection {* Equality and wellsortedness *}

subsection {* Partiality *}

text {* @{text "code_abort"}, examples: maps *}

end