start phasing out old SPASS
authorblanchet
Mon, 21 May 2012 11:31:52 +0200
changeset 47949 fafbb2607366
parent 47948 0524790d2112
child 47950 9cb132898ac8
start phasing out old SPASS
src/HOL/TPTP/atp_theory_export.ML
src/HOL/Tools/ATP/atp_systems.ML
--- a/src/HOL/TPTP/atp_theory_export.ML	Mon May 21 11:31:52 2012 +0200
+++ b/src/HOL/TPTP/atp_theory_export.ML	Mon May 21 11:31:52 2012 +0200
@@ -118,7 +118,7 @@
   let
     val thy = Proof_Context.theory_of ctxt
     val prob_file = File.tmp_path (Path.explode "prob")
-    val atp = case format of DFG _ => spass_newN | _ => eN
+    val atp = case format of DFG _ => spassN | _ => eN
     val {exec, arguments, proof_delims, known_failures, ...} =
       get_atp thy atp ()
     val ord = effective_term_order ctxt atp
--- a/src/HOL/Tools/ATP/atp_systems.ML	Mon May 21 11:31:52 2012 +0200
+++ b/src/HOL/Tools/ATP/atp_systems.ML	Mon May 21 11:31:52 2012 +0200
@@ -50,8 +50,6 @@
   val satallaxN : string
   val snarkN : string
   val spassN : string
-  val spass_oldN : string
-  val spass_newN : string
   val vampireN : string
   val waldmeisterN : string
   val z3_tptpN : string
@@ -142,8 +140,6 @@
 val satallaxN = "satallax"
 val snarkN = "snark"
 val spassN = "spass"
-val spass_oldN = "spass_old" (* for experiments *)
-val spass_newN = "spass_new" (* for experiments *)
 val vampireN = "vampire"
 val waldmeisterN = "waldmeister"
 val z3_tptpN = "z3_tptp"
@@ -370,7 +366,7 @@
    "required_vars" and "script/spass"). *)
 val spass_old_config : atp_config =
   {exec = (["ISABELLE_ATP"], "scripts/spass"),
-   required_vars = [["SPASS_OLD_HOME", "SPASS_HOME"]],
+   required_vars = [["SPASS_HOME"]],
    arguments = fn _ => fn _ => fn sos => fn timeout => fn _ =>
      ("-Auto -PGiven=0 -PProblem=0 -Splits=0 -FullRed=0 -DocProof \
       \-VarWeight=3 -TimeLimit=" ^ string_of_int (to_secs 1 timeout))
@@ -393,8 +389,6 @@
       (0.334, (false, ((50, DFG DFG_Unsorted, "mono_tags??", liftingN, false), no_sosN)))]
      |> (if Config.get ctxt force_sos then hd #> apfst (K 1.0) #> single else I)}
 
-val spass_old = (spass_oldN, fn () => spass_old_config)
-
 val spass_new_H1SOS = "-Heuristic=1 -SOS"
 val spass_new_H2 = "-Heuristic=2"
 val spass_new_H2SOS = "-Heuristic=2 -SOS"
@@ -422,8 +416,6 @@
       (0.1000, (false, ((300, DFG DFG_Sorted, "mono_native", combsN, true), spass_new_H2SOS))),
       (0.1000, (false, ((100, DFG DFG_Sorted, "mono_native", combs_and_liftingN, true), spass_new_H2NuVS0)))]}
 
-val spass_new = (spass_newN, fn () => spass_new_config)
-
 val spass =
   (spassN, fn () => if is_new_spass_version () then spass_new_config
                     else spass_old_config)
@@ -649,8 +641,7 @@
 fun effective_term_order ctxt atp =
   let val ord = Config.get ctxt term_order in
     if ord = smartN then
-      if atp = spass_newN orelse
-         (atp = spassN andalso is_new_spass_version ()) then
+      if atp = spassN andalso is_new_spass_version () then
         {is_lpo = false, gen_weights = true, gen_prec = true, gen_simp = false}
       else
         {is_lpo = false, gen_weights = false, gen_prec = false,
@@ -665,10 +656,10 @@
   end
 
 val atps=
-  [alt_ergo, e, leo2, dummy_thf, satallax, spass_old, spass_new, spass,
-   vampire, z3_tptp, remote_e, remote_e_sine, remote_e_tofof, remote_iprover,
-   remote_iprover_eq, remote_leo2, remote_satallax, remote_vampire,
-   remote_z3_tptp, remote_snark, remote_waldmeister]
+  [alt_ergo, e, leo2, dummy_thf, satallax, spass, vampire, z3_tptp, remote_e,
+   remote_e_sine, remote_e_tofof, remote_iprover, remote_iprover_eq,
+   remote_leo2, remote_satallax, remote_vampire, remote_z3_tptp, remote_snark,
+   remote_waldmeister]
 
 val setup = fold add_atp atps