src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 46320 0b8b73b49848
parent 46301 e2e52c7d25c9
child 46340 cac402c486b0
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML	Mon Jan 23 17:40:31 2012 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML	Mon Jan 23 17:40:32 2012 +0100
@@ -9,11 +9,11 @@
 signature SLEDGEHAMMER_PROVERS =
 sig
   type failure = ATP_Proof.failure
-  type locality = ATP_Translate.locality
-  type type_enc = ATP_Translate.type_enc
-  type reconstructor = ATP_Reconstruct.reconstructor
-  type play = ATP_Reconstruct.play
-  type minimize_command = ATP_Reconstruct.minimize_command
+  type locality = ATP_Problem_Generate.locality
+  type type_enc = ATP_Problem_Generate.type_enc
+  type reconstructor = ATP_Proof_Reconstruct.reconstructor
+  type play = ATP_Proof_Reconstruct.play
+  type minimize_command = ATP_Proof_Reconstruct.minimize_command
   type relevance_fudge = Sledgehammer_Filter.relevance_fudge
 
   datatype mode = Auto_Try | Try | Normal | Auto_Minimize | Minimize
@@ -119,8 +119,8 @@
 open ATP_Problem
 open ATP_Proof
 open ATP_Systems
-open ATP_Translate
-open ATP_Reconstruct
+open ATP_Problem_Generate
+open ATP_Proof_Reconstruct
 open Metis_Tactic
 open Sledgehammer_Util
 open Sledgehammer_Filter