--- a/ProgTutorial/Recipes/TimeLimit.thy Mon Oct 12 17:07:17 2009 +0200
+++ b/ProgTutorial/Recipes/TimeLimit.thy Tue Oct 13 22:57:25 2009 +0200
@@ -1,5 +1,5 @@
theory TimeLimit
-imports "../Base"
+imports "../Appendix"
begin
section {* Restricting the Runtime of a Function\label{rec:timeout} *}