ProgTutorial/Recipes/Timing.thy
changeset 346 0fea8b7a14a1
parent 239 b63c72776f03
child 456 89fccd3d5055
--- a/ProgTutorial/Recipes/Timing.thy	Mon Oct 12 17:07:17 2009 +0200
+++ b/ProgTutorial/Recipes/Timing.thy	Tue Oct 13 22:57:25 2009 +0200
@@ -1,5 +1,5 @@
 theory Timing
-imports "../Base"
+imports "../Appendix"
 begin
 
 section {* Measuring Time\label{rec:timing} *}