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