ProgTutorial/Solutions.thy
changeset 346 0fea8b7a14a1
parent 329 5dffcab68680
child 351 f118240ab44a
--- a/ProgTutorial/Solutions.thy	Mon Oct 12 17:07:17 2009 +0200
+++ b/ProgTutorial/Solutions.thy	Tue Oct 13 22:57:25 2009 +0200
@@ -2,6 +2,14 @@
 imports FirstSteps "Recipes/Timing"
 begin
 
+(*<*)
+setup{*
+open_file_with_prelude 
+  "Solutions_Code.thy"
+  ["theory Solutions", "imports FirstSteps", "begin"]
+*}
+(*>*)
+
 chapter {* Solutions to Most Exercises\label{ch:solutions} *}
 
 text {* \solution{fun:revsum} *}