src/HOL/Mirabelle/Tools/mirabelle_metis.ML
changeset 46320 0b8b73b49848
parent 45524 43ca06e6c168
child 46365 547d1a1dcaf6
--- a/src/HOL/Mirabelle/Tools/mirabelle_metis.ML	Mon Jan 23 17:40:31 2012 +0100
+++ b/src/HOL/Mirabelle/Tools/mirabelle_metis.ML	Mon Jan 23 17:40:32 2012 +0100
@@ -19,7 +19,8 @@
     val facts = Facts.props (Proof_Context.facts_of (Proof.context_of pre))
 
     fun metis ctxt =
-      Metis_Tactic.metis_tac [] ATP_Translate.lam_liftingN ctxt (thms @ facts)
+      Metis_Tactic.metis_tac [] ATP_Problem_Generate.lam_liftingN ctxt
+                             (thms @ facts)
   in
     (if Mirabelle.can_apply timeout metis pre then "succeeded" else "failed")
     |> prefix (metis_tag id)