src/HOL/ex/Codegenerator_Pretty.thy
author wenzelm
Thu, 03 Jun 2010 22:17:36 +0200
changeset 37305 9763792e4ac7
parent 31378 d1cbf6393964
permissions -rw-r--r--
diagnostic commands 'ML_val' and 'ML_command' may refer to antiquotations @{Isar.state} and @{Isar.goal};


(* Author: Florian Haftmann, TU Muenchen *)

header {* Generating code using pretty literals and natural number literals  *}

theory Codegenerator_Pretty
imports "~~/src/HOL/ex/Codegenerator_Candidates" Code_Char Efficient_Nat
begin

declare isnorm.simps [code del]

end