further improved type system setup based on Judgment Days
authorblanchet
Fri, 06 May 2011 13:35:00 +0200
changeset 42710 84fcce345b5d
parent 42709 e7af132d48fe
child 42711 159c4d1d4c42
further improved type system setup based on Judgment Days
src/HOL/Tools/ATP/atp_systems.ML
--- a/src/HOL/Tools/ATP/atp_systems.ML	Fri May 06 13:34:59 2011 +0200
+++ b/src/HOL/Tools/ATP/atp_systems.ML	Fri May 06 13:35:00 2011 +0200
@@ -74,6 +74,11 @@
    best_slices : Proof.context -> (real * (bool * int)) list,
    best_type_systems : string list}
 
+(* "best_slices" and "best_type_systems" must be found empirically, taking a
+    wholistic approach since the ATPs are run in parallel. "best_type_systems"
+    should be of the form [sound] or [unsound, sound], where "sound" is a sound
+    type system and "unsound" is an unsound one. *)
+
 val known_perl_failures =
   [(CantConnect, "HTTP error"),
    (NoPerl, "env: perl"),
@@ -213,9 +218,6 @@
         (0.33334, (true, 200 (* FUDGE *))) (* fun_weight *)]
      else
        [(1.0, (true, 250 (* FUDGE *)))],
-   (* Actual order, according to Judgment Day: "mangled_preds!",
-      "mangled_tags!", "mangled_tags?", "mangled_preds?". But E "mangled_preds?"
-      works well in combination with Vampire "mangled_tags!". *)
    best_type_systems = ["mangled_preds?"]}
 
 val e = (eN, e_config)
@@ -248,8 +250,7 @@
    best_slices =
      K [(0.66667, (false, 150 (* FUDGE *))) (* with SOS *),
         (0.33333, (true, 150 (* FUDGE *))) (* without SOS *)],
-   best_type_systems =
-     ["args", "mangled_preds!", "mangled_tags!", "mangled_tags?"]}
+   best_type_systems = ["mangled_preds"]}
 
 val spass = (spassN, spass_config)
 
@@ -286,8 +287,7 @@
    best_slices =
      K [(0.66667, (false, 450 (* FUDGE *))) (* with SOS *),
         (0.33333, (true, 450 (* FUDGE *))) (* without SOS *)],
-   best_type_systems =
-     ["mangled_tags!", "mangled_preds!", "mangled_preds?"]}
+   best_type_systems = ["mangled_tags!", "mangled_preds?"]}
 
 val vampire = (vampireN, vampire_config)