Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
(* 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