doc-src/IsarAdvanced/Codegen/Thy/Introduction.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 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