ProgTutorial/Appendix.thy
changeset 346 0fea8b7a14a1
parent 189 069d525f8f1d
child 356 43df2d59fb98
--- a/ProgTutorial/Appendix.thy	Mon Oct 12 17:07:17 2009 +0200
+++ b/ProgTutorial/Appendix.thy	Tue Oct 13 22:57:25 2009 +0200
@@ -1,8 +1,15 @@
 
 theory Appendix
-imports Main
+imports Base
 begin
 
+(*<*)
+setup{*
+open_file_with_prelude 
+  "Recipes_Code.thy"
+  ["theory Recipes", "imports Main", "begin"]
+*}
+(*>*)
 
 text {* \appendix *}