ProgTutorial/Recipes/Sat.thy
changeset 441 520127b708e6
parent 346 0fea8b7a14a1
child 458 242e81f4d461
--- a/ProgTutorial/Recipes/Sat.thy	Tue Jul 20 13:34:44 2010 +0100
+++ b/ProgTutorial/Recipes/Sat.thy	Wed Jul 28 19:09:49 2010 +0200
@@ -1,6 +1,6 @@
 
 theory Sat
-imports "../Appendix" "../FirstSteps" 
+imports "../Appendix" "../First_Steps" 
 begin
 
 section {* SAT Solvers\label{rec:sat} *}
@@ -59,7 +59,7 @@
   @{ML table'} is:
 
   @{ML_response_fake [display,gray]
-  "map (apfst (string_of_term @{context})) (Termtab.dest table')"
+  "map (apfst (Syntax.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