added new portfolio for Vampire 4.8
authordesharna
Wed, 18 Oct 2023 10:41:12 +0200
changeset 78788 5a14f2cc1ea0
parent 78787 a7e4b412cc7c
child 78789 f2e845c3e65c
added new portfolio for Vampire 4.8
src/HOL/Tools/ATP/atp_problem.ML
src/HOL/Tools/Sledgehammer/sledgehammer_atp_systems.ML
--- a/src/HOL/Tools/ATP/atp_problem.ML	Tue Oct 17 12:10:58 2023 +0200
+++ b/src/HOL/Tools/ATP/atp_problem.ML	Wed Oct 18 10:41:12 2023 +0200
@@ -493,7 +493,7 @@
         "[" ^ commas (map of_term ts) ^ "]"
       else if is_tptp_equal s then
         space_implode (" " ^ tptp_equal ^ " ") (map of_term ts)
-        |> (is_format_higher_order format orelse is_format_with_fool format) ? parens
+        |> (is_format_higher_order format orelse true) ? parens
       else if s = tptp_ho_forall orelse s = tptp_ho_exists then
         (case ts of
           [AAbs (((s', ty), tm), [])] =>
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_atp_systems.ML	Tue Oct 17 12:10:58 2023 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_atp_systems.ML	Wed Oct 18 10:41:12 2023 +0200
@@ -1,6 +1,7 @@
 (*  Title:      HOL/Tools/Sledgehammer/sledgehammer_atp_systems.ML
     Author:     Fabian Immler, TU Muenchen
     Author:     Jasmin Blanchette, TU Muenchen
+    Author:     Martin Desharnais, MPI-INF Saarbruecken
 
 Setup for supported ATPs.
 *)
@@ -62,7 +63,9 @@
 val TX0 = TFF (Monomorphic, With_FOOL {with_ite = true, with_let = true})
 val TX1 = TFF (Polymorphic, With_FOOL {with_ite = true, with_let = true})
 val TH0 = THF (Monomorphic, {with_ite = true, with_let = true}, THF_With_Choice)
+val TH0_MINUS = THF (Monomorphic, {with_ite = false, with_let = false}, THF_Without_Choice)
 val TH1 = THF (Polymorphic, {with_ite = true, with_let = true}, THF_With_Choice)
+val TH1_MINUS = THF (Polymorphic, {with_ite = false, with_let = false}, THF_Without_Choice)
 
 val default_max_mono_iters = 3 (* FUDGE *)
 val default_max_new_mono_instances = 100 (* FUDGE *)
@@ -361,21 +364,35 @@
 
 (* Vampire *)
 
-val vampire_basic_options =
-  "--proof tptp --output_axiom_names on" ^
+local
+
+val old_vampire_basic_options =
+  ["--proof tptp",
+   "--output_axiom_names on"] @
   (if ML_System.platform_is_windows
-   then ""  (*time slicing is not support in the Windows version of Vampire*)
-   else " --mode casc")
+   then []  (*time slicing is not support in the Windows version of Vampire*)
+   else ["--mode casc"])
+
+val new_vampire_basic_options =
+  ["--input_syntax tptp",
+   "--proof tptp",
+   "--output_axiom_names on"] @
+  (if ML_System.platform_is_windows
+   then []  (*time slicing is not support in the Windows version of Vampire*)
+   else ["--mode portfolio", "--schedule snake_slh"])
 
 val vampire_full_proof_options =
-  " --proof_extra free --forced_options avatar=off:equality_proxy=off:general_splitting=off:inequality_splitting=0:naming=0"
+  ["--proof_extra free",
+   "--forced_options avatar=off:equality_proxy=off:general_splitting=off:inequality_splitting=0:naming=0"]
 
-val vampire_config : atp_config =
+fun make_vampire_config vampire_basic_options good_max_new_mono_instances good_slices : atp_config =
   {exec = (["VAMPIRE_HOME"], ["vampire"]),
-   arguments = fn _ => fn full_proofs => fn sos => fn timeout => fn problem =>
-     [vampire_basic_options ^ (if full_proofs then " " ^ vampire_full_proof_options else "") ^
-       " -t " ^ string_of_int (to_secs 1 timeout) ^ " --input_file " ^ File.bash_path problem
-       |> sos = sosN ? prefix "--sos on "],
+   arguments = fn _ => fn full_proofs => fn extra_options => fn timeout => fn problem =>
+     vampire_basic_options @
+     (if full_proofs then vampire_full_proof_options else []) @
+     (if extra_options <> "" then [extra_options] else []) @
+     ["-t " ^ string_of_int (to_secs 1 timeout),
+      "--input_file " ^ File.bash_path problem],
    proof_delims =
      [("=========== Refutation ==========",
        "======= End of refutation =======")] @
@@ -389,28 +406,56 @@
      known_szs_status_failures,
    prem_role = Hypothesis,
    generate_isabelle_info = false,
-   good_slices =
-     let
-       (* Older versions of Vampire have unsound handling of Booleans. *)
-       val mono_native =
-         if string_ord (getenv "VAMPIRE_VERSION", "4.8") <> LESS then "mono_native_fool"
-         else "mono_native"
-     in
-       (* FUDGE *)
-       K [((2, false, false, 512, meshN), (TX1, mono_native, combsN, false, sosN)),
-        ((2, false, false, 1024, meshN), (TX1, mono_native, liftingN, false, sosN)),
-        ((2, false, false, 256, mashN), (TX1, mono_native, liftingN, false, no_sosN)),
-        ((2, false, true, 512, mepoN), (TF1, "poly_native", liftingN, false, no_sosN)),
-        ((2, false, false, 16, meshN), (TX1, mono_native, liftingN, false, no_sosN)),
-        ((2, false, false, 32, meshN), (TX1, mono_native, combsN, false, no_sosN)),
-        ((2, false, false, 64, meshN), (TX1, mono_native, combs_or_liftingN, false, no_sosN)),
-        ((2, false, false, 128, meshN), (TX1, mono_native, liftingN, false, no_sosN))]
-      end,
+   good_slices = K good_slices,
    good_max_mono_iters = default_max_mono_iters,
-   good_max_new_mono_instances = 2 * default_max_new_mono_instances (* FUDGE *)}
+   good_max_new_mono_instances = good_max_new_mono_instances}
+
+val old_vampire_config : atp_config =
+  (* FUDGE *)
+  make_vampire_config old_vampire_basic_options (2 * default_max_new_mono_instances)
+  [((2, false, false, 512, meshN), (TX1, "mono_native", combsN, false, sosN)),
+   ((2, false, false, 1024, meshN), (TX1, "mono_native", liftingN, false, sosN)),
+   ((2, false, false, 256, mashN), (TX1, "mono_native", liftingN, false, no_sosN)),
+   ((2, false, true, 512, mepoN), (TF1, "poly_native", liftingN, false, no_sosN)),
+   ((2, false, false, 16, meshN), (TX1, "mono_native", liftingN, false, no_sosN)),
+   ((2, false, false, 32, meshN), (TX1, "mono_native", combsN, false, no_sosN)),
+   ((2, false, false, 64, meshN), (TX1, "mono_native", combs_or_liftingN, false, no_sosN)),
+   ((2, false, false, 128, meshN), (TX1, "mono_native", liftingN, false, no_sosN))]
 
-val vampire = (vampireN, fn () => vampire_config)
+val new_vampire_config : atp_config =
+  let val infinity = 1000 in
+    (* FUDGE: this solved 998/1500 (66.53 %) using MePo when testing *)
+    make_vampire_config new_vampire_basic_options 256
+    [(((infinity, false, false,  512, meshN), (TX0, "mono_native_fool", liftingN, false, ""))),
+     (((infinity, false, false, 2048, meshN), (TX0, "mono_native_fool", combsN, false, ""))),
+     (((infinity, false, false,  128, meshN), (TX0, "mono_native_fool", liftingN, false, ""))),
+     (((infinity, false, false, 1024, meshN), (TF1, "poly_native", liftingN, false, ""))),
+     (((infinity, false, false,  256, meshN), (TH0_MINUS, "mono_native_higher", keep_lamsN, false, ""))),
+     (((infinity, false, false, 1024, meshN), (TX0, "mono_native_fool", liftingN, false, ""))),
+     (((infinity, false, false,  256, meshN), (TX0, "mono_native_fool", liftingN, false, ""))),
+     (((infinity, false, false, 2048, meshN), (TF1, "poly_native", combsN, false, ""))),
+     (((infinity, false, false,  256, meshN), (TX1, "poly_native_fool", liftingN, false, ""))),
+     (((infinity, false, false,  512, meshN), (TF0, "mono_native", liftingN, false, ""))),
+     (((infinity, false, false, 2048, meshN), (TF0, "mono_native", liftingN, false, ""))),
+     (((infinity, false, false,   64, meshN), (TF1, "poly_native", combsN, false, ""))),
+     (((infinity, false, false,  256, meshN), (TH1_MINUS, "poly_native_higher", keep_lamsN, false, ""))),
+     (((infinity, false, false,  256, meshN), (TF0, "mono_native", combsN, false, ""))),
+     (((infinity, false, false,  256, meshN), (TF0, "mono_native", liftingN, false, ""))),
+     (((infinity, false, false,   32, meshN), (TH0_MINUS, "mono_native_higher", keep_lamsN, false, ""))),
+     (((infinity, false, false,  512, meshN), (TH0_MINUS, "mono_native_higher", keep_lamsN, false, ""))),
+     (((infinity, false, false,  512, meshN), (TX0, "mono_native_fool", combsN, false, ""))),
+     (((infinity, false, false, 1024, meshN), (TX1, "poly_native_fool", combsN, false, "")))]
+  end
 
+in
+
+val vampire = (vampireN, fn () =>
+  if string_ord (getenv "VAMPIRE_VERSION", "4.8") <> LESS then
+    new_vampire_config
+  else
+    old_vampire_config)
+
+end
 
 (* Zipperposition *)