one-step Isar proofs are not always pointless
authorblanchet
Thu, 29 Apr 2010 17:39:46 +0200
changeset 36563 bba1e5f2b643
parent 36562 c6c2661bf08e
child 36564 96f767f546e7
one-step Isar proofs are not always pointless
src/HOL/Tools/Sledgehammer/sledgehammer_proof_reconstruct.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_proof_reconstruct.ML	Thu Apr 29 17:31:08 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_proof_reconstruct.ML	Thu Apr 29 17:39:46 2010 +0200
@@ -924,9 +924,7 @@
         suffix ^ "\n"
       end
     and do_block ind proof = do_steps "{ " " }" (ind + 1) proof
-    (* One-step proofs are pointless; better use the Metis one-liner. *)
-    and do_proof [_] = ""
-      | do_proof proof =
+    and do_proof proof =
         (if i <> 1 then "prefer " ^ string_of_int i ^ "\n" else "") ^
         do_indent 0 ^ "proof -\n" ^
         do_steps "" "" 1 proof ^