--- a/ProgTutorial/Recipes/Sat.thy Sat Oct 03 13:01:39 2009 +0200
+++ b/ProgTutorial/Recipes/Sat.thy Sat Oct 03 19:10:23 2009 +0200
@@ -1,6 +1,6 @@
theory Sat
-imports Main "../Base"
+imports Main "../FirstSteps"
begin
section {* SAT Solvers\label{rec:sat} *}
@@ -59,7 +59,7 @@
@{ML table'} is:
@{ML_response_fake [display,gray]
- "map (apfst (Syntax.string_of_term @{context})) (Termtab.dest table')"
+ "map (apfst (string_of_term @{context})) (Termtab.dest table')"
"(\<forall>x. P x, 1)"}
In the print out of the tabel, we used some pretty printing scaffolding