src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML
changeset 47974 08d2dcc2dab9
parent 47972 96c9b8381909
child 48250 1065c307fafe
--- a/src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML	Wed May 23 21:19:48 2012 +0200
+++ b/src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML	Wed May 23 21:19:48 2012 +0200
@@ -481,15 +481,6 @@
            | Fail "inappropriate" => failed ATP_Proof.Inappropriate
     val time_prover = run_time |> Time.toMilliseconds
     val msg = message (preplay ()) ^ message_tail
-    val (outcome, used_facts) =
-      (* Repair incomplete or missing proofs. Better do it here and not in
-         Sledgehammer, so that actual Sledgehammer users get a chance to report
-         the issue. FIXME: This is a temporary hack. *)
-      if outcome = SOME ATP_Proof.ProofIncomplete orelse
-         outcome = SOME ATP_Proof.ProofMissing then
-        (NONE, [])
-      else
-        (outcome, used_facts)
   in
     case outcome of
       NONE => (msg, SH_OK (time_isa, time_prover, used_facts))