Sledgehammer should be called in "prove" mode;
authorblanchet
Tue, 14 Sep 2010 15:39:57 +0200
changeset 39364 61f0d36840c5
parent 39363 1c4e38d635e1
child 39365 9cab71c20613
Sledgehammer should be called in "prove" mode; otherwise the proof text won't fit into the proof document
src/HOL/Tools/Sledgehammer/sledgehammer.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer.ML	Tue Sep 14 14:47:53 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer.ML	Tue Sep 14 15:39:57 2010 +0200
@@ -438,6 +438,7 @@
     0 => (priority "No subgoal!"; (false, state))
   | n =>
     let
+      val _ = Proof.assert_backward state
       val thy = Proof.theory_of state
       val timer = Timer.startRealTimer ()
       val _ = () |> not blocking ? kill_atps