src/HOL/Code_Evaluation.thy
changeset 33473 3b275a0bf18c
parent 32740 9dd0a2f83429
child 33553 35f2b30593a8
--- a/src/HOL/Code_Evaluation.thy	Thu Nov 05 14:47:27 2009 +0100
+++ b/src/HOL/Code_Evaluation.thy	Fri Nov 06 08:11:58 2009 +0100
@@ -243,6 +243,26 @@
 hide const dummy_term App valapp
 hide (open) const Const termify valtermify term_of term_of_num
 
+subsection {* Tracing of generated and evaluated code *}
+
+definition tracing :: "String.literal => 'a => 'a"
+where
+  [code del]: "tracing s x = x"
+
+ML {*
+structure Code_Evaluation =
+struct
+
+fun tracing s x = (Output.tracing s; x)
+
+end
+*}
+
+code_const "tracing :: String.literal => 'a => 'a"
+  (Eval "Code'_Evaluation.tracing")
+
+hide (open) const tracing
+code_reserved Eval Code_Evaluation
 
 subsection {* Evaluation setup *}