src/HOL/Tools/Metis/metis_tactics.ML
author blanchet
Tue, 31 May 2011 16:38:36 +0200
changeset 43085 0a2f5b86bdd7
parent 43050 59284a13abc4
child 43089 c2ec08b0d217
permissions -rw-r--r--
first step in sharing more code between ATP and Metis translation
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
39958
88c9aa5666de tuned comments
blanchet
parents: 39953
diff changeset
     1
(*  Title:      HOL/Tools/Metis/metis_tactics.ML
38027
505657ddb047 standardize "Author" tags
blanchet
parents: 38016
diff changeset
     2
    Author:     Kong W. Susanto, Cambridge University Computer Laboratory
505657ddb047 standardize "Author" tags
blanchet
parents: 38016
diff changeset
     3
    Author:     Lawrence C. Paulson, Cambridge University Computer Laboratory
505657ddb047 standardize "Author" tags
blanchet
parents: 38016
diff changeset
     4
    Author:     Jasmin Blanchette, TU Muenchen
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
     5
    Copyright   Cambridge University 2007
23447
1f16190e3836 tuned comments;
wenzelm
parents: 23442
diff changeset
     6
29266
4a478f9d2847 use regular Term.add_vars, Term.add_frees etc.;
wenzelm
parents: 28700
diff changeset
     7
HOL setup for the Metis prover.
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
     8
*)
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
     9
35826
1590abc3d42a renamed Sledgehammer structures
blanchet
parents: 35825
diff changeset
    10
signature METIS_TACTICS =
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    11
sig
43050
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    12
  val metisN : string
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    13
  val metisF_N : string
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    14
  val metisFT_N : string
39979
b13515940b53 added "trace_meson" configuration option, replacing old-fashioned reference
blanchet
parents: 39978
diff changeset
    15
  val trace : bool Config.T
40665
1a65f0c74827 added "verbose" option to Metis to shut up its warnings if necessary
blanchet
parents: 40262
diff changeset
    16
  val verbose : bool Config.T
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    17
  val type_lits : bool Config.T
