src/HOL/Codegenerator_Test/Candidates_Pretty.thy
changeset 37695 71e84a203c19
parent 31378 d1cbf6393964
child 42842 6ef538f6a8ab
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Codegenerator_Test/Candidates_Pretty.thy	Fri Jul 02 14:23:18 2010 +0200
@@ -0,0 +1,10 @@
+
+(* Author: Florian Haftmann, TU Muenchen *)
+
+header {* Generating code using pretty literals and natural number literals  *}
+
+theory Candidates_Pretty
+imports Candidates Code_Char Efficient_Nat
+begin
+
+end