src/HOL/Tools/ATP/atp_satallax.ML
changeset 57707 0242e9578828
parent 57706 94476c92f892
child 57710 323a57d7455c
--- a/src/HOL/Tools/ATP/atp_satallax.ML	Wed Jul 30 14:03:12 2014 +0200
+++ b/src/HOL/Tools/ATP/atp_satallax.ML	Wed Jul 30 14:03:12 2014 +0200
@@ -170,7 +170,7 @@
   | find_assumptions_to_inline ths [] _ _ = ths
 
 fun inline_if_needed_and_simplify th assms to_inline no_inline =
-    (case find_assumptions_to_inline [] assms to_inline no_inline of
+    (case find_assumptions_to_inline [th] assms to_inline no_inline of
       [] => ATerm (("$true", [dummy_atype]), [])
   | l => foldl1 (fn (a, b) => ATerm ((tptp_or, [dummy_atype]), [a, b])) l)
 
@@ -315,7 +315,7 @@
           (Scan.finite Symbol.stopper (Scan.repeat1 (parse_line local_name problem) >> flat)))
            #> fst)
       else
-        (Scan.error (!! (fn f => raise UNRECOGNIZED_ATP_PROOF ())
+        (Scan.error (!! (fn _ => raise UNRECOGNIZED_ATP_PROOF ())
           (Scan.finite Symbol.stopper (Scan.repeat1 (parse_tstp_thf0_satallax_line))))
           #> fst
           #> rev