src/HOL/Tools/Metis/metis_translate.ML
author blanchet
Mon, 06 Jun 2011 20:36:36 +0200
changeset 43211 77c432fe28ff
parent 43205 23b81469499f
child 43212 050a03afe024
permissions -rw-r--r--
enable new Metis
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_translate.ML
38027
505657ddb047 standardize "Author" tags
blanchet
parents: 38024
diff changeset
     2
    Author:     Jia Meng, Cambridge University Computer Laboratory and NICTA
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
     3
    Author:     Kong W. Susanto, Cambridge University Computer Laboratory
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
     4
    Author:     Lawrence C. Paulson, Cambridge University Computer Laboratory
36393
be73a2b2443b support readable names even when Isar proof reconstruction is enabled -- useful for debugging
blanchet
parents: 36378
diff changeset
     5
    Author:     Jasmin Blanchette, TU Muenchen
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     6
39494
bf7dd4902321 rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
blanchet
parents: 39355
diff changeset
     7
Translation of HOL to FOL for Metis.
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     8
*)
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     9
39494
bf7dd4902321 rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
blanchet
parents: 39355
diff changeset
    10
signature METIS_TRANSLATE =
24310
af4af9993922 proper signature;
wenzelm
parents: 24183
diff changeset
    11
sig
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
    12
  type type_literal = ATP_Translate.type_literal
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    13
43205
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
    14
  datatype mode = FO | HO | FT | Type_Sys of string
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
    15
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
    16
  datatype isa_thm =
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
    17
    Isa_Reflexive_or_Trivial |
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
    18
    Isa_Raw of thm
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
    19
40157
a2f01956220e renaming
blanchet
parents: 40145
diff changeset
    20
  type metis_problem =
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
    21
    {axioms : (Metis_Thm.thm * isa_thm) list,
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    22
     tfrees : type_literal list,
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    23
     old_skolems : (string * term) list}
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    24
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    25
  val metis_equal : string
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    26
  val metis_predicator : string
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    27
  val metis_app_op : string
43106
6ec2a3c7b69e fixed new path finder for type information tag
blanchet
parents: 43104
diff changeset
    28
  val metis_type_tag : string
42098
f978caf60bbe more robust handling of variables in new Skolemizer
blanchet
parents: 41491
diff changeset
    29
  val metis_generated_var_prefix : string
43104
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
    30
  val metis_name_table : ((string * int) * (string * bool)) list
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    31
  val reveal_old_skolem_terms : (string * term) list -> term -> term
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
    32
  val string_of_mode : mode -> string
40157
a2f01956220e renaming
blanchet
parents: 40145
diff changeset
    33
  val prepare_metis_problem :
43205
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
    34
    Proof.context -> mode -> thm list -> thm list
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    35
    -> mode * int Symtab.table * metis_problem
24310
af4af9993922 proper signature;
wenzelm
parents: 24183
diff changeset
    36
end
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    37
39494
bf7dd4902321 rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
blanchet
parents: 39355
diff changeset
    38
structure Metis_Translate : METIS_TRANSLATE =
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    39
struct
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    40
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
    41
open ATP_Problem
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
    42
open ATP_Translate
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    43
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    44
val metis_equal = "="
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    45
val metis_predicator = "{}"
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    46
val metis_app_op = "."
43104
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
    47
val metis_type_tag = ":"
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
    48
val metis_generated_var_prefix = "_"
17150
ce2a1aeb42aa DFG output now works for untyped rules (ML "ResClause.untyped();")
quigley
parents: 16976
diff changeset
    49
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    50
val metis_name_table =
43104
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
    51
  [((tptp_equal, 2), (metis_equal, false)),
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
    52
   ((tptp_old_equal, 2), (metis_equal, false)),
43174
f497a1e97d37 skip "hBOOL" in new Metis path finder
blanchet
parents: 43173
diff changeset
    53
   ((prefixed_predicator_name, 1), (metis_predicator, false)),
43130
d73fc2e55308 implemented missing hAPP and ti cases of new path finder
blanchet
parents: 43129
diff changeset
    54
   ((prefixed_app_op_name, 2), (metis_app_op, false)),
d73fc2e55308 implemented missing hAPP and ti cases of new path finder
blanchet
parents: 43129
diff changeset
    55
   ((prefixed_type_tag_name, 2), (metis_type_tag, true))]
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
    56
