src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML
changeset 52196 2281f33e8da6
parent 52150 41c885784e04
child 52366 ff89424b5094
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Tue May 28 08:36:12 2013 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Tue May 28 08:52:41 2013 +0200
@@ -649,7 +649,13 @@
      fact_names, lifted, sym_tab, atp_proof, goal)
     (one_line_params as (_, _, _, _, subgoal, subgoal_count)) =
   let
-    val ((params, hyp_ts, concl_t), ctxt) = strip_subgoal goal subgoal ctxt
+    val (params, hyp_ts, concl_t) = strip_subgoal goal subgoal ctxt
+    val (_, ctxt) =
+      params
+      |> map (fn (s, T) => (Binding.name s, SOME T, NoSyn))
+      |> (fn fixes =>
+             ctxt |> Variable.set_body false
+                  |> Proof_Context.add_fixes fixes)
     val one_line_proof = one_line_proof_text 0 one_line_params
     val type_enc =
       if is_typed_helper_used_in_atp_proof atp_proof then full_typesN