--- a/ProgTutorial/FirstSteps.thy Tue Sep 29 22:10:48 2009 +0200
+++ b/ProgTutorial/FirstSteps.thy Thu Oct 01 10:19:21 2009 +0200
@@ -885,6 +885,20 @@
project_bool (nth list 1)
*}
+ML {*
+ Context.the_thread_data ();
+ Context.display_names @{theory};
+ Context.pretty_thy @{theory}
+ |> Pretty.string_of
+ |> tracing
+*}
+
+text {*
+ \begin{readmore}
+ @{ML_file "Pure/ML-Systems/universal.ML"}
+ \end{readmore}
+*}
+
(**************************************************)
(* bak *)
(**************************************************)