Improved error msg "Proved wrong thm"
authornipkow
Mon, 20 Jun 1994 12:25:28 +0200
changeset 432 0d1071ac599c
parent 431 da3d07d4349b
child 433 1e4f420523ae
Improved error msg "Proved wrong thm"
src/Pure/thm.ML
--- a/src/Pure/thm.ML	Mon Jun 20 12:13:08 1994 +0200
+++ b/src/Pure/thm.ML	Mon Jun 20 12:25:28 1994 +0200
@@ -1192,8 +1192,10 @@
 
 fun termless tu = (termord tu = LESS);
 
-fun check_conv(thm as Thm{hyps,prop,...}, prop0) =
-  let fun err() = (trace_thm "Proved wrong thm (Check subgoaler?)" thm; None)
+fun check_conv(thm as Thm{hyps,prop,sign,...}, prop0) =
+  let fun err() = (trace_thm "Proved wrong thm (Check subgoaler?)" thm;
+                   trace_term "Should have proved" sign prop0;
+                   None)
       val (lhs0,_) = Logic.dest_equals(Logic.strip_imp_concl prop0)
   in case prop of
        Const("==",_) $ lhs $ rhs =>