39891
8e12f1956fcd "meson_new_skolemizer" -> "metis_new_skolemizer" option (since Meson doesn't support the new skolemizer (yet))
blanchet
parents: 39890
diff changeset
    18
  val new_skolemizer : bool Config.T
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    19
  val metis_tac : Proof.context -> thm list -> int -> tactic
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    20
  val metisF_tac : Proof.context -> thm list -> int -> tactic
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    21
  val metisFT_tac : Proof.context -> thm list -> int -> tactic
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
    22
  val metisHO_tac : Proof.context -> thm list -> int -> tactic
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    23
  val setup : theory -> theory
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    24
end
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    25
35826
1590abc3d42a renamed Sledgehammer structures
blanchet
parents: 35825
diff changeset
    26
structure Metis_Tactics : METIS_TACTICS =
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    27
struct
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    28
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43050
diff changeset
    29
open ATP_Translate
39494
bf7dd4902321 rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
blanchet
parents: 39450
diff changeset
    30
open Metis_Translate
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    31
open Metis_Reconstruct
35826
1590abc3d42a renamed Sledgehammer structures
blanchet
parents: 35825
diff changeset
    32
43050
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    33
fun method_binding_for_mode HO = @{binding metis}
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    34
  | method_binding_for_mode FO = @{binding metisF}
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    35
  | method_binding_for_mode FT = @{binding metisFT}
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    36
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    37
val metisN = Binding.qualified_name_of (method_binding_for_mode HO)
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    38
val metisF_N = Binding.qualified_name_of (method_binding_for_mode FO)
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    39
val metisFT_N = Binding.qualified_name_of (method_binding_for_mode FT)
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
    40
42616
92715b528e78 added Attrib.setup_config_XXX conveniences, with implicit setup of the background theory;
wenzelm
parents: 42552
diff changeset
    41
val type_lits = Attrib.setup_config_bool @{binding metis_type_lits} (K true)
92715b528e78 added Attrib.setup_config_XXX conveniences, with implicit setup of the background theory;
wenzelm
parents: 42552
diff changeset
    42
val new_skolemizer = Attrib.setup_config_bool @{binding metis_new_skolemizer} (K false)
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    43
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    44
fun is_false t = t aconv (HOLogic.mk_Trueprop HOLogic.false_const);
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    45
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    46
fun have_common_thm ths1 ths2 =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    47
  exists (member Thm.eq_thm ths1) (map Meson.make_meta_clause ths2)
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    48
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
    49
(*Determining which axiom clauses are actually used*)
39419
c9accfd621a5 "Metis." -> "Metis_" to reflect change in "metis.ML"
blanchet
parents: 39376
diff changeset
    50
fun used_axioms axioms (th, Metis_Proof.Axiom _) = SOME (lookth axioms th)
32994
ccc07fbbfefd removed some unreferenced material;
wenzelm
parents: 32956
diff changeset
    51
  | used_axioms _ _ = NONE;
24855
161eb8381b49 metis method: used theorems
paulson
parents: 24827
diff changeset
    52
39450
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    53
val clause_params =
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    54
  {ordering = Metis_KnuthBendixOrder.default,
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    55
   orderLiterals = Metis_Clause.UnsignedLiteralOrder,
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    56
   orderTerms = true}
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    57
val active_params =
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    58
  {clause = clause_params,
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    59
   prefactor = #prefactor Metis_Active.default,
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    60
   postfactor = #postfactor Metis_Active.default}
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    61
val waiting_params =
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    62
  {symbolsWeight = 1.0,
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    63
   variablesWeight = 0.0,
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    64
   literalsWeight = 0.0,
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
    65
   models = []}
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    66
val resolution_params = {active = active_params, waiting = waiting_params}
37573
7f987e8582a7 fewer dependencies
blanchet
parents: 37572
diff changeset
    67
37516
c81c86bfc18a have "metis" method and "metis_tac" fall back on "metisFT" upon failure, following a suggestion by Larry
blanchet
parents: 37509
diff changeset
    68
(* Main function to start Metis proof and reconstruction *)
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
    69
fun FOL_SOLVE (mode :: fallback_modes) ctxt cls ths0 =
42361
23f352990944 modernized structure Proof_Context;
wenzelm
parents: 42341
diff changeset
    70
  let val thy = Proof_Context.theory_of ctxt
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    71
      val type_lits = Config.get ctxt type_lits
39901
75d792edf634 make "cnf_axiom" work (after a fashion) in the absence of the axiom of choice
blanchet
parents: 39899
diff changeset
    72
      val new_skolemizer =
39950
f3c4849868b8 got rid of overkill "meson_choice" attribute;
blanchet
parents: 39946
diff changeset
    73
        Config.get ctxt new_skolemizer orelse null (Meson.choice_theorems thy)
35826
1590abc3d42a renamed Sledgehammer structures
blanchet
parents: 35825
diff changeset
    74
      val th_cls_pairs =
39894
35ae5cf8c96a encode number of skolem assumptions in them, for more efficient retrieval later
blanchet
parents: 39892
diff changeset
    75
        map2 (fn j => fn th =>
35ae5cf8c96a encode number of skolem assumptions in them, for more efficient retrieval later
blanchet
parents: 39892
diff changeset
    76
                (Thm.get_name_hint th,
39901
75d792edf634 make "cnf_axiom" work (after a fashion) in the absence of the axiom of choice
blanchet
parents: 39899
diff changeset
    77
                 Meson_Clausify.cnf_axiom ctxt new_skolemizer j th))
39894
35ae5cf8c96a encode number of skolem assumptions in them, for more efficient retrieval later
blanchet
parents: 39892
diff changeset
    78
             (0 upto length ths0 - 1) ths0
39887
74939e2afb95 second step in introducing the new Skolemizer -- notably, added procedure for discharging Skolem assumptions
blanchet
parents: 39886
diff changeset
    79
      val thss = map (snd o snd) th_cls_pairs
39938
0a2091f86eb4 fixed two bugs in new skolemizer: instantiations now take types into consideration, and rotate_tac is given the proper offset
blanchet
parents: 39937
diff changeset
    80
      val dischargers = map (fst o snd) th_cls_pairs
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    81
      val _ = trace_msg ctxt (fn () => "FOL_SOLVE: CONJECTURE CLAUSES")
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    82
      val _ = app (fn th => trace_msg ctxt (fn () => Display.string_of_thm ctxt th)) cls
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    83
      val _ = trace_msg ctxt (fn () => "THEOREM CLAUSES")
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    84
      val _ = app (app (fn th => trace_msg ctxt (fn () => Display.string_of_thm ctxt th))) thss
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39721
diff changeset
    85
      val (mode, {axioms, tfrees, old_skolems}) =
40157
a2f01956220e renaming
blanchet
parents: 39979
diff changeset
    86
        prepare_metis_problem mode ctxt type_lits cls thss
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
    87
      val _ = if null tfrees then ()
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    88
              else (trace_msg ctxt (fn () => "TFREE CLAUSES");
37643
f576af716aa6 rewrote the TPTP problem generation code more or less from scratch;
blanchet
parents: 37632
diff changeset
    89
                    app (fn TyLitFree ((s, _), (s', _)) =>
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    90
                            trace_msg ctxt (fn () => s ^ "(" ^ s' ^ ")")) tfrees)
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    91
      val _ = trace_msg ctxt (fn () => "CLAUSES GIVEN TO METIS")
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
    92
      val thms = map #1 axioms
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    93
      val _ = app (fn th => trace_msg ctxt (fn () => Metis_Thm.toString th)) thms
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    94
      val _ = trace_msg ctxt (fn () => "mode = " ^ string_of_mode mode)
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
    95
      val _ = trace_msg ctxt (fn () => "START METIS PROVE PROCESS")
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
    96
  in
33317
b4534348b8fd standardized filter/filter_out;
wenzelm
parents: 33316
diff changeset
    97
      case filter (is_false o prop_of) cls of
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
    98
          false_th::_ => [false_th RS @{thm FalseE}]
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
    99
        | [] =>
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   100
      case Metis_Resolution.new resolution_params {axioms = thms, conjecture = []}
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   101
           |> Metis_Resolution.loop of
39419
c9accfd621a5 "Metis." -> "Metis_" to reflect change in "metis.ML"
blanchet
parents: 39376
diff changeset
   102
          Metis_Resolution.Contradiction mth =>
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   103
            let val _ = trace_msg ctxt (fn () => "METIS RECONSTRUCTION START: " ^
39419
c9accfd621a5 "Metis." -> "Metis_" to reflect change in "metis.ML"
blanchet
parents: 39376
diff changeset
   104
                          Metis_Thm.toString mth)
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   105
                val ctxt' = fold Variable.declare_constraints (map prop_of cls) ctxt
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   106
                             (*add constraints arising from converting goal to clause form*)
39419
c9accfd621a5 "Metis." -> "Metis_" to reflect change in "metis.ML"
blanchet
parents: 39376
diff changeset
   107
                val proof = Metis_Proof.proof mth
42341
5a00af7f4978 removed obsolete Skolem counter in new Skolemizer
blanchet
parents: 42336
diff changeset
   108
                val result = fold (replay_one_inference ctxt' mode old_skolems)
5a00af7f4978 removed obsolete Skolem counter in new Skolemizer
blanchet
parents: 42336
diff changeset
   109
                                  proof axioms
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   110
                and used = map_filter (used_axioms axioms) proof
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   111
                val _ = trace_msg ctxt (fn () => "METIS COMPLETED...clauses actually used:")
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   112
                val _ = app (fn th => trace_msg ctxt (fn () => Display.string_of_thm ctxt th)) used
39887
74939e2afb95 second step in introducing the new Skolemizer -- notably, added procedure for discharging Skolem assumptions
blanchet
parents: 39886
diff changeset
   113
                val unused = th_cls_pairs |> map_filter (fn (name, (_, cls)) =>
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   114
                  if have_common_thm used cls then NONE else SOME name)
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   115
            in
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   116
                if not (null cls) andalso not (have_common_thm used cls) then
42650
552eae49f97d reintroduce this idea of running "metisFT" after a failed "metis" -- I took it out in e85ce10cef1a because I couldn't think of a reasonable use case, but now that ATPs use sound encodings and include dangerous facts (e.g. True_or_False) it makes more sense than ever to run "metisFT" after "metis"
blanchet
parents: 42616
diff changeset
   117
                  verbose_warning ctxt "The assumptions are inconsistent"
36383
6adf1068ac0f better error reporting;
blanchet
parents: 36230
diff changeset
   118
                else
6adf1068ac0f better error reporting;
blanchet
parents: 36230
diff changeset
   119
                  ();
6adf1068ac0f better error reporting;
blanchet
parents: 36230
diff changeset
   120
                if not (null unused) then
42650
552eae49f97d reintroduce this idea of running "metisFT" after a failed "metis" -- I took it out in e85ce10cef1a because I couldn't think of a reasonable use case, but now that ATPs use sound encodings and include dangerous facts (e.g. True_or_False) it makes more sense than ever to run "metisFT" after "metis"
blanchet
parents: 42616
diff changeset
   121
                  verbose_warning ctxt ("Unused theorems: " ^ commas_quote unused)
36230
43d10a494c91 added warning about inconsistent context to Metis;
blanchet
parents: 36170
diff changeset
   122
                else
43d10a494c91 added warning about inconsistent context to Metis;
blanchet
parents: 36170
diff changeset
   123
                  ();
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   124
                case result of
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   125
                    (_,ith)::_ =>
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   126
                        (trace_msg ctxt (fn () => "Success: " ^ Display.string_of_thm ctxt ith);
39887
74939e2afb95 second step in introducing the new Skolemizer -- notably, added procedure for discharging Skolem assumptions
blanchet
parents: 39886
diff changeset
   127
                         [discharge_skolem_premises ctxt dischargers ith])
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   128
                  | _ => (trace_msg ctxt (fn () => "Metis: No result"); [])
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   129
            end
39419
c9accfd621a5 "Metis." -> "Metis_" to reflect change in "metis.ML"
blanchet
parents: 39376
diff changeset
   130
        | Metis_Resolution.Satisfiable _ =>
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   131
            (trace_msg ctxt (fn () => "Metis: No first-order proof with the lemmas supplied");
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   132
             if null fallback_modes then
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   133
               ()
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   134
             else
42650
552eae49f97d reintroduce this idea of running "metisFT" after a failed "metis" -- I took it out in e85ce10cef1a because I couldn't think of a reasonable use case, but now that ATPs use sound encodings and include dangerous facts (e.g. True_or_False) it makes more sense than ever to run "metisFT" after "metis"
blanchet
parents: 42616
diff changeset
   135
               raise METIS ("FOL_SOLVE",
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   136
                            "No first-order proof with the lemmas supplied");
38097
5e4ad2df09f3 revert exception throwing in FOL_SOLVE, since they're not caught anyway
blanchet
parents: 38028
diff changeset
   137
             [])
42733
01ef1c3d9cfd more robust exception handling in Metis (also works if there are several subgoals)
blanchet
parents: 42650
diff changeset
   138
  end
01ef1c3d9cfd more robust exception handling in Metis (also works if there are several subgoals)
blanchet
parents: 42650
diff changeset
   139
  handle METIS (loc, msg) =>
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   140
         case fallback_modes of
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   141
           [] => error ("Failed to replay Metis proof in Isabelle." ^
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   142
                        (if Config.get ctxt verbose then "\n" ^ loc ^ ": " ^ msg
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   143
                         else ""))
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   144
         | mode :: _ =>
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   145
           (verbose_warning ctxt
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   146
                ("Falling back on " ^
43050
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
   147
                 quote (Binding.qualified_name_of
59284a13abc4 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents: 43034
diff changeset
   148
                            (method_binding_for_mode mode)) ^ "...");
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   149
            FOL_SOLVE fallback_modes ctxt cls ths0)
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   150
42847
blanchet
parents: 42747
diff changeset
   151
val neg_clausify =
38028
22dcaec5fa77 minor refactoring
blanchet
parents: 38027
diff changeset
   152
  single
22dcaec5fa77 minor refactoring
blanchet
parents: 38027
diff changeset
   153
  #> Meson.make_clauses_unsorted
39890
a1695e2169d0 finished renaming file and module
blanchet
parents: 39887
diff changeset
   154
  #> map Meson_Clausify.introduce_combinators_in_theorem
38028
22dcaec5fa77 minor refactoring
blanchet
parents: 38027
diff changeset
   155
  #> Meson.finish_cnf
22dcaec5fa77 minor refactoring
blanchet
parents: 38027
diff changeset
   156
39269
c2795d8a2461 use definitional CNF for the goal if at least one of the premisses would lead to too many clauses in Meson
blanchet
parents: 39267
diff changeset
   157
fun preskolem_tac ctxt st0 =
c2795d8a2461 use definitional CNF for the goal if at least one of the premisses would lead to too many clauses in Meson
blanchet
parents: 39267
diff changeset
   158
  (if exists (Meson.has_too_many_clauses ctxt)
c2795d8a2461 use definitional CNF for the goal if at least one of the premisses would lead to too many clauses in Meson
blanchet
parents: 39267
diff changeset
   159
             (Logic.prems_of_goal (prop_of st0) 1) then
42336
d63d43e85879 improve definitional CNF on goal by moving "not" past the quantifiers
blanchet
parents: 40665
diff changeset
   160
     Simplifier.full_simp_tac (Meson_Clausify.ss_only @{thms not_all not_ex}) 1
d63d43e85879 improve definitional CNF on goal by moving "not" past the quantifiers
blanchet
parents: 40665
diff changeset
   161
     THEN cnf.cnfx_rewrite_tac ctxt 1
39269
c2795d8a2461 use definitional CNF for the goal if at least one of the premisses would lead to too many clauses in Meson
blanchet
parents: 39267
diff changeset
   162
   else
c2795d8a2461 use definitional CNF for the goal if at least one of the premisses would lead to too many clauses in Meson
blanchet
parents: 39267
diff changeset
   163
     all_tac) st0
c2795d8a2461 use definitional CNF for the goal if at least one of the premisses would lead to too many clauses in Meson
blanchet
parents: 39267
diff changeset
   164
38652
e063be321438 perform eta-expansion of quantifier bodies in Sledgehammer translation when needed + transform elim rules later;
blanchet
parents: 38632
diff changeset
   165
val type_has_top_sort =
e063be321438 perform eta-expansion of quantifier bodies in Sledgehammer translation when needed + transform elim rules later;
blanchet
parents: 38632
diff changeset
   166
  exists_subtype (fn TFree (_, []) => true | TVar (_, []) => true | _ => false)
e063be321438 perform eta-expansion of quantifier bodies in Sledgehammer translation when needed + transform elim rules later;
blanchet
parents: 38632
diff changeset
   167
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   168
fun generic_metis_tac modes ctxt ths i st0 =
37926
e6ff246c0cdb renamings + only need second component of name pool to reconstruct proofs
blanchet
parents: 37925
diff changeset
   169
  let
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   170
    val _ = trace_msg ctxt (fn () =>
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   171
        "Metis called with theorems " ^
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   172
        cat_lines (map (Display.string_of_thm ctxt) ths))
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   173
  in
37626
1146291fe718 move blacklisting completely out of the clausifier;
blanchet
parents: 37625
diff changeset
   174
    if exists_type type_has_top_sort (prop_of st0) then
42650
552eae49f97d reintroduce this idea of running "metisFT" after a failed "metis" -- I took it out in e85ce10cef1a because I couldn't think of a reasonable use case, but now that ATPs use sound encodings and include dangerous facts (e.g. True_or_False) it makes more sense than ever to run "metisFT" after "metis"
blanchet
parents: 42616
diff changeset
   175
      (verbose_warning ctxt "Proof state contains the universal sort {}";
40665
1a65f0c74827 added "verbose" option to Metis to shut up its warnings if necessary
blanchet
parents: 40262
diff changeset
   176
       Seq.empty)
35568
8fbbfc39508f renamed type_has_empty_sort to type_has_topsort -- {} is the full universal sort;
wenzelm
parents: 34087
diff changeset
   177
    else
42847
blanchet
parents: 42747
diff changeset
   178
      Meson.MESON (preskolem_tac ctxt) (maps neg_clausify)
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   179
                  (fn cls => resolve_tac (FOL_SOLVE modes ctxt cls ths) 1)
39594
624d6c0e220d revert b96941dddd04 and c13b4589fddf, which dramatically inflate proof terms
blanchet
parents: 39560
diff changeset
   180
                  ctxt i st0
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   181
  end
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   182
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   183
val metis_modes = [HO, FT]
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   184
val metisF_modes = [FO, FT]
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   185
val metisFT_modes = [FT]
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   186
val metisHO_modes = [HO]
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   187
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   188
val metis_tac = generic_metis_tac metis_modes
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   189
val metisF_tac = generic_metis_tac metisF_modes
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   190
val metisFT_tac = generic_metis_tac metisFT_modes
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   191
val metisHO_tac = generic_metis_tac metisHO_modes
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   192
38632
9cde57cdd0e3 treat "using X by metis" (more or less) the same as "by (metis X)"
blanchet
parents: 38614
diff changeset
   193
(* Whenever "X" has schematic type variables, we treat "using X by metis" as
9cde57cdd0e3 treat "using X by metis" (more or less) the same as "by (metis X)"
blanchet
parents: 38614
diff changeset
   194
   "by (metis X)", to prevent "Subgoal.FOCUS" from freezing the type variables.
9cde57cdd0e3 treat "using X by metis" (more or less) the same as "by (metis X)"
blanchet
parents: 38614
diff changeset
   195
   We don't do it for nonschematic facts "X" because this breaks a few proofs
9cde57cdd0e3 treat "using X by metis" (more or less) the same as "by (metis X)"
blanchet
parents: 38614
diff changeset
   196
   (in the rare and subtle case where a proof relied on extensionality not being
38994
7c655a491bce fiddled with fudge factor (based on Mirabelle)
blanchet
parents: 38864
diff changeset
   197
   applied) and brings few benefits. *)
38632
9cde57cdd0e3 treat "using X by metis" (more or less) the same as "by (metis X)"
blanchet
parents: 38614
diff changeset
   198
val has_tvar =
9cde57cdd0e3 treat "using X by metis" (more or less) the same as "by (metis X)"
blanchet
parents: 38614
diff changeset
   199
  exists_type (exists_subtype (fn TVar _ => true | _ => false)) o prop_of
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   200
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   201
fun setup_method (modes as mode :: _) =
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   202
  Method.setup (method_binding_for_mode mode)
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   203
    (Attrib.thms >> (fn ths => fn ctxt =>
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   204
       METHOD (fn facts =>
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   205
                  let
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   206
                    val (schem_facts, nonschem_facts) =
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   207
                      List.partition has_tvar facts
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   208
                  in
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   209
                    HEADGOAL (Method.insert_tac nonschem_facts THEN'
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   210
                              CHANGED_PROP
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   211
                              o generic_metis_tac modes ctxt (schem_facts @ ths))
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   212
                  end)))
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   213
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   214
val setup =
43034
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   215
  [(metis_modes, "Metis for FOL and HOL problems"),
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   216
   (metisF_modes, "Metis for FOL problems"),
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   217
   (metisFT_modes, "Metis for FOL/HOL problems with fully-typed translation")]
18259246abb5 try both "metis" and (on failure) "metisFT" in replay
blanchet
parents: 42847
diff changeset
   218
  |> fold (uncurry setup_method)
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   219
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   220
end;