src/HOL/Tools/Metis/metis_tactic.ML
author blanchet
Fri, 27 Jun 2014 18:27:37 +0200
changeset 57408 39b3562e9edc
parent 57263 2b6a96cc64c9
child 58818 ee85e7b82d00
permissions -rw-r--r--
tuned whitespace and parentheses
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
44651
5d6a11e166cf renamed "Metis_Tactics" to "Metis_Tactic", now that there is only one Metis tactic ("metisFT" is legacy)
blanchet
parents: 44634
diff changeset
     1
(*  Title:      HOL/Tools/Metis/metis_tactic.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
44651
5d6a11e166cf renamed "Metis_Tactics" to "Metis_Tactic", now that there is only one Metis tactic ("metisFT" is legacy)
blanchet
parents: 44634
diff changeset
    10
signature METIS_TACTIC =
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    11
sig
39979
b13515940b53 added "trace_meson" configuration option, replacing old-fashioned reference
blanchet
parents: 39978
diff changeset
    12
  val trace : bool Config.T
40665
1a65f0c74827 added "verbose" option to Metis to shut up its warnings if necessary
blanchet
parents: 40262
diff changeset
    13
  val verbose : bool Config.T
50705
0e943b33d907 use new skolemizer for reconstructing skolemization steps in Isar proofs (because the old skolemizer messes up the order of the Skolem arguments)
blanchet
parents: 50694
diff changeset
    14
  val new_skolem : bool Config.T
47039
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
    15
  val advisory_simp : bool Config.T
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
    16
  val metis_tac_unused : string list -> string -> Proof.context -> thm list -> int -> thm ->
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
    17
    thm list * thm Seq.seq
54756
blanchet
parents: 54742
diff changeset
    18
  val metis_tac : string list -> string -> Proof.context -> thm list -> int -> tactic
45521
0cd6e59bd0b5 give each time slice its own lambda translation
blanchet
parents: 45519
diff changeset
    19
  val metis_lam_transs : string list
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
    20
  val parse_metis_options : (string list option * string option) parser
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    21
  val setup : theory -> theory
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    22
end
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    23
44651
5d6a11e166cf renamed "Metis_Tactics" to "Metis_Tactic", now that there is only one Metis tactic ("metisFT" is legacy)
blanchet
parents: 44634
diff changeset
    24
structure Metis_Tactic : METIS_TACTIC =
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    25
struct
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    26
46320
0b8b73b49848 renamed two files to make room for a new file
blanchet
parents: 46301
diff changeset
    27
open ATP_Problem_Generate
0b8b73b49848 renamed two files to make room for a new file
blanchet
parents: 46301
diff changeset
    28
open ATP_Proof_Reconstruct
0b8b73b49848 renamed two files to make room for a new file
blanchet
parents: 46301
diff changeset
    29
open Metis_Generate
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    30
open Metis_Reconstruct
35826
1590abc3d42a renamed Sledgehammer structures
blanchet
parents: 35825
diff changeset
    31
54756
blanchet
parents: 54742
diff changeset
    32
val new_skolem = Attrib.setup_config_bool @{binding metis_new_skolem} (K false)
blanchet
parents: 54742
diff changeset
    33
val advisory_simp = Attrib.setup_config_bool @{binding metis_advisory_simp} (K true)
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    34
43134
0c82e00ba63e make sure no warnings are given for polymorphic facts where we use a monomorphic instance
blanchet
parents: 43133
diff changeset
    35
(* Designed to work also with monomorphic instances of polymorphic theorems. *)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    36
fun have_common_thm ths1 ths2 =
54756
blanchet
parents: 54742
diff changeset
    37
  exists (member (Term.aconv_untyped o pairself prop_of) ths1) (map Meson.make_meta_clause ths2)
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
    38
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
    39
(*Determining which axiom clauses are actually used*)
39419
c9accfd621a5 "Metis." -> "Metis_" to reflect change in "metis.ML"
blanchet
parents: 39376
diff changeset
    40
fun used_axioms axioms (th, Metis_Proof.Axiom _) = SOME (lookth axioms th)
43128
a19826080596 tuned names
blanchet
parents: 43103
diff changeset
    41
  | used_axioms _ _ = NONE
24855
161eb8381b49 metis method: used theorems
paulson
parents: 24827
diff changeset
    42
43129
4301f1c123d6 support lightweight tags in new Metis
blanchet
parents: 43128
diff changeset
    43
(* Lightweight predicate type information comes in two flavors, "t = t'" and
4301f1c123d6 support lightweight tags in new Metis
blanchet
parents: 43128
diff changeset
    44
   "t => t'", where "t" and "t'" are the same term modulo type tags.
4301f1c123d6 support lightweight tags in new Metis
blanchet
parents: 43128
diff changeset
    45
   In Isabelle, type tags are stripped away, so we are left with "t = t" or
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43136
diff changeset
    46
   "t => t". Type tag idempotence is also handled this way. *)
52031
9a9238342963 tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents: 51717
diff changeset
    47
fun reflexive_or_trivial_of_metis ctxt type_enc sym_tab concealed mth =
43136
cf5cda219058 handle lightweight tags sym theorems gracefully in the presence of TVars with interesting type classes
blanchet
parents: 43135
diff changeset
    48
  let val thy = Proof_Context.theory_of ctxt in
57408
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    49
    (case hol_clause_of_metis ctxt type_enc sym_tab concealed mth of
43136
cf5cda219058 handle lightweight tags sym theorems gracefully in the presence of TVars with interesting type classes
blanchet
parents: 43135
diff changeset
    50
      Const (@{const_name HOL.eq}, _) $ _ $ t =>
44408
30ea62ab4f16 made reconstruction of type tag equalities "\?x = \?x" reliable
blanchet
parents: 44402
diff changeset
    51
      let
30ea62ab4f16 made reconstruction of type tag equalities "\?x = \?x" reliable
blanchet
parents: 44402
diff changeset
    52
        val ct = cterm_of thy t
30ea62ab4f16 made reconstruction of type tag equalities "\?x = \?x" reliable
blanchet
parents: 44402
diff changeset
    53
        val cT = ctyp_of_term ct
30ea62ab4f16 made reconstruction of type tag equalities "\?x = \?x" reliable
blanchet
parents: 44402
diff changeset
    54
      in refl |> Drule.instantiate' [SOME cT] [SOME ct] end
43136
cf5cda219058 handle lightweight tags sym theorems gracefully in the presence of TVars with interesting type classes
blanchet
parents: 43135
diff changeset
    55
    | Const (@{const_name disj}, _) $ t1 $ t2 =>
cf5cda219058 handle lightweight tags sym theorems gracefully in the presence of TVars with interesting type classes
blanchet
parents: 43135
diff changeset
    56
      (if can HOLogic.dest_not t1 then t2 else t1)
cf5cda219058 handle lightweight tags sym theorems gracefully in the presence of TVars with interesting type classes
blanchet
parents: 43135
diff changeset
    57
      |> HOLogic.mk_Trueprop |> cterm_of thy |> Thm.trivial
57408
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    58
    | _ => raise Fail "expected reflexive or trivial clause")
43136
cf5cda219058 handle lightweight tags sym theorems gracefully in the presence of TVars with interesting type classes
blanchet
parents: 43135
diff changeset
    59
  end
43129
4301f1c123d6 support lightweight tags in new Metis
blanchet
parents: 43128
diff changeset
    60
  |> Meson.make_meta_clause
4301f1c123d6 support lightweight tags in new Metis
blanchet
parents: 43128
diff changeset
    61
52031
9a9238342963 tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents: 51717
diff changeset
    62
fun lam_lifted_of_metis ctxt type_enc sym_tab concealed mth =
45511
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    63
  let
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    64
    val thy = Proof_Context.theory_of ctxt
54742
7a86358a3c0b proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
wenzelm
parents: 54500
diff changeset
    65
    val tac = rewrite_goals_tac ctxt @{thms lambda_def [abs_def]} THEN rtac refl 1
52031
9a9238342963 tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents: 51717
diff changeset
    66
    val t = hol_clause_of_metis ctxt type_enc sym_tab concealed mth
45511
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    67
    val ct = cterm_of thy (HOLogic.mk_Trueprop t)
54883
dd04a8b654fc proper context for norm_hhf and derived operations;
wenzelm
parents: 54756
diff changeset
    68
  in Goal.prove_internal ctxt [] ct (K tac) |> Meson.make_meta_clause end
45511
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    69
45570
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    70
fun add_vars_and_frees (t $ u) = fold (add_vars_and_frees) [t, u]
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    71
  | add_vars_and_frees (Abs (_, _, t)) = add_vars_and_frees t
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    72
  | add_vars_and_frees (t as Var _) = insert (op =) t
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    73
  | add_vars_and_frees (t as Free _) = insert (op =) t
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    74
  | add_vars_and_frees _ = I
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    75
45569
eb30a5490543 wrap lambdas earlier, to get more control over beta/eta
blanchet
parents: 45568
diff changeset
    76
fun introduce_lam_wrappers ctxt th =
45511
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    77
  if Meson_Clausify.is_quasi_lambda_free (prop_of th) then
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    78
    th
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    79
  else
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    80
    let
45570
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    81
      val thy = Proof_Context.theory_of ctxt
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    82
      fun conv first ctxt ct =
45511
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    83
        if Meson_Clausify.is_quasi_lambda_free (term_of ct) then
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
    84
          Thm.reflexive ct
57408
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    85
        else
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    86
          (case term_of ct of
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    87
            Abs (_, _, u) =>
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    88
            if first then
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    89
              (case add_vars_and_frees u [] of
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    90
                [] =>
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    91
                Conv.abs_conv (conv false o snd) ctxt ct
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    92
                |> (fn th => Meson.first_order_resolve th @{thm Metis.eq_lambdaI})
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    93
              | v :: _ =>
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    94
                Abs (Name.uu, fastype_of v, abstract_over (v, term_of ct)) $ v
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    95
                |> cterm_of thy
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    96
                |> Conv.comb_conv (conv true ctxt))
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    97
            else
45570
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
    98
              Conv.abs_conv (conv false o snd) ctxt ct
57408
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
    99
          | Const (@{const_name Meson.skolem}, _) $ _ => Thm.reflexive ct
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
   100
          | _ => Conv.comb_conv (conv true ctxt) ct)
45570
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   101
      val eq_th = conv true ctxt (cprop_of th)
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   102
      (* We replace the equation's left-hand side with a beta-equivalent term
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   103
         so that "Thm.equal_elim" works below. *)
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   104
      val t0 $ _ $ t2 = prop_of eq_th
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   105
      val eq_ct = t0 $ prop_of th $ t2 |> cterm_of thy
54883
dd04a8b654fc proper context for norm_hhf and derived operations;
wenzelm
parents: 54756
diff changeset
   106
      val eq_th' = Goal.prove_internal ctxt [] eq_ct (K (rtac eq_th 1))
45570
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   107
    in Thm.equal_elim eq_th' th end
45511
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
   108
47039
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   109
fun clause_params ordering =
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   110
  {ordering = ordering,
44492
a330c0608da8 avoid using ":" for anything but systematic type tag annotations, because Hurd's Metis gives it that special semantics
blanchet
parents: 44411
diff changeset
   111
   orderLiterals = Metis_Clause.UnsignedLiteralOrder,
39450
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
   112
   orderTerms = true}
47039
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   113
fun active_params ordering =
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   114
  {clause = clause_params ordering,
39450
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
   115
   prefactor = #prefactor Metis_Active.default,
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
   116
   postfactor = #postfactor Metis_Active.default}
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
   117
val waiting_params =
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
   118
  {symbolsWeight = 1.0,
47047
10bece4ac87e more conservative Metis defaults, for backward compatiblity (as illustrated by one "metis" call in "Auth/KerberosV")
blanchet
parents: 47045
diff changeset
   119
   variablesWeight = 0.05,
10bece4ac87e more conservative Metis defaults, for backward compatiblity (as illustrated by one "metis" call in "Auth/KerberosV")
blanchet
parents: 47045
diff changeset
   120
   literalsWeight = 0.01,
39450
7e9879fbb7c5 supply the Metis parameter defaults as argument, instead of patching the Metis sources;
blanchet
parents: 39419
diff changeset
   121
   models = []}
47039
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   122
fun resolution_params ordering =
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   123
  {active = active_params ordering, waiting = waiting_params}
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   124
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   125
fun kbo_advisory_simp_ordering ord_info =
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   126
  let
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   127
    fun weight (m, _) =
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   128
      AList.lookup (op =) ord_info (Metis_Name.toString m) |> the_default 1
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   129
    fun precedence p =
57408
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
   130
      (case int_ord (pairself weight p) of
47039
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   131
        EQUAL => #precedence Metis_KnuthBendixOrder.default p
57408
39b3562e9edc tuned whitespace and parentheses
blanchet
parents: 57263
diff changeset
   132
      | ord => ord)
47039
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   133
  in {weight = weight, precedence = precedence} end
37573
7f987e8582a7 fewer dependencies
blanchet
parents: 37572
diff changeset
   134
55285
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   135
fun metis_call type_enc lam_trans =
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   136
  let
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   137
    val type_enc =
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   138
      (case AList.find (fn (enc, encs) => enc = hd encs) type_enc_aliases type_enc of
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   139
        [alias] => alias
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   140
      | _ => type_enc)
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   141
    val opts =
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   142
      [] |> type_enc <> partial_typesN ? cons type_enc
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   143
         |> lam_trans <> default_metis_lam_trans ? cons lam_trans
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   144
  in metisN ^ (if null opts then "" else " (" ^ commas opts ^ ")") end
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
   145
50875
bfb626265782 less brutal Metis failure -- the brutality was accidentally introduced by df8ae0590be2
blanchet
parents: 50705
diff changeset
   146
exception METIS_UNPROVABLE of unit
bfb626265782 less brutal Metis failure -- the brutality was accidentally introduced by df8ae0590be2
blanchet
parents: 50705
diff changeset
   147
37516
c81c86bfc18a have "metis" method and "metis_tac" fall back on "metisFT" upon failure, following a suggestion by Larry
blanchet
parents: 37509
diff changeset
   148
(* Main function to start Metis proof and reconstruction *)
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   149
fun FOL_SOLVE unused (type_enc :: fallback_type_encs) lam_trans ctxt cls ths0 =
42361
23f352990944 modernized structure Proof_Context;
wenzelm
parents: 42341
diff changeset
   150
  let val thy = Proof_Context.theory_of ctxt
50705
0e943b33d907 use new skolemizer for reconstructing skolemization steps in Isar proofs (because the old skolemizer messes up the order of the Skolem arguments)
blanchet
parents: 50694
diff changeset
   151
      val new_skolem =
0e943b33d907 use new skolemizer for reconstructing skolemization steps in Isar proofs (because the old skolemizer messes up the order of the Skolem arguments)
blanchet
parents: 50694
diff changeset
   152
        Config.get ctxt new_skolem orelse null (Meson.choice_theorems thy)
46365
547d1a1dcaf6 rename lambda translation schemes
blanchet
parents: 46320
diff changeset
   153
      val do_lams =
547d1a1dcaf6 rename lambda translation schemes
blanchet
parents: 46320
diff changeset
   154
        (lam_trans = liftingN orelse lam_trans = lam_liftingN)
547d1a1dcaf6 rename lambda translation schemes
blanchet
parents: 46320
diff changeset
   155
        ? introduce_lam_wrappers ctxt
35826
1590abc3d42a renamed Sledgehammer structures
blanchet
parents: 35825
diff changeset
   156
      val th_cls_pairs =
39894
35ae5cf8c96a encode number of skolem assumptions in them, for more efficient retrieval later
blanchet
parents: 39892
diff changeset
   157
        map2 (fn j => fn th =>
35ae5cf8c96a encode number of skolem assumptions in them, for more efficient retrieval later
blanchet
parents: 39892
diff changeset
   158
                (Thm.get_name_hint th,
45570
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   159
                 th |> Drule.eta_contraction_rule
57263
2b6a96cc64c9 simplified code
blanchet
parents: 55523
diff changeset
   160
                    |> Meson_Clausify.cnf_axiom ctxt new_skolem (lam_trans = combsN) j
45570
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   161
                    ||> map do_lams))
39894
35ae5cf8c96a encode number of skolem assumptions in them, for more efficient retrieval later
blanchet
parents: 39892
diff changeset
   162
             (0 upto length ths0 - 1) ths0
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   163
      val ths = maps (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
   164
      val dischargers = map (fst o snd) th_cls_pairs
45570
6d95a66cce00 pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
blanchet
parents: 45569
diff changeset
   165
      val cls = cls |> map (Drule.eta_contraction_rule #> do_lams)
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   166
      val _ = trace_msg ctxt (K "FOL_SOLVE: CONJECTURE CLAUSES")
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   167
      val _ = app (fn th => trace_msg ctxt (fn () => Display.string_of_thm ctxt th)) cls
44411
e3629929b171 change Metis's default settings if type information axioms are generated
blanchet
parents: 44408
diff changeset
   168
      val _ = trace_msg ctxt (fn () => "type_enc = " ^ type_enc)
52031
9a9238342963 tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents: 51717
diff changeset
   169
      val type_enc = type_enc_of_string Strict type_enc
47039
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   170
      val (sym_tab, axioms, ord_info, concealed) =
57263
2b6a96cc64c9 simplified code
blanchet
parents: 55523
diff changeset
   171
        generate_metis_problem ctxt type_enc lam_trans cls ths
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43136
diff changeset
   172
      fun get_isa_thm mth Isa_Reflexive_or_Trivial =
52031
9a9238342963 tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents: 51717
diff changeset
   173
          reflexive_or_trivial_of_metis ctxt type_enc sym_tab concealed mth
45511
9b0f8ca4388e continued implementation of lambda-lifting in Metis
blanchet
parents: 45508
diff changeset
   174
        | get_isa_thm mth Isa_Lambda_Lifted =
52031
9a9238342963 tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents: 51717
diff changeset
   175
          lam_lifted_of_metis ctxt type_enc sym_tab concealed mth
45569
eb30a5490543 wrap lambdas earlier, to get more control over beta/eta
blanchet
parents: 45568
diff changeset
   176
        | get_isa_thm _ (Isa_Raw ith) = ith
eb30a5490543 wrap lambdas earlier, to get more control over beta/eta
blanchet
parents: 45568
diff changeset
   177
      val axioms = axioms |> map (fn (mth, ith) => (mth, get_isa_thm mth ith))
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   178
      val _ = trace_msg ctxt (K "ISABELLE CLAUSES")
45559
22d6fb988306 avoid spurious messages in "lam_lifting" mode
blanchet
parents: 45558
diff changeset
   179
      val _ = app (fn (_, ith) => trace_msg ctxt (fn () => Display.string_of_thm ctxt ith)) axioms
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   180
      val _ = trace_msg ctxt (K "METIS CLAUSES")
45559
22d6fb988306 avoid spurious messages in "lam_lifting" mode
blanchet
parents: 45558
diff changeset
   181
      val _ = app (fn (mth, _) => trace_msg ctxt (fn () => Metis_Thm.toString mth)) axioms
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   182
      val _ = trace_msg ctxt (K "START METIS PROVE PROCESS")
47039
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   183
      val ordering =
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   184
        if Config.get ctxt advisory_simp then
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   185
          kbo_advisory_simp_ordering (ord_info ())
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   186
        else
1b36a05a070d added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents: 47015
diff changeset
   187
          Metis_KnuthBendixOrder.default
50875
bfb626265782 less brutal Metis failure -- the brutality was accidentally introduced by df8ae0590be2
blanchet
parents: 50705
diff changeset
   188
    fun fall_back () =
bfb626265782 less brutal Metis failure -- the brutality was accidentally introduced by df8ae0590be2
blanchet
parents: 50705
diff changeset
   189
      (verbose_warning ctxt
55257
abfd7b90bba2 rationalized threading of 'metis' arguments
blanchet
parents: 55239
diff changeset
   190
           ("Falling back on " ^ quote (metis_call (hd fallback_type_encs) lam_trans) ^ "...");
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   191
       FOL_SOLVE unused fallback_type_encs lam_trans ctxt cls ths0)
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   192
  in
50875
bfb626265782 less brutal Metis failure -- the brutality was accidentally introduced by df8ae0590be2
blanchet
parents: 50705
diff changeset
   193
    (case filter (fn t => prop_of t aconv @{prop False}) cls of
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   194
       false_th :: _ => [false_th RS @{thm FalseE}]
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   195
     | [] =>
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   196
     (case Metis_Resolution.loop (Metis_Resolution.new (resolution_params ordering)
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   197
         {axioms = axioms |> map fst, conjecture = []}) of
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   198
       Metis_Resolution.Contradiction mth =>
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   199
       let
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   200
         val _ = trace_msg ctxt (fn () => "METIS RECONSTRUCTION START: " ^ Metis_Thm.toString mth)
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   201
         val ctxt' = fold Variable.declare_constraints (map prop_of cls) ctxt
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   202
                      (*add constraints arising from converting goal to clause form*)
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   203
         val proof = Metis_Proof.proof mth
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   204
         val result = fold (replay_one_inference ctxt' type_enc concealed sym_tab) proof axioms
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   205
         val used = map_filter (used_axioms axioms) proof
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   206
         val _ = trace_msg ctxt (K "METIS COMPLETED; clauses actually used:")
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   207
         val _ = app (fn th => trace_msg ctxt (fn () => Display.string_of_thm ctxt th)) used
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   208
         val (used_th_cls_pairs, unused_th_cls_pairs) =
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   209
           List.partition (have_common_thm used o snd o snd) th_cls_pairs
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   210
         val unused_ths = maps (snd o snd) unused_th_cls_pairs
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   211
         val unused_names = map fst unused_th_cls_pairs
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   212
       in
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   213
         unused := unused_ths;
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   214
         if not (null unused_names) then
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   215
           verbose_warning ctxt ("Unused theorems: " ^ commas_quote unused_names)
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   216
         else
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   217
           ();
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   218
         if not (null cls) andalso not (have_common_thm used cls) then
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   219
           verbose_warning ctxt "The assumptions are inconsistent"
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   220
         else
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   221
           ();
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   222
         (case result of
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   223
           (_, ith) :: _ =>
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   224
           (trace_msg ctxt (fn () => "Success: " ^ Display.string_of_thm ctxt ith);
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   225
            [discharge_skolem_premises ctxt dischargers ith])
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   226
         | _ => (trace_msg ctxt (K "Metis: No result"); []))
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   227
       end
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   228
     | Metis_Resolution.Satisfiable _ =>
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   229
       (trace_msg ctxt (K "Metis: No first-order proof with the supplied lemmas");
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   230
        raise METIS_UNPROVABLE ()))
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   231
    handle METIS_UNPROVABLE () => if null fallback_type_encs then [] else fall_back ()
50875
bfb626265782 less brutal Metis failure -- the brutality was accidentally introduced by df8ae0590be2
blanchet
parents: 50705
diff changeset
   232
         | METIS_RECONSTRUCT (loc, msg) =>
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   233
           if null fallback_type_encs then
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   234
             (verbose_warning ctxt ("Failed to replay Metis proof\n" ^ loc ^ ": " ^ msg); [])
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   235
           else
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   236
             fall_back ())
42733
01ef1c3d9cfd more robust exception handling in Metis (also works if there are several subgoals)
blanchet
parents: 42650
diff changeset
   237
  end
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   238
45508
b216dc1b3630 started implementing lambda-lifting in Metis
blanchet
parents: 45042
diff changeset
   239
fun neg_clausify ctxt combinators =
38028
22dcaec5fa77 minor refactoring
blanchet
parents: 38027
diff changeset
   240
  single
43964
9338aa218f09 thread proper context through, to make sure that "using [[meson_max_clauses = 200]]" is not ignored when clausifying the conjecture
blanchet
parents: 43963
diff changeset
   241
  #> Meson.make_clauses_unsorted ctxt
55236
8d61b0aa7a0d proper context for printing;
wenzelm
parents: 54914
diff changeset
   242
  #> combinators ? map (Meson_Clausify.introduce_combinators_in_theorem ctxt)
38028
22dcaec5fa77 minor refactoring
blanchet
parents: 38027
diff changeset
   243
  #> Meson.finish_cnf
22dcaec5fa77 minor refactoring
blanchet
parents: 38027
diff changeset
   244
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
   245
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
   246
  (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
   247
             (Logic.prems_of_goal (prop_of st0) 1) then
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50875
diff changeset
   248
     Simplifier.full_simp_tac (Meson_Clausify.ss_only @{thms not_all not_ex} ctxt) 1
55239
97921d23ebe3 more standard file/module names;
wenzelm
parents: 55236
diff changeset
   249
     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
   250
   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
   251
     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
   252
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   253
fun metis_tac_unused type_encs0 lam_trans ctxt ths i st0 =
37926
e6ff246c0cdb renamings + only need second component of name pool to reconstruct proofs
blanchet
parents: 37925
diff changeset
   254
  let
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   255
    val unused = Unsynchronized.ref []
55520
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   256
    val type_encs = if null type_encs0 then partial_type_encs else type_encs0
39978
11bfb7e7cc86 added "trace_metis" configuration option, replacing old-fashioned references
blanchet
parents: 39964
diff changeset
   257
    val _ = trace_msg ctxt (fn () =>
55315
54b0352fb46d removed legacy 'metisFT' method
blanchet
parents: 55285
diff changeset
   258
      "Metis called with theorems\n" ^ cat_lines (map (Display.string_of_thm ctxt) ths))
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   259
    val type_encs = type_encs |> maps unalias_type_enc
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   260
    val combs = (lam_trans = combsN)
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   261
    fun tac clause = resolve_tac (FOL_SOLVE unused type_encs lam_trans ctxt clause ths) 1
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   262
    val seq = Meson.MESON (preskolem_tac ctxt) (maps (neg_clausify ctxt combs)) tac ctxt i st0
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   263
  in
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   264
    (!unused, seq)
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   265
  end
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   266
55521
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   267
fun metis_tac type_encs lam_trans ctxt ths i = snd o metis_tac_unused type_encs lam_trans ctxt ths i
241c6a2fdda1 added a version of the Metis tactic that returns the unused facts
blanchet
parents: 55520
diff changeset
   268
55520
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   269
(* Whenever "X" has schematic type variables, we treat "using X by metis" as "by (metis X)" to
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   270
   prevent "Subgoal.FOCUS" from freezing the type variables. We don't do it for nonschematic facts
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   271
   "X" because this breaks a few proofs (in the rare and subtle case where a proof relied on
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   272
   extensionality not being applied) and brings few benefits. *)
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   273
val has_tvar = 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
   274
55315
54b0352fb46d removed legacy 'metisFT' method
blanchet
parents: 55285
diff changeset
   275
fun metis_method ((override_type_encs, lam_trans), ths) ctxt facts =
55520
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   276
  let val (schem_facts, nonschem_facts) = List.partition has_tvar facts in
43099
blanchet
parents: 43094
diff changeset
   277
    HEADGOAL (Method.insert_tac nonschem_facts THEN'
55520
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   278
      CHANGED_PROP o metis_tac (these override_type_encs)
f6fc6d5339f1 tuned code
blanchet
parents: 55315
diff changeset
   279
        (the_default default_metis_lam_trans lam_trans) ctxt (schem_facts @ ths))
43099
blanchet
parents: 43094
diff changeset
   280
  end
43100
49347c6354b5 parse optional type system specification
blanchet
parents: 43099
diff changeset
   281
46365
547d1a1dcaf6 rename lambda translation schemes
blanchet
parents: 46320
diff changeset
   282
val metis_lam_transs = [hide_lamsN, liftingN, combsN]
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   283
45578
66f31d77b05f more robust options
blanchet
parents: 45570
diff changeset
   284
fun set_opt _ x NONE = SOME x
66f31d77b05f more robust options
blanchet
parents: 45570
diff changeset
   285
  | set_opt get x (SOME x0) =
55523
9429e7b5b827 removed final periods in messages for proof methods
blanchet
parents: 55521
diff changeset
   286
    error ("Cannot specify both " ^ quote (get x0) ^ " and " ^ quote (get x))
54756
blanchet
parents: 54742
diff changeset
   287
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   288
fun consider_opt s =
54756
blanchet
parents: 54742
diff changeset
   289
  if member (op =) metis_lam_transs s then apsnd (set_opt I s) else apfst (set_opt hd [s])
45514
973bb7846505 parse lambda translation option in Metis
blanchet
parents: 45513
diff changeset
   290
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   291
val parse_metis_options =
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   292
  Scan.optional
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   293
      (Args.parens (Parse.short_ident
46949
94aa7b81bcf6 prefer formally checked @{keyword} parser;
wenzelm
parents: 46904
diff changeset
   294
                    -- Scan.option (@{keyword ","} |-- Parse.short_ident))
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   295
       >> (fn (s, s') =>
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   296
              (NONE, NONE) |> consider_opt s
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   297
                           |> (case s' of SOME s' => consider_opt s' | _ => I)))
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   298
      (NONE, NONE)
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45514
diff changeset
   299
32956
c39860141415 tuned white space;
wenzelm
parents: 32955
diff changeset
   300
val setup =
55315
54b0352fb46d removed legacy 'metisFT' method
blanchet
parents: 55285
diff changeset
   301
  Method.setup @{binding metis}
54b0352fb46d removed legacy 'metisFT' method
blanchet
parents: 55285
diff changeset
   302
    (Scan.lift parse_metis_options -- Attrib.thms >> (METHOD oo metis_method))
54b0352fb46d removed legacy 'metisFT' method
blanchet
parents: 55285
diff changeset
   303
    "Metis for FOL and HOL problems"
23442
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   304
028e39e5e8f3 The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff changeset
   305
end;