tentatively tag hypotheses as definition -- this sometimes help the "tptp_sledgehammer" tool (e.g. SEU466^1.p)
authorblanchet
Thu, 26 Apr 2012 00:29:46 +0200
changeset 47772 993a44ef9928
parent 47771 ba321ce6f344
child 47773 7292038cad2a
tentatively tag hypotheses as definition -- this sometimes help the "tptp_sledgehammer" tool (e.g. SEU466^1.p)
src/HOL/Tools/ATP/atp_systems.ML
--- a/src/HOL/Tools/ATP/atp_systems.ML	Thu Apr 26 00:28:06 2012 +0200
+++ b/src/HOL/Tools/ATP/atp_systems.ML	Thu Apr 26 00:29:46 2012 +0200
@@ -362,7 +362,7 @@
      [("% Higher-Order Unsat Core BEGIN", "% Higher-Order Unsat Core END")],
    known_failures = known_szs_status_failures,
    conj_sym_kind = Axiom,
-   prem_kind = Hypothesis,
+   prem_kind = Definition (* motivated by "isabelle tptp_sledgehammer" tool *),
    best_slices =
      (* FUDGE *)
      K [(1.0, (true, ((100, satallax_thf0, "mono_native_higher", keep_lamsN, false), "")))]}