src/HOL/Tools/ATP_Manager/atp_wrapper.ML
changeset 36235 61159615a0c5
parent 36231 bede2d49ba3b
child 36264 3c2490917710
--- a/src/HOL/Tools/ATP_Manager/atp_wrapper.ML	Tue Apr 20 14:39:42 2010 +0200
+++ b/src/HOL/Tools/ATP_Manager/atp_wrapper.ML	Tue Apr 20 16:04:36 2010 +0200
@@ -67,7 +67,7 @@
   | (failure :: _) => SOME failure
 
 fun generic_prover overlord get_facts prepare write_file cmd args failure_strs
-        proof_text name ({debug, full_types, ...} : params)
+        proof_text name ({debug, full_types, explicit_apply, ...} : params)
         ({subgoal, goal, relevance_override, axiom_clauses, filtered_clauses}
          : problem) =
   let
@@ -128,7 +128,7 @@
       if Config.get ctxt measure_runtime then split_time s else (s, 0)
     fun run_on probfile =
       if File.exists cmd then
-        write_file full_types probfile clauses
+        write_file full_types explicit_apply probfile clauses
         |> pair (apfst split_time' (bash_output (cmd_line probfile)))
       else error ("Bad executable: " ^ Path.implode cmd ^ ".");