--- a/ProgTutorial/Recipes/Sat.thy Mon Oct 12 17:07:17 2009 +0200
+++ b/ProgTutorial/Recipes/Sat.thy Tue Oct 13 22:57:25 2009 +0200
@@ -1,6 +1,6 @@
theory Sat
-imports Main "../FirstSteps"
+imports "../Appendix" "../FirstSteps"
begin
section {* SAT Solvers\label{rec:sat} *}