src/HOL/SAT.thy
changeset 49985 5b4b0e4e5205
parent 48891 c0eafbd55de3
child 49989 34d0ac1bdac6
--- a/src/HOL/SAT.thy	Wed Oct 31 11:23:21 2012 +0100
+++ b/src/HOL/SAT.thy	Wed Oct 31 11:23:21 2012 +0100
@@ -8,7 +8,7 @@
 header {* Reconstructing external resolution proofs for propositional logic *}
 
 theory SAT
-imports Refute
+imports Hilbert_Choice List Sledgehammer
 begin
 
 ML_file "Tools/sat_funcs.ML"