40145
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    57
fun predicate_of thy ((@{const Not} $ P), pos) = predicate_of thy (P, not pos)
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    58
  | predicate_of thy (t, pos) =
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    59
    (combterm_from_term thy [] (Envir.eta_contract t), pos)
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    60
40145
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    61
fun literals_of_term1 args thy (@{const Trueprop} $ P) =
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    62
    literals_of_term1 args thy P
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    63
  | literals_of_term1 args thy (@{const HOL.disj} $ P $ Q) =
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    64
    literals_of_term1 (literals_of_term1 args thy P) thy Q
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    65
  | literals_of_term1 (lits, ts) thy P =
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
    66
    let val ((pred, ts'), pol) = predicate_of thy (P, true) in
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
    67
      ((pol, pred) :: lits, union (op =) ts ts')
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    68
    end
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    69
val literals_of_term = literals_of_term1 ([], [])
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    70
39896
13b3a2ba9ea7 encode axiom number and cluster number in all zapped quantifiers to help discharging new skolemizer assumptions
blanchet
parents: 39890
diff changeset
    71
fun old_skolem_const_name i j num_T_args =
13b3a2ba9ea7 encode axiom number and cluster number in all zapped quantifiers to help discharging new skolemizer assumptions
blanchet
parents: 39890
diff changeset
    72
  old_skolem_const_prefix ^ Long_Name.separator ^
41491
a2ad5b824051 eliminated Int.toString;
wenzelm
parents: 41156
diff changeset
    73
  (space_implode Long_Name.separator (map string_of_int [i, j, num_T_args]))
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    74
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    75
fun conceal_old_skolem_terms i old_skolems t =
39953
aa54f347e5e2 hide uninteresting MESON/Metis constants and facts and remove "meson_" prefix to (now hidden) fact names
blanchet
parents: 39946
diff changeset
    76
  if exists_Const (curry (op =) @{const_name Meson.skolem} o fst) t then
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    77
    let
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    78
      fun aux old_skolems
39953
aa54f347e5e2 hide uninteresting MESON/Metis constants and facts and remove "meson_" prefix to (now hidden) fact names
blanchet
parents: 39946
diff changeset
    79
             (t as (Const (@{const_name Meson.skolem}, Type (_, [_, T])) $ _)) =
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    80
          let
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    81
            val (old_skolems, s) =
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    82
              if i = ~1 then
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    83
                (old_skolems, @{const_name undefined})
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    84
              else case AList.find (op aconv) old_skolems t of
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    85
                s :: _ => (old_skolems, s)
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    86
              | [] =>
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    87
                let
39896
13b3a2ba9ea7 encode axiom number and cluster number in all zapped quantifiers to help discharging new skolemizer assumptions
blanchet
parents: 39890
diff changeset
    88
                  val s = old_skolem_const_name i (length old_skolems)
13b3a2ba9ea7 encode axiom number and cluster number in all zapped quantifiers to help discharging new skolemizer assumptions
blanchet
parents: 39890
diff changeset
    89
                                                (length (Term.add_tvarsT T []))
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    90
                in ((s, t) :: old_skolems, s) end
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    91
          in (old_skolems, Const (s, T)) end
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    92
        | aux old_skolems (t1 $ t2) =
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
    93
          let
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    94
            val (old_skolems, t1) = aux old_skolems t1
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    95
            val (old_skolems, t2) = aux old_skolems t2
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    96
          in (old_skolems, t1 $ t2) end
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    97
        | aux old_skolems (Abs (s, T, t')) =
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    98
          let val (old_skolems, t') = aux old_skolems t' in
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
    99
            (old_skolems, Abs (s, T, t'))
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
   100
          end
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   101
        | aux old_skolems t = (old_skolems, t)
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   102
    in aux old_skolems t end
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
   103
  else
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   104
    (old_skolems, t)
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
   105
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   106
fun reveal_old_skolem_terms old_skolems =
37632
df12f798df99 move function
blanchet
parents: 37625
diff changeset
   107
  map_aterms (fn t as Const (s, _) =>
39896
13b3a2ba9ea7 encode axiom number and cluster number in all zapped quantifiers to help discharging new skolemizer assumptions
blanchet
parents: 39890
diff changeset
   108
                 if String.isPrefix old_skolem_const_prefix s then
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   109
                   AList.lookup (op =) old_skolems s |> the
37632
df12f798df99 move function
blanchet
parents: 37625
diff changeset
   110
                   |> map_types Type_Infer.paramify_vars
df12f798df99 move function
blanchet
parents: 37625
diff changeset
   111
                 else
df12f798df99 move function
blanchet
parents: 37625
diff changeset
   112
                   t
df12f798df99 move function
blanchet
parents: 37625
diff changeset
   113
               | t => t)
df12f798df99 move function
blanchet
parents: 37625
diff changeset
   114
37577
5379f41a1322 merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
blanchet
parents: 37575
diff changeset
   115
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   116
(* ------------------------------------------------------------------------- *)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   117
(* HOL to FOL  (Isabelle to Metis)                                           *)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   118
(* ------------------------------------------------------------------------- *)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   119
43205
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
   120
(* first-order, higher-order, fully-typed, ATP type system *)
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
   121
datatype mode = FO | HO | FT | Type_Sys of string
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   122
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   123
fun string_of_mode FO = "FO"
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   124
  | string_of_mode HO = "HO"
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   125
  | string_of_mode FT = "FT"
43205
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
   126
  | string_of_mode (Type_Sys type_sys) = "Type_Sys " ^ type_sys
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   127
42745
b817c6f91a98 reenabled equality proxy in Metis for higher-order reasoning
blanchet
parents: 42727
diff changeset
   128
fun fn_isa_to_met_sublevel "equal" = "c_fequal"
41139
cb1cbae54dbf add Metis support for higher-order propositional reasoning
blanchet
parents: 41138
diff changeset
   129
  | fn_isa_to_met_sublevel "c_False" = "c_fFalse"
cb1cbae54dbf add Metis support for higher-order propositional reasoning
blanchet
parents: 41138
diff changeset
   130
  | fn_isa_to_met_sublevel "c_True" = "c_fTrue"
cb1cbae54dbf add Metis support for higher-order propositional reasoning
blanchet
parents: 41138
diff changeset
   131
  | fn_isa_to_met_sublevel "c_Not" = "c_fNot"
cb1cbae54dbf add Metis support for higher-order propositional reasoning
blanchet
parents: 41138
diff changeset
   132
  | fn_isa_to_met_sublevel "c_conj" = "c_fconj"
cb1cbae54dbf add Metis support for higher-order propositional reasoning
blanchet
parents: 41138
diff changeset
   133
  | fn_isa_to_met_sublevel "c_disj" = "c_fdisj"
cb1cbae54dbf add Metis support for higher-order propositional reasoning
blanchet
parents: 41138
diff changeset
   134
  | fn_isa_to_met_sublevel "c_implies" = "c_fimplies"
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   135
  | fn_isa_to_met_sublevel x = x
42758
865ce93ce025 handle equality proxy in a more backward-compatible way
blanchet
parents: 42745
diff changeset
   136
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   137
fun fn_isa_to_met_toplevel "equal" = metis_equal
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   138
  | fn_isa_to_met_toplevel x = x
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   139
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   140
fun metis_lit b c args = (b, (c, args));
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   141
42562
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   142
fun metis_term_from_typ (Type (s, Ts)) =
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   143
    Metis_Term.Fn (make_fixed_type_const s, map metis_term_from_typ Ts)
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   144
  | metis_term_from_typ (TFree (s, _)) =
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   145
    Metis_Term.Fn (make_fixed_type_var s, [])
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   146
  | metis_term_from_typ (TVar (x, _)) =
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   147
    Metis_Term.Var (make_schematic_type_var x)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   148
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   149
(*These two functions insert type literals before the real literals. That is the
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   150
  opposite order from TPTP linkup, but maybe OK.*)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   151
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   152
fun hol_term_to_fol_FO tm =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   153
  case strip_combterm_comb tm of
42562
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   154
      (CombConst ((c, _), _, Ts), tms) =>
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   155
        let val tyargs = map metis_term_from_typ Ts
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   156
            val args = map hol_term_to_fol_FO tms
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   157
        in Metis_Term.Fn (c, tyargs @ args) end
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   158
    | (CombVar ((v, _), _), []) => Metis_Term.Var v
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   159
    | _ => raise Fail "non-first-order combterm"
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   160
42562
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   161
fun hol_term_to_fol_HO (CombConst ((a, _), _, Ts)) =
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   162
    Metis_Term.Fn (fn_isa_to_met_sublevel a, map metis_term_from_typ Ts)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   163
  | hol_term_to_fol_HO (CombVar ((s, _), _)) = Metis_Term.Var s
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   164
  | hol_term_to_fol_HO (CombApp (tm1, tm2)) =
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   165
    Metis_Term.Fn (metis_app_op, map hol_term_to_fol_HO [tm1, tm2])
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   166
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   167
(*The fully-typed translation, to avoid type errors*)
42562
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   168
fun tag_with_type tm T =
43104
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   169
  Metis_Term.Fn (metis_type_tag, [tm, metis_term_from_typ T])
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   170
41138
eb80538166b6 implemented partially-typed "tags" type encoding
blanchet
parents: 40259
diff changeset
   171
fun hol_term_to_fol_FT (CombVar ((s, _), ty)) =
eb80538166b6 implemented partially-typed "tags" type encoding
blanchet
parents: 40259
diff changeset
   172
    tag_with_type (Metis_Term.Var s) ty
eb80538166b6 implemented partially-typed "tags" type encoding
blanchet
parents: 40259
diff changeset
   173
  | hol_term_to_fol_FT (CombConst ((a, _), ty, _)) =
eb80538166b6 implemented partially-typed "tags" type encoding
blanchet
parents: 40259
diff changeset
   174
    tag_with_type (Metis_Term.Fn (fn_isa_to_met_sublevel a, [])) ty
eb80538166b6 implemented partially-typed "tags" type encoding
blanchet
parents: 40259
diff changeset
   175
  | hol_term_to_fol_FT (tm as CombApp (tm1,tm2)) =
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   176
    tag_with_type
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   177
        (Metis_Term.Fn (metis_app_op, map hol_term_to_fol_FT [tm1, tm2]))
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   178
        (combtyp_of tm)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   179
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
   180
fun hol_literal_to_fol FO (pos, tm) =
42562
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   181
      let
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   182
        val (CombConst((p, _), _, Ts), tms) = strip_combterm_comb tm
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   183
        val tylits = if p = "equal" then [] else map metis_term_from_typ Ts
f1d903f789b1 killed needless datatype "combtyp" in Metis
blanchet
parents: 42561
diff changeset
   184
        val lits = map hol_term_to_fol_FO tms
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   185
      in metis_lit pos (fn_isa_to_met_toplevel p) (tylits @ lits) end
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
   186
  | hol_literal_to_fol HO (pos, tm) =
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   187
     (case strip_combterm_comb tm of
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   188
          (CombConst(("equal", _), _, _), tms) =>
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   189
            metis_lit pos metis_equal (map hol_term_to_fol_HO tms)
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   190
        | _ => metis_lit pos metis_predicator [hol_term_to_fol_HO tm])
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
   191
  | hol_literal_to_fol FT (pos, tm) =
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   192
     (case strip_combterm_comb tm of
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   193
          (CombConst(("equal", _), _, _), tms) =>
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   194
            metis_lit pos metis_equal (map hol_term_to_fol_FT tms)
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   195
        | _ => metis_lit pos metis_predicator [hol_term_to_fol_FT tm])
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   196
40145
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
   197
fun literals_of_hol_term thy mode t =
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
   198
  let val (lits, types_sorts) = literals_of_term thy t in
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
   199
    (map (hol_literal_to_fol mode) lits, types_sorts)
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
   200
  end
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   201
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   202
(*Sign should be "true" for conjecture type constraints, "false" for type lits in clauses.*)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   203
fun metis_of_type_literals pos (TyLitVar ((s, _), (s', _))) =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   204
    metis_lit pos s [Metis_Term.Var s']
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   205
  | metis_of_type_literals pos (TyLitFree ((s, _), (s', _))) =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   206
    metis_lit pos s [Metis_Term.Fn (s',[])]
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   207
42352
blanchet
parents: 42107
diff changeset
   208
fun has_default_sort _ (TVar _) = false
blanchet
parents: 42107
diff changeset
   209
  | has_default_sort ctxt (TFree (x, s)) =
blanchet
parents: 42107
diff changeset
   210
    (s = the_default [] (Variable.def_sort ctxt (x, ~1)));
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   211
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   212
fun metis_of_tfree tf =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   213
  Metis_Thm.axiom (Metis_LiteralSet.singleton (metis_of_type_literals true tf));
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   214
43090
f6331d785128 removed obscure option
blanchet
parents: 43087
diff changeset
   215
fun hol_thm_to_fol is_conjecture ctxt mode j old_skolems th =
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   216
  let
42361
23f352990944 modernized structure Proof_Context;
wenzelm
parents: 42352
diff changeset
   217
    val thy = Proof_Context.theory_of ctxt
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   218
    val (old_skolems, (mlits, types_sorts)) =
39888
40ef95149770 ignore Skolem assumption (if any)
blanchet
parents: 39887
diff changeset
   219
     th |> prop_of |> Logic.strip_imp_concl
40ef95149770 ignore Skolem assumption (if any)
blanchet
parents: 39887
diff changeset
   220
        |> conceal_old_skolem_terms j old_skolems
40145
04a05b2a7a36 no need to encode theorem number twice in skolem names
blanchet
parents: 39962
diff changeset
   221
        ||> (HOLogic.dest_Trueprop #> literals_of_hol_term thy mode)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   222
  in
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   223
    if is_conjecture then
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   224
      (Metis_Thm.axiom (Metis_LiteralSet.fromList mlits),
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
   225
       raw_type_literals_for_types types_sorts, old_skolems)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   226
    else
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   227
      let
42352
blanchet
parents: 42107
diff changeset
   228
        val tylits = types_sorts |> filter_out (has_default_sort ctxt)
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
   229
                                 |> raw_type_literals_for_types
43090
f6331d785128 removed obscure option
blanchet
parents: 43087
diff changeset
   230
        val mtylits = map (metis_of_type_literals false) tylits
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   231
      in
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   232
        (Metis_Thm.axiom (Metis_LiteralSet.fromList(mtylits @ mlits)), [],
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   233
         old_skolems)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   234
      end
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   235
  end;
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   236
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   237
(* ------------------------------------------------------------------------- *)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   238
(* Logic maps manage the interface between HOL and first-order logic.        *)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   239
(* ------------------------------------------------------------------------- *)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   240
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   241
datatype isa_thm =
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   242
  Isa_Reflexive_or_Trivial |
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   243
  Isa_Raw of thm
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   244
40157
a2f01956220e renaming
blanchet
parents: 40145
diff changeset
   245
type metis_problem =
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   246
  {axioms : (Metis_Thm.thm * isa_thm) list,
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   247
   tfrees : type_literal list,
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   248
   old_skolems : (string * term) list}
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   249
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   250
fun is_quasi_fol_clause thy =
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   251
  Meson.is_fol_term thy o snd o conceal_old_skolem_terms ~1 [] o prop_of
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   252
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   253
(*Extract TFree constraints from context to include as conjecture clauses*)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   254
fun init_tfrees ctxt =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   255
  let fun add ((a,i),s) Ts = if i = ~1 then TFree(a,s) :: Ts else Ts in
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   256
    Vartab.fold add (#2 (Variable.constraints_of ctxt)) []
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
   257
    |> raw_type_literals_for_types
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   258
  end;
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   259
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   260
fun const_in_metis c (pred, tm_list) =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   261
  let
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   262
    fun in_mterm (Metis_Term.Var _) = false
41156
blanchet
parents: 41140
diff changeset
   263
      | in_mterm (Metis_Term.Fn (nm, tm_list)) =
blanchet
parents: 41140
diff changeset
   264
        c = nm orelse exists in_mterm tm_list
blanchet
parents: 41140
diff changeset
   265
  in c = pred orelse exists in_mterm tm_list end
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   266
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   267
(* ARITY CLAUSE *)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   268
fun m_arity_cls (TConsLit ((c, _), (t, _), args)) =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   269
    metis_lit true c [Metis_Term.Fn(t, map (Metis_Term.Var o fst) args)]
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   270
  | m_arity_cls (TVarLit ((c, _), (s, _))) =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   271
    metis_lit false c [Metis_Term.Var s]
43125
ddf63baabdec distinguish different kinds of typing informations in the fact name
blanchet
parents: 43109
diff changeset
   272
(* TrueI is returned as the Isabelle counterpart because there isn't any. *)
43086
blanchet
parents: 43085
diff changeset
   273
fun arity_cls ({prem_lits, concl_lits, ...} : arity_clause) =
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   274
  (TrueI,
42895
c8d9bce88f89 name tuning
blanchet
parents: 42894
diff changeset
   275
   Metis_Thm.axiom (Metis_LiteralSet.fromList
c8d9bce88f89 name tuning
blanchet
parents: 42894
diff changeset
   276
                        (map m_arity_cls (concl_lits :: prem_lits))));
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   277
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   278
(* CLASSREL CLAUSE *)
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   279
fun m_class_rel_cls (subclass, _) (superclass, _) =
43091
blanchet
parents: 43090
diff changeset
   280
  [metis_lit false subclass [Metis_Term.Var "T"],
blanchet
parents: 43090
diff changeset
   281
   metis_lit true superclass [Metis_Term.Var "T"]]
43086
blanchet
parents: 43085
diff changeset
   282
fun class_rel_cls ({subclass, superclass, ...} : class_rel_clause) =
43091
blanchet
parents: 43090
diff changeset
   283
  (TrueI, m_class_rel_cls subclass superclass
blanchet
parents: 43090
diff changeset
   284
          |> Metis_LiteralSet.fromList |> Metis_Thm.axiom)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   285
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   286
fun type_ext thy tms =
43091
blanchet
parents: 43090
diff changeset
   287
  let
blanchet
parents: 43090
diff changeset
   288
    val subs = tfree_classes_of_terms tms
blanchet
parents: 43090
diff changeset
   289
    val supers = tvar_classes_of_terms tms
43189
blanchet
parents: 43180
diff changeset
   290
    val tycons = type_constrs_of_terms thy tms
43091
blanchet
parents: 43090
diff changeset
   291
    val (supers', arity_clauses) = make_arity_clauses thy tycons supers
blanchet
parents: 43090
diff changeset
   292
    val class_rel_clauses = make_class_rel_clauses thy subs supers'
blanchet
parents: 43090
diff changeset
   293
  in map class_rel_cls class_rel_clauses @ map arity_cls arity_clauses end
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   294
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   295
val proxy_defs = map (fst o snd o snd) proxy_table
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   296
val prepare_helper =
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   297
  Meson.make_meta_clause #> rewrite_rule (map safe_mk_meta_eq proxy_defs)
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   298
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   299
fun metis_name_from_atp s ary =
43104
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   300
  AList.lookup (op =) metis_name_table (s, ary) |> the_default (s, false)
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   301
fun metis_term_from_atp (ATerm (s, tms)) =
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   302
  if is_tptp_variable s then
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   303
    Metis_Term.Var s
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   304
  else
43104
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   305
    let val (s, swap) = metis_name_from_atp s (length tms) in
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   306
      Metis_Term.Fn (s, tms |> map metis_term_from_atp |> swap ? rev)
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   307
    end
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   308
fun metis_atom_from_atp (AAtom tm) =
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   309
    (case metis_term_from_atp tm of
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   310
       Metis_Term.Fn x => x
81d1b15aa0ae use ":" for type information (looks good in Metis's output) and handle it in new path finder
blanchet
parents: 43103
diff changeset
   311
     | _ => raise Fail "non CNF -- expected function")
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   312
  | metis_atom_from_atp _ = raise Fail "not CNF -- expected atom"
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   313
fun metis_literal_from_atp (AConn (ANot, [phi])) =
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   314
    (false, metis_atom_from_atp phi)
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   315
  | metis_literal_from_atp phi = (true, metis_atom_from_atp phi)
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   316
fun metis_literals_from_atp (AConn (AOr, [phi1, phi2])) =
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   317
    uncurry (union (op =)) (pairself metis_literals_from_atp (phi1, phi2))
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   318
  | metis_literals_from_atp phi = [metis_literal_from_atp phi]
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   319
fun metis_axiom_from_atp clauses (Formula (ident, _, phi, _, _)) =
43173
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   320
    let
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   321
      fun some isa =
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   322
        SOME (phi |> metis_literals_from_atp |> Metis_LiteralSet.fromList
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   323
                  |> Metis_Thm.axiom, isa)
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   324
    in
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   325
      if ident = type_tag_idempotence_helper_name orelse
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   326
         String.isPrefix lightweight_tags_sym_formula_prefix ident then
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   327
        Isa_Reflexive_or_Trivial |> some
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   328
      else if String.isPrefix helper_prefix ident then
43194
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   329
        case (String.isSuffix typed_helper_suffix ident,
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   330
              space_explode "_" ident) of
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   331
          (needs_fairly_sound, _ :: const :: j :: _) =>
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   332
          nth ((const, needs_fairly_sound)
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   333
               |> AList.lookup (op =) helper_table |> the)
43173
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   334
              (the (Int.fromString j) - 1)
43194
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   335
          |> prepare_helper
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   336
          |> Isa_Raw |> some
43173
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   337
        | _ => raise Fail ("malformed helper identifier " ^ quote ident)
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   338
      else case try (unprefix conjecture_prefix) ident of
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   339
        SOME s =>
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   340
        let val j = the (Int.fromString s) in
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   341
          if j = length clauses then NONE
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   342
          else Meson.make_meta_clause (nth clauses j) |> Isa_Raw |> some
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   343
        end
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   344
      | NONE => TrueI |> Isa_Raw |> some
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   345
    end
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   346
  | metis_axiom_from_atp _ _ = raise Fail "not CNF -- expected formula"
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   347
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   348
(* Function to generate metis clauses, including comb and type clauses *)
43205
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
   349
fun prepare_metis_problem ctxt (mode as Type_Sys type_sys) conj_clauses
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
   350
                          fact_clauses =
43091
blanchet
parents: 43090
diff changeset
   351
    let
43205
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
   352
      val type_sys = type_sys_from_string type_sys
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   353
      val explicit_apply = NONE
43109
8c9046951dcb monomorphize in the new Metis if the type system calls for it
blanchet
parents: 43106
diff changeset
   354
      val clauses =
8c9046951dcb monomorphize in the new Metis if the type system calls for it
blanchet
parents: 43106
diff changeset
   355
        conj_clauses @ fact_clauses
8c9046951dcb monomorphize in the new Metis if the type system calls for it
blanchet
parents: 43106
diff changeset
   356
        |> (if polymorphism_of_type_sys type_sys = Polymorphic then
8c9046951dcb monomorphize in the new Metis if the type system calls for it
blanchet
parents: 43106
diff changeset
   357
              I
8c9046951dcb monomorphize in the new Metis if the type system calls for it
blanchet
parents: 43106
diff changeset
   358
            else
8c9046951dcb monomorphize in the new Metis if the type system calls for it
blanchet
parents: 43106
diff changeset
   359
              map (pair 0)
8c9046951dcb monomorphize in the new Metis if the type system calls for it
blanchet
parents: 43106
diff changeset
   360
              #> rpair ctxt
8c9046951dcb monomorphize in the new Metis if the type system calls for it
blanchet
parents: 43106
diff changeset
   361
              #-> Monomorph.monomorph Monomorph.all_schematic_consts_of
43132
44cd26bfc30c ensured monomorphized facts have normalized zero var indexes, so that "find_var" doesn't fail later on
blanchet
parents: 43130
diff changeset
   362
              #> fst #> maps (map (zero_var_indexes o snd)))
43180
283114859d6c conceal old Skolems in new Metis
blanchet
parents: 43175
diff changeset
   363
      val (old_skolems, props) =
283114859d6c conceal old Skolems in new Metis
blanchet
parents: 43175
diff changeset
   364
        fold_rev (fn clause => fn (old_skolems, props) =>
43190
494fde207706 don't translate new Skolemizer assumptions in new Metis
blanchet
parents: 43189
diff changeset
   365
                     clause |> prop_of |> Logic.strip_imp_concl
494fde207706 don't translate new Skolemizer assumptions in new Metis
blanchet
parents: 43189
diff changeset
   366
                            |> conceal_old_skolem_terms (length clauses)
494fde207706 don't translate new Skolemizer assumptions in new Metis
blanchet
parents: 43189
diff changeset
   367
                                                        old_skolems
494fde207706 don't translate new Skolemizer assumptions in new Metis
blanchet
parents: 43189
diff changeset
   368
                            ||> (fn prop => prop :: props))
43180
283114859d6c conceal old Skolems in new Metis
blanchet
parents: 43175
diff changeset
   369
             clauses ([], [])
43193
e11bd628f1a5 improved ATP clausifier so it can deal with "x => (y <=> z)"
blanchet
parents: 43190
diff changeset
   370
(*
e11bd628f1a5 improved ATP clausifier so it can deal with "x => (y <=> z)"
blanchet
parents: 43190
diff changeset
   371
val _ = tracing ("PROPS:\n" ^ cat_lines (map (Syntax.string_of_term ctxt) props))
e11bd628f1a5 improved ATP clausifier so it can deal with "x => (y <=> z)"
blanchet
parents: 43190
diff changeset
   372
*)
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   373
      val (atp_problem, _, _, _, _, _, sym_tab) =
43098
e88e974c4846 proper handling of type variable classes in new Metis
blanchet
parents: 43096
diff changeset
   374
        prepare_atp_problem ctxt CNF Hypothesis Axiom type_sys explicit_apply
43180
283114859d6c conceal old Skolems in new Metis
blanchet
parents: 43175
diff changeset
   375
                            false false props @{prop False} []
43193
e11bd628f1a5 improved ATP clausifier so it can deal with "x => (y <=> z)"
blanchet
parents: 43190
diff changeset
   376
(*
e11bd628f1a5 improved ATP clausifier so it can deal with "x => (y <=> z)"
blanchet
parents: 43190
diff changeset
   377
val _ = tracing ("ATP PROBLEM: " ^ cat_lines (tptp_strings_for_atp_problem CNF atp_problem))
e11bd628f1a5 improved ATP clausifier so it can deal with "x => (y <=> z)"
blanchet
parents: 43190
diff changeset
   378
*)
43211
77c432fe28ff enable new Metis
blanchet
parents: 43205
diff changeset
   379
      (* "rev" is for compatibility *)
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   380
      val axioms =
43173
b98daa96d043 don't pass "~ " to new Metis
blanchet
parents: 43160
diff changeset
   381
        atp_problem |> maps (map_filter (metis_axiom_from_atp clauses) o snd)
43211
77c432fe28ff enable new Metis
blanchet
parents: 43205
diff changeset
   382
                    |> rev
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   383
    in
43205
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
   384
      (mode, sym_tab, {axioms = axioms, tfrees = [], old_skolems = old_skolems})
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   385
    end
43205
23b81469499f more preparations towards hijacking Metis
blanchet
parents: 43199
diff changeset
   386
  | prepare_metis_problem ctxt mode conj_clauses fact_clauses =
43087
b870759ce0f3 added new metis mode, with no implementation yet
blanchet
parents: 43086
diff changeset
   387
    let
b870759ce0f3 added new metis mode, with no implementation yet
blanchet
parents: 43086
diff changeset
   388
      val thy = Proof_Context.theory_of ctxt
b870759ce0f3 added new metis mode, with no implementation yet
blanchet
parents: 43086
diff changeset
   389
      (* The modes FO and FT are sticky. HO can be downgraded to FO. *)
b870759ce0f3 added new metis mode, with no implementation yet
blanchet
parents: 43086
diff changeset
   390
      val mode =
b870759ce0f3 added new metis mode, with no implementation yet
blanchet
parents: 43086
diff changeset
   391
        if mode = HO andalso
43091
blanchet
parents: 43090
diff changeset
   392
           forall (forall (is_quasi_fol_clause thy))
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   393
                  [conj_clauses, fact_clauses] then
43087
b870759ce0f3 added new metis mode, with no implementation yet
blanchet
parents: 43086
diff changeset
   394
          FO
b870759ce0f3 added new metis mode, with no implementation yet
blanchet
parents: 43086
diff changeset
   395
        else
b870759ce0f3 added new metis mode, with no implementation yet
blanchet
parents: 43086
diff changeset
   396
          mode
41139
cb1cbae54dbf add Metis support for higher-order propositional reasoning
blanchet
parents: 41138
diff changeset
   397
      fun add_thm is_conjecture (isa_ith, metis_ith)
40157
a2f01956220e renaming
blanchet
parents: 40145
diff changeset
   398
                  {axioms, tfrees, old_skolems} : metis_problem =
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   399
        let
39886
8a9f0c97d550 first step towards a new skolemizer that doesn't require "Eps"
blanchet
parents: 39720
diff changeset
   400
          val (mth, tfree_lits, old_skolems) =
43090
f6331d785128 removed obscure option
blanchet
parents: 43087
diff changeset
   401
            hol_thm_to_fol is_conjecture ctxt mode (length axioms) old_skolems
f6331d785128 removed obscure option
blanchet
parents: 43087
diff changeset
   402
                           metis_ith
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   403
        in
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   404
          {axioms = (mth, Isa_Raw isa_ith) :: axioms,
43091
blanchet
parents: 43090
diff changeset
   405
           tfrees = union (op =) tfree_lits tfrees, old_skolems = old_skolems}
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   406
        end;
43091
blanchet
parents: 43090
diff changeset
   407
      fun add_type_thm (ith, mth) {axioms, tfrees, old_skolems} =
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   408
        {axioms = (mth, Isa_Raw ith) :: axioms, tfrees = tfrees,
43091
blanchet
parents: 43090
diff changeset
   409
         old_skolems = old_skolems}
blanchet
parents: 43090
diff changeset
   410
      fun add_tfrees {axioms, tfrees, old_skolems} =
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   411
        {axioms = map (rpair (Isa_Raw TrueI) o metis_of_tfree)
43129
4301f1c123d6 support lightweight tags in new Metis
blanchet
parents: 43128
diff changeset
   412
                      (distinct (op =) tfrees) @ axioms,
43091
blanchet
parents: 43090
diff changeset
   413
         tfrees = tfrees, old_skolems = old_skolems}
blanchet
parents: 43090
diff changeset
   414
      val problem =
blanchet
parents: 43090
diff changeset
   415
        {axioms = [], tfrees = init_tfrees ctxt, old_skolems = []}
blanchet
parents: 43090
diff changeset
   416
        |> fold (add_thm true o `Meson.make_meta_clause) conj_clauses
blanchet
parents: 43090
diff changeset
   417
        |> add_tfrees
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   418
        |> fold (add_thm false o `Meson.make_meta_clause) fact_clauses
43091
blanchet
parents: 43090
diff changeset
   419
      val clause_lists = map (Metis_Thm.clause o #1) (#axioms problem)
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   420
      fun is_used c =
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   421
        exists (Metis_LiteralSet.exists (const_in_metis c o #2)) clause_lists
43091
blanchet
parents: 43090
diff changeset
   422
      val problem =
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   423
        if mode = FO then
43091
blanchet
parents: 43090
diff changeset
   424
          problem
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   425
        else
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   426
          let
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   427
            val helper_ths =
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43003
diff changeset
   428
              helper_table
43194
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   429
              |> filter (is_used o prefix const_prefix o fst o fst)
ef3ff8856245 fixed type helper indices in new Metis
blanchet
parents: 43193
diff changeset
   430
              |> maps (fn ((_, needs_full_types), thms) =>
41140
9c68004b8c9d added Sledgehammer support for higher-order propositional reasoning
blanchet
parents: 41139
diff changeset
   431
                          if needs_full_types andalso mode <> FT then []
43159
29b55f292e0b added support for helpers in new Metis, so far only for polymorphic type encodings
blanchet
parents: 43132
diff changeset
   432
                          else map (`prepare_helper) thms)
43091
blanchet
parents: 43090
diff changeset
   433
          in problem |> fold (add_thm false) helper_ths end
43092
93ec303e1917 more work on new metis that exploits the powerful new type encodings
blanchet
parents: 43091
diff changeset
   434
      val type_ths = type_ext thy (map prop_of (conj_clauses @ fact_clauses))
43094
269300fb83d0 more work on new Metis
blanchet
parents: 43093
diff changeset
   435
    in (mode, Symtab.empty, fold add_type_thm type_ths problem) end
39497
fa16349939b7 complete refactoring of Metis along the lines of Sledgehammer
blanchet
parents: 39494
diff changeset
   436
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   437
end;