src/HOL/Tools/ATP/atp_proof_reconstruct.ML
author blanchet
Fri, 25 Oct 2024 15:31:58 +0200
changeset 81254 d3c0734059ee
parent 79734 0fa4bebbdd75
child 81519 cdc43c0fdbfc
permissions -rw-r--r--
variable instantiation in Sledgehammer and Metis
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
46320
0b8b73b49848 renamed two files to make room for a new file
blanchet
parents: 45887
diff changeset
     1
(*  Title:      HOL/Tools/ATP/atp_proof_reconstruct.ML
38027
505657ddb047 standardize "Author" tags
blanchet
parents: 38019
diff changeset
     2
    Author:     Lawrence C. Paulson, Cambridge University Computer Laboratory
505657ddb047 standardize "Author" tags
blanchet
parents: 38019
diff changeset
     3
    Author:     Claire Quigley, Cambridge University Computer Laboratory
36392
c00c57850eb7 cosmetics: rename internal functions
blanchet
parents: 36369
diff changeset
     4
    Author:     Jasmin Blanchette, TU Muenchen
21978
72c21698a055 Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
paulson
parents:
diff changeset
     5
49914
23e36a4d28f1 refactor code
blanchet
parents: 49881
diff changeset
     6
Basic proof reconstruction from ATP proofs.
33310
44f9665c2091 proper header;
wenzelm
parents: 33243
diff changeset
     7
*)
44f9665c2091 proper header;
wenzelm
parents: 33243
diff changeset
     8
46320
0b8b73b49848 renamed two files to make room for a new file
blanchet
parents: 45887
diff changeset
     9
signature ATP_PROOF_RECONSTRUCT =
24425
ca97c6f3d9cd Returning both a "one-line" proof and a structured proof
paulson
parents: 24387
diff changeset
    10
sig
54811
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
    11
  type 'a atp_type = 'a ATP_Problem.atp_type
53586
bd5fa6425993 prefixed types and some functions with "atp_" for disambiguation
blanchet
parents: 52758
diff changeset
    12
  type ('a, 'b) atp_term = ('a, 'b) ATP_Problem.atp_term
bd5fa6425993 prefixed types and some functions with "atp_" for disambiguation
blanchet
parents: 52758
diff changeset
    13
  type ('a, 'b, 'c, 'd) atp_formula = ('a, 'b, 'c, 'd) ATP_Problem.atp_formula
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
    14
  type stature = ATP_Problem_Generate.stature
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
    15
  type atp_step_name = ATP_Proof.atp_step_name
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
    16
  type ('a, 'b) atp_step = ('a, 'b) ATP_Proof.atp_step
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
    17
  type 'a atp_proof = 'a ATP_Proof.atp_proof
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    18
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    19
  val metisN : string
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    20
  val full_typesN : string
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    21
  val partial_typesN : string
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    22
  val no_typesN : string
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    23
  val really_full_type_enc : string
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    24
  val full_type_enc : string
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    25
  val partial_type_enc : string
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    26
  val no_type_enc : string
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    27
  val full_type_encs : string list
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    28
  val partial_type_encs : string list
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
    29
  val default_metis_lam_trans : string
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
    30
58653
4b44c227c0e0 improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
blanchet
parents: 58652
diff changeset
    31
  val leo2_extcnf_equal_neg_rule : string
4b44c227c0e0 improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
blanchet
parents: 58652
diff changeset
    32
  val satallax_tab_rule_prefix : string
79734
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
    33
  val zipperposition_cnf_rule : string
58653
4b44c227c0e0 improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
blanchet
parents: 58652
diff changeset
    34
49983
33e18e9916a8 use metaquantification when possible in Isar proofs
blanchet
parents: 49914
diff changeset
    35
  val forall_of : term -> term -> term
33e18e9916a8 use metaquantification when possible in Isar proofs
blanchet
parents: 49914
diff changeset
    36
  val exists_of : term -> term -> term
57767
5bc204ca27ce centralized boolean simplification so that e.g. LEO-II benefits from it
blanchet
parents: 57765
diff changeset
    37
  val simplify_bool : term -> term
57792
9cb24c835284 rationalize Skolem names
blanchet
parents: 57790
diff changeset
    38
  val var_name_of_typ : typ -> string
57765
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
    39
  val rename_bound_vars : term -> term
55285
e88ad20035f4 merged 'reconstructors' and 'proof methods'
blanchet
parents: 55257
diff changeset
    40
  val type_enc_aliases : (string * string list) list
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    41
  val unalias_type_enc : string -> string list
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
    42
  val term_of_atp : Proof.context -> ATP_Problem.atp_format -> ATP_Problem_Generate.type_enc ->
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
    43
    bool -> int Symtab.table -> typ option -> (string, string atp_type) atp_term -> term
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
    44
  val prop_of_atp : Proof.context -> ATP_Problem.atp_format -> ATP_Problem_Generate.type_enc ->
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
    45
    bool -> int Symtab.table ->
54811
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
    46
    (string, string, (string, string atp_type) atp_term, string) atp_formula -> term
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
    47
77432
e51aa922079a tweaked Sledgehammer interaction
blanchet
parents: 77430
diff changeset
    48
  val is_conjecture_used_in_proof : string atp_proof -> bool
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
    49
  val used_facts_in_atp_proof : Proof.context -> (string * stature) list -> string atp_proof ->
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
    50
    (string * stature) list
55257
abfd7b90bba2 rationalized threading of 'metis' arguments
blanchet
parents: 55195
diff changeset
    51
  val atp_proof_prefers_lifting : string atp_proof -> bool
81254
d3c0734059ee variable instantiation in Sledgehammer and Metis
blanchet
parents: 79734
diff changeset
    52
  val is_lam_def_used_in_atp_proof : string atp_proof -> bool
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
    53
  val is_typed_helper_used_in_atp_proof : string atp_proof -> bool
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
    54
  val replace_dependencies_in_line : atp_step_name * atp_step_name list -> ('a, 'b) atp_step ->
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
    55
    ('a, 'b) atp_step
81254
d3c0734059ee variable instantiation in Sledgehammer and Metis
blanchet
parents: 79734
diff changeset
    56
  val uncombine_term : theory -> term -> term
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
    57
  val termify_atp_proof : Proof.context -> string -> ATP_Problem.atp_format ->
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
    58
    ATP_Problem_Generate.type_enc -> string Symtab.table -> (string * term) list ->
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
    59
    int Symtab.table -> string atp_proof -> (term, string) atp_step list
57267
8b87114357bd integrated new Waldmeister code with 'sledgehammer' command
blanchet
parents: 57263
diff changeset
    60
  val repair_waldmeister_endgame : (term, 'a) atp_step list -> (term, 'a) atp_step list
57699
a6cf197c1f1e also try 'metis' with 'full_types'
blanchet
parents: 57697
diff changeset
    61
  val infer_formulas_types : Proof.context -> term list -> term list
72401
2783779b7dd3 removed obsolete unmaintained experimental prover Pirate
blanchet
parents: 70940
diff changeset
    62
  val introduce_spass_skolems : (term, string) atp_step list -> (term, string) atp_step list
79734
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
    63
  val regroup_zipperposition_skolems : (term, string) atp_step list -> (term, string) atp_step list
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
    64
  val factify_atp_proof : (string * 'a) list -> term list -> term -> (term, string) atp_step list ->
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
    65
    (term, string) atp_step list
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
    66
  val termify_atp_abduce_candidate : Proof.context -> string -> ATP_Problem.atp_format ->
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
    67
    ATP_Problem_Generate.type_enc -> string Symtab.table -> (string * term) list ->
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
    68
    int Symtab.table -> (string, string, (string, string atp_type) atp_term, string) atp_formula ->
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
    69
    term
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
    70
  val top_abduce_candidates : int -> term list -> term list
77602
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
    71
  val sort_propositions_by_provability : Proof.context -> term list -> term list
24425
ca97c6f3d9cd Returning both a "one-line" proof and a structured proof
paulson
parents: 24387
diff changeset
    72
end;
21978
72c21698a055 Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
paulson
parents:
diff changeset
    73
46320
0b8b73b49848 renamed two files to make room for a new file
blanchet
parents: 45887
diff changeset
    74
structure ATP_Proof_Reconstruct : ATP_PROOF_RECONSTRUCT =
21978
72c21698a055 Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
paulson
parents:
diff changeset
    75
struct
72c21698a055 Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
paulson
parents:
diff changeset
    76
43085
0a2f5b86bdd7 first step in sharing more code between ATP and Metis translation
blanchet
parents: 43062
diff changeset
    77
open ATP_Util
38028
22dcaec5fa77 minor refactoring
blanchet
parents: 38027
diff changeset
    78
open ATP_Problem
39452
70a57e40f795 factored out TSTP/SPASS/Vampire proof parsing;
blanchet
parents: 39425
diff changeset
    79
open ATP_Proof
46320
0b8b73b49848 renamed two files to make room for a new file
blanchet
parents: 45887
diff changeset
    80
open ATP_Problem_Generate
21978
72c21698a055 Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
paulson
parents:
diff changeset
    81
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    82
val metisN = "metis"
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    83
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    84
val full_typesN = "full_types"
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    85
val partial_typesN = "partial_types"
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    86
val no_typesN = "no_types"
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    87
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    88
val really_full_type_enc = "mono_tags"
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    89
val full_type_enc = "poly_guards_query"
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    90
val partial_type_enc = "poly_args"
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    91
val no_type_enc = "erased"
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    92
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    93
val full_type_encs = [full_type_enc, really_full_type_enc]
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    94
val partial_type_encs = partial_type_enc :: full_type_encs
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    95
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    96
val type_enc_aliases =
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    97
  [(full_typesN, full_type_encs),
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    98
   (partial_typesN, partial_type_encs),
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
    99
   (no_typesN, [no_type_enc])]
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
   100
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
   101
fun unalias_type_enc s =
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
   102
  AList.lookup (op =) type_enc_aliases s |> the_default [s]
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
   103
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   104
val default_metis_lam_trans = combsN
45519
cd6e78cb6ee8 make metis reconstruction handling more flexible
blanchet
parents: 45511
diff changeset
   105
58653
4b44c227c0e0 improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
blanchet
parents: 58652
diff changeset
   106
val leo2_extcnf_equal_neg_rule = "extcnf_equal_neg"
4b44c227c0e0 improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
blanchet
parents: 58652
diff changeset
   107
val satallax_tab_rule_prefix = "tab_"
79734
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   108
val zipperposition_cnf_rule = "cnf"
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   109
val pseudo_zipperposition_conjunct = "conjunct"
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   110
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   111
val pseudo_zipperposition_skolemization_suffix = ".skolem"
58653
4b44c227c0e0 improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
blanchet
parents: 58652
diff changeset
   112
50670
eaa540986291 properly take the existential closure of skolems
blanchet
parents: 49983
diff changeset
   113
fun term_name' (Var ((s, _), _)) = perhaps (try Name.dest_skolem) s
52034
11b48e7a4e7e correctly 'repair' the monomorphization context for SMT solvers from Sledgehammer
blanchet
parents: 52031
diff changeset
   114
  | term_name' _ = ""
50670
eaa540986291 properly take the existential closure of skolems
blanchet
parents: 49983
diff changeset
   115
eaa540986291 properly take the existential closure of skolems
blanchet
parents: 49983
diff changeset
   116
fun lambda' v = Term.lambda_name (term_name' v, v)
eaa540986291 properly take the existential closure of skolems
blanchet
parents: 49983
diff changeset
   117
78693
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   118
fun If_const T = Const (\<^const_name>\<open>If\<close>, HOLogic.boolT --> T --> T --> T)
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   119
50670
eaa540986291 properly take the existential closure of skolems
blanchet
parents: 49983
diff changeset
   120
fun forall_of v t = HOLogic.all_const (fastype_of v) $ lambda' v t
eaa540986291 properly take the existential closure of skolems
blanchet
parents: 49983
diff changeset
   121
fun exists_of v t = HOLogic.exists_const (fastype_of v) $ lambda' v t
39425
5d97fd83ab37 fix parsing of higher-order formulas;
blanchet
parents: 39374
diff changeset
   122
43135
8c32a0160b0d more uniform handling of tfree sort inference in ATP reconstruction code, based on what Metis always has done
blanchet
parents: 43131
diff changeset
   123
fun make_tfree ctxt w =
8c32a0160b0d more uniform handling of tfree sort inference in ATP reconstruction code, based on what Metis always has done
blanchet
parents: 43131
diff changeset
   124
  let val ww = "'" ^ w in
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   125
    TFree (ww, the_default \<^sort>\<open>type\<close> (Variable.def_sort ctxt (ww, ~1)))
43135
8c32a0160b0d more uniform handling of tfree sort inference in ATP reconstruction code, based on what Metis always has done
blanchet
parents: 43131
diff changeset
   126
  end
8c32a0160b0d more uniform handling of tfree sort inference in ATP reconstruction code, based on what Metis always has done
blanchet
parents: 43131
diff changeset
   127
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   128
fun simplify_bool ((all as Const (\<^const_name>\<open>All\<close>, _)) $ Abs (s, T, t)) =
57767
5bc204ca27ce centralized boolean simplification so that e.g. LEO-II benefits from it
blanchet
parents: 57765
diff changeset
   129
    let val t' = simplify_bool t in
5bc204ca27ce centralized boolean simplification so that e.g. LEO-II benefits from it
blanchet
parents: 57765
diff changeset
   130
      if loose_bvar1 (t', 0) then all $ Abs (s, T, t') else t'
5bc204ca27ce centralized boolean simplification so that e.g. LEO-II benefits from it
blanchet
parents: 57765
diff changeset
   131
    end
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   132
  | simplify_bool (Const (\<^const_name>\<open>Not\<close>, _) $ t) = s_not (simplify_bool t)
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   133
  | simplify_bool (Const (\<^const_name>\<open>conj\<close>, _) $ t $ u) =
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   134
    s_conj (simplify_bool t, simplify_bool u)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   135
  | simplify_bool (Const (\<^const_name>\<open>disj\<close>, _) $ t $ u) =
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   136
    s_disj (simplify_bool t, simplify_bool u)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   137
  | simplify_bool (Const (\<^const_name>\<open>implies\<close>, _) $ t $ u) =
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   138
    s_imp (simplify_bool t, simplify_bool u)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   139
  | simplify_bool ((t as Const (\<^const_name>\<open>HOL.eq\<close>, _)) $ u $ v) =
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   140
    (case (u, v) of
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   141
      (Const (\<^const_name>\<open>True\<close>, _), _) => v
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   142
    | (u, Const (\<^const_name>\<open>True\<close>, _)) => u
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   143
    | (Const (\<^const_name>\<open>False\<close>, _), v) => s_not v
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   144
    | (u, Const (\<^const_name>\<open>False\<close>, _)) => s_not u
74379
9ea507f63bcb clarified antiquotations;
wenzelm
parents: 74050
diff changeset
   145
    | _ => if u aconv v then \<^Const>\<open>True\<close> else t $ simplify_bool u $ simplify_bool v)
57767
5bc204ca27ce centralized boolean simplification so that e.g. LEO-II benefits from it
blanchet
parents: 57765
diff changeset
   146
  | simplify_bool (t $ u) = simplify_bool t $ simplify_bool u
5bc204ca27ce centralized boolean simplification so that e.g. LEO-II benefits from it
blanchet
parents: 57765
diff changeset
   147
  | simplify_bool (Abs (s, T, t)) = Abs (s, T, simplify_bool t)
5bc204ca27ce centralized boolean simplification so that e.g. LEO-II benefits from it
blanchet
parents: 57765
diff changeset
   148
  | simplify_bool t = t
5bc204ca27ce centralized boolean simplification so that e.g. LEO-II benefits from it
blanchet
parents: 57765
diff changeset
   149
57765
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   150
fun single_letter upper s =
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   151
  let val s' = if String.isPrefix "o" s orelse String.isPrefix "O" s then "z" else s in
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   152
    String.extract (Name.desymbolize (SOME upper) (Long_Name.base_name s'), 0, SOME 1)
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   153
  end
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   154
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   155
fun var_name_of_typ (Type (\<^type_name>\<open>fun\<close>, [_, T])) =
57765
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   156
    if body_type T = HOLogic.boolT then "p" else "f"
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   157
  | var_name_of_typ (Type (\<^type_name>\<open>set\<close>, [T])) =
58600
c9e8ad426ab1 get rid of 'individual' type in DFG proofs
blanchet
parents: 58599
diff changeset
   158
    let fun default () = single_letter true (var_name_of_typ T) in
58599
733b7a3277b2 slightly nicer names
blanchet
parents: 58597
diff changeset
   159
      (case T of
733b7a3277b2 slightly nicer names
blanchet
parents: 58597
diff changeset
   160
        Type (s, [T1, T2]) => if String.isSuffix "prod" s andalso T1 = T2 then "r" else default ()
733b7a3277b2 slightly nicer names
blanchet
parents: 58597
diff changeset
   161
      | _ => default ())
733b7a3277b2 slightly nicer names
blanchet
parents: 58597
diff changeset
   162
    end
57765
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   163
  | var_name_of_typ (Type (s, Ts)) =
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   164
    if String.isSuffix "list" s then var_name_of_typ (the_single Ts) ^ "s"
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   165
    else single_letter false (Long_Name.base_name s)
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   166
  | var_name_of_typ (TFree (s, _)) = single_letter false (perhaps (try (unprefix "'")) s)
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   167
  | var_name_of_typ (TVar ((s, _), T)) = var_name_of_typ (TFree (s, T))
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   168
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   169
fun rename_bound_vars (t $ u) = rename_bound_vars t $ rename_bound_vars u
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   170
  | rename_bound_vars (Abs (_, T, t)) = Abs (var_name_of_typ T, T, rename_bound_vars t)
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   171
  | rename_bound_vars t = t
f1108245ba11 better handling of variable names
blanchet
parents: 57717
diff changeset
   172
54820
d9ab86c044fd extended ATP types with sorts
blanchet
parents: 54819
diff changeset
   173
exception ATP_CLASS of string list
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   174
exception ATP_TYPE of string atp_type list
54811
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   175
exception ATP_TERM of (string, string atp_type) atp_term list
53586
bd5fa6425993 prefixed types and some functions with "atp_" for disambiguation
blanchet
parents: 52758
diff changeset
   176
exception ATP_FORMULA of
54811
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   177
  (string, string, (string, string atp_type) atp_term, string) atp_formula list
37991
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   178
exception SAME of unit
21978
72c21698a055 Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
paulson
parents:
diff changeset
   179
54820
d9ab86c044fd extended ATP types with sorts
blanchet
parents: 54819
diff changeset
   180
fun class_of_atp_class cls =
d9ab86c044fd extended ATP types with sorts
blanchet
parents: 54819
diff changeset
   181
  (case unprefix_and_unascii class_prefix cls of
d9ab86c044fd extended ATP types with sorts
blanchet
parents: 54819
diff changeset
   182
    SOME s => s
d9ab86c044fd extended ATP types with sorts
blanchet
parents: 54819
diff changeset
   183
  | NONE => raise ATP_CLASS [cls])
d9ab86c044fd extended ATP types with sorts
blanchet
parents: 54819
diff changeset
   184
57697
44341963ade3 correctly translate THF functions from terms to types
blanchet
parents: 57635
diff changeset
   185
fun atp_type_of_atp_term (ATerm ((s, _), us)) =
44341963ade3 correctly translate THF functions from terms to types
blanchet
parents: 57635
diff changeset
   186
  let val tys = map atp_type_of_atp_term us in
44341963ade3 correctly translate THF functions from terms to types
blanchet
parents: 57635
diff changeset
   187
    if s = tptp_fun_type then
44341963ade3 correctly translate THF functions from terms to types
blanchet
parents: 57635
diff changeset
   188
      (case tys of
44341963ade3 correctly translate THF functions from terms to types
blanchet
parents: 57635
diff changeset
   189
        [ty1, ty2] => AFun (ty1, ty2)
44341963ade3 correctly translate THF functions from terms to types
blanchet
parents: 57635
diff changeset
   190
      | _ => raise ATP_TYPE tys)
44341963ade3 correctly translate THF functions from terms to types
blanchet
parents: 57635
diff changeset
   191
    else
44341963ade3 correctly translate THF functions from terms to types
blanchet
parents: 57635
diff changeset
   192
      AType ((s, []), tys)
37991
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   193
  end
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   194
58477
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   195
(* Type variables are given the basic sort "HOL.type". Some will later be constrained by information
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   196
   from type literals, or by type inference. *)
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   197
fun typ_of_atp_type ctxt (ty as AType ((a, clss), tys)) =
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   198
    let val Ts = map (typ_of_atp_type ctxt) tys in
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   199
      (case unprefix_and_unascii native_type_prefix a of
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   200
        SOME b => typ_of_atp_type ctxt (atp_type_of_atp_term (unmangled_type b))
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   201
      | NONE =>
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   202
        (case unprefix_and_unascii type_const_prefix a of
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   203
          SOME b => Type (invert_const b, Ts)
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   204
        | NONE =>
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   205
          if not (null tys) then
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   206
            raise ATP_TYPE [ty] (* only "tconst"s have type arguments *)
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   207
          else
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   208
            (case unprefix_and_unascii tfree_prefix a of
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   209
              SOME b => make_tfree ctxt b
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   210
            | NONE =>
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   211
              (* The term could be an Isabelle variable or a variable from the ATP, say "X1" or "_5018".
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   212
                 Sometimes variables from the ATP are indistinguishable from Isabelle variables, which
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   213
                 forces us to use a type parameter in all cases. *)
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   214
              Type_Infer.param 0 ("'" ^ perhaps (unprefix_and_unascii tvar_prefix) a,
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   215
                (if null clss then \<^sort>\<open>type\<close> else map class_of_atp_class clss)))))
58477
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   216
    end
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   217
  | typ_of_atp_type ctxt (AFun (ty1, ty2)) = typ_of_atp_type ctxt ty1 --> typ_of_atp_type ctxt ty2
8438bae06e63 parse back type of SPASS proof variables
blanchet
parents: 58091
diff changeset
   218
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   219
fun typ_of_atp_term ctxt = typ_of_atp_type ctxt o atp_type_of_atp_term
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   220
54789
blanchet
parents: 54788
diff changeset
   221
(* Type class literal applied to a type. Returns triple of polarity, class, type. *)
52031
9a9238342963 tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents: 51878
diff changeset
   222
fun type_constraint_of_term ctxt (u as ATerm ((a, _), us)) =
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   223
  (case (unprefix_and_unascii class_prefix a, map (typ_of_atp_term ctxt) us) of
42606
0c76cf483899 show sorts not just types in Isar proofs + tuning
blanchet
parents: 42595
diff changeset
   224
    (SOME b, [T]) => (b, T)
54789
blanchet
parents: 54788
diff changeset
   225
  | _ => raise ATP_TERM [u])
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   226
43907
073ab5379842 pass type arguments to lambda-lifted Frees, to account for polymorphism
blanchet
parents: 43863
diff changeset
   227
(* Accumulate type constraints in a formula: negative type literals. *)
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   228
fun add_var (key, z) = Vartab.map_default (key, []) (cons z)
42606
0c76cf483899 show sorts not just types in Isar proofs + tuning
blanchet
parents: 42595
diff changeset
   229
fun add_type_constraint false (cl, TFree (a ,_)) = add_var ((a, ~1), cl)
0c76cf483899 show sorts not just types in Isar proofs + tuning
blanchet
parents: 42595
diff changeset
   230
  | add_type_constraint false (cl, TVar (ix, _)) = add_var (ix, cl)
0c76cf483899 show sorts not just types in Isar proofs + tuning
blanchet
parents: 42595
diff changeset
   231
  | add_type_constraint _ _ = I
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   232
57789
a73255cffb5b don't rename variables which will be renamed later anyway
blanchet
parents: 57788
diff changeset
   233
fun repair_var_name s =
55185
a0bd8d6414e6 centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
blanchet
parents: 54822
diff changeset
   234
  (case unprefix_and_unascii schematic_var_prefix s of
57789
a73255cffb5b don't rename variables which will be renamed later anyway
blanchet
parents: 57788
diff changeset
   235
    SOME s' => s'
a73255cffb5b don't rename variables which will be renamed later anyway
blanchet
parents: 57788
diff changeset
   236
  | NONE => s)
55185
a0bd8d6414e6 centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
blanchet
parents: 54822
diff changeset
   237
54789
blanchet
parents: 54788
diff changeset
   238
(* The number of type arguments of a constant, zero if it's monomorphic. For (instances of) Skolem
blanchet
parents: 54788
diff changeset
   239
   pseudoconstants, this information is encoded in the constant name. *)
52125
ac7830871177 improved handling of free variables' types in Isar proofs
blanchet
parents: 52034
diff changeset
   240
fun robust_const_num_type_args thy s =
43907
073ab5379842 pass type arguments to lambda-lifted Frees, to account for polymorphism
blanchet
parents: 43863
diff changeset
   241
  if String.isPrefix skolem_const_prefix s then
46711
f745bcc4a1e5 more explicit Long_Name operations (NB: analyzing qualifiers is inherently fragile);
wenzelm
parents: 46435
diff changeset
   242
    s |> Long_Name.explode |> List.last |> Int.fromString |> the
45554
09ad83de849c don't pass "lam_lifted" option to "metis" unless there's a good reason
blanchet
parents: 45553
diff changeset
   243
  else if String.isPrefix lam_lifted_prefix s then
09ad83de849c don't pass "lam_lifted" option to "metis" unless there's a good reason
blanchet
parents: 45553
diff changeset
   244
    if String.isPrefix lam_lifted_poly_prefix s then 2 else 0
43907
073ab5379842 pass type arguments to lambda-lifted Frees, to account for polymorphism
blanchet
parents: 43863
diff changeset
   245
  else
073ab5379842 pass type arguments to lambda-lifted Frees, to account for polymorphism
blanchet
parents: 43863
diff changeset
   246
    (s, Sign.the_const_type thy s) |> Sign.const_typargs thy |> length
073ab5379842 pass type arguments to lambda-lifted Frees, to account for polymorphism
blanchet
parents: 43863
diff changeset
   247
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   248
fun slack_fastype_of t = fastype_of t handle TERM _ => Type_Infer.anyT \<^sort>\<open>type\<close>
43182
649bada59658 slacker version of "fastype_of", in case a function has dummy type
blanchet
parents: 43176
diff changeset
   249
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   250
val spass_skolem_prefixes = ["skc", "skf"]
79734
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   251
val zipperposition_skolem_prefix = "sk"
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   252
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   253
fun is_spass_skolem s =
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   254
  exists (fn pre => String.isPrefix pre s) spass_skolem_prefixes
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   255
79734
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   256
val is_zipperposition_skolem = String.isPrefix zipperposition_skolem_prefix
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   257
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   258
fun is_reverse_skolem s =
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   259
  exists (fn pre => String.isPrefix pre s) (zipperposition_skolem_prefix :: spass_skolem_prefixes)
50703
76a2e506c125 swap Vampire's Skolem arguments to bring them in line with what E and metis's new skolemizer do (helps Isar proof reconstruction in some cases)
blanchet
parents: 50693
diff changeset
   260
78693
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   261
val zip_internal_ite_prefix = "zip_internal_ite_"
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   262
57257
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   263
fun var_index_of_textual textual = if textual then 0 else 1
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   264
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   265
fun quantify_over_var textual quant_of var_s var_T t =
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   266
  let
57790
a04e8a39ca9a tuned code
blanchet
parents: 57789
diff changeset
   267
    val vars =
a04e8a39ca9a tuned code
blanchet
parents: 57789
diff changeset
   268
      ((var_s, var_index_of_textual textual), var_T) ::
a04e8a39ca9a tuned code
blanchet
parents: 57789
diff changeset
   269
      filter (fn ((s, _), _) => s = var_s) (Term.add_vars t [])
57257
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   270
    val normTs = vars |> AList.group (op =) |> map (apsnd hd)
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   271
    fun norm_var_types (Var (x, T)) =
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   272
        Var (x, the_default T (AList.lookup (op =) normTs x))
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   273
      | norm_var_types t = t
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   274
  in t |> map_aterms norm_var_types |> fold_rev quant_of (map Var normTs) end
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   275
78697
8ca71c0ae31f avoid legacy binding errors in Sledgehammer Isar proofs
blanchet
parents: 78696
diff changeset
   276
(* This assumes that distinct names are mapped to distinct names by
8ca71c0ae31f avoid legacy binding errors in Sledgehammer Isar proofs
blanchet
parents: 78696
diff changeset
   277
   "Variable.variant_frees". This does not hold in general but should hold for
8ca71c0ae31f avoid legacy binding errors in Sledgehammer Isar proofs
blanchet
parents: 78696
diff changeset
   278
   ATP-generated Skolem function names, since these end with a digit and
8ca71c0ae31f avoid legacy binding errors in Sledgehammer Isar proofs
blanchet
parents: 78696
diff changeset
   279
   "variant_frees" appends letters. *)
8ca71c0ae31f avoid legacy binding errors in Sledgehammer Isar proofs
blanchet
parents: 78696
diff changeset
   280
fun desymbolize_and_fresh_up ctxt s =
8ca71c0ae31f avoid legacy binding errors in Sledgehammer Isar proofs
blanchet
parents: 78696
diff changeset
   281
  fst (hd (Variable.variant_frees ctxt [] [(Name.desymbolize (SOME false) s, ())]))
57790
a04e8a39ca9a tuned code
blanchet
parents: 57789
diff changeset
   282
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   283
(* Higher-order translation. Variables are typed (although we don't use that information). Lambdas
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   284
   are typed. The code is similar to "term_of_atp_fo". *)
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   285
fun term_of_atp_ho ctxt sym_tab =
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   286
  let
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   287
    val thy = Proof_Context.theory_of ctxt
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   288
    val var_index = var_index_of_textual true
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   289
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   290
    fun do_term opt_T u =
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   291
      (case u of
78696
ef89f1beee95 parse applie lambdas correctly plus deal gracefully with lambda-lifting in Zipperposition
blanchet
parents: 78693
diff changeset
   292
        AAbs (((var, ty), term), us) =>
57257
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   293
        let
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   294
          val typ = typ_of_atp_type ctxt ty
57789
a73255cffb5b don't rename variables which will be renamed later anyway
blanchet
parents: 57788
diff changeset
   295
          val var_name = repair_var_name var
57257
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   296
          val tm = do_term NONE term
78696
ef89f1beee95 parse applie lambdas correctly plus deal gracefully with lambda-lifting in Zipperposition
blanchet
parents: 78693
diff changeset
   297
          val lam = quantify_over_var true lambda' var_name typ tm
ef89f1beee95 parse applie lambdas correctly plus deal gracefully with lambda-lifting in Zipperposition
blanchet
parents: 78693
diff changeset
   298
          val args = map (do_term NONE) us
ef89f1beee95 parse applie lambdas correctly plus deal gracefully with lambda-lifting in Zipperposition
blanchet
parents: 78693
diff changeset
   299
        in
ef89f1beee95 parse applie lambdas correctly plus deal gracefully with lambda-lifting in Zipperposition
blanchet
parents: 78693
diff changeset
   300
          list_comb (lam, args)
ef89f1beee95 parse applie lambdas correctly plus deal gracefully with lambda-lifting in Zipperposition
blanchet
parents: 78693
diff changeset
   301
        end
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   302
      | ATerm ((s, tys), us) =>
74050
blanchet
parents: 72967
diff changeset
   303
        if s = "" (* special marker generated on parse error *) then
blanchet
parents: 72967
diff changeset
   304
          error "Isar proof reconstruction failed because the ATP proof contains unparsable \
blanchet
parents: 72967
diff changeset
   305
            \material"
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   306
        else if s = tptp_equal then
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   307
          list_comb (Const (\<^const_name>\<open>HOL.eq\<close>, Type_Infer.anyT \<^sort>\<open>type\<close>),
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   308
            map (do_term NONE) us)
75052
9e1d486e2d9f careful with partial applications
blanchet
parents: 75048
diff changeset
   309
        else if s = tptp_not_equal andalso length us = 2 then
75048
e926618f9474 handle TPTP '!=' more gracefully in Isar proof reconstruction
blanchet
parents: 74379
diff changeset
   310
          \<^const>\<open>HOL.Not\<close> $ list_comb (Const (\<^const_name>\<open>HOL.eq\<close>, Type_Infer.anyT \<^sort>\<open>type\<close>),
e926618f9474 handle TPTP '!=' more gracefully in Isar proof reconstruction
blanchet
parents: 74379
diff changeset
   311
            map (do_term NONE) us)
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   312
        else if not (null us) then
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   313
          let
57820
wenzelm
parents: 57792
diff changeset
   314
            val args = map (do_term NONE) us
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   315
            val opt_T' = SOME (map slack_fastype_of args ---> the_default dummyT opt_T)
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   316
            val func = do_term opt_T' (ATerm ((s, tys), []))
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   317
          in foldl1 (op $) (func :: args) end
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   318
        else if s = tptp_or then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   319
          HOLogic.disj
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   320
        else if s = tptp_and then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   321
          HOLogic.conj
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   322
        else if s = tptp_implies then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   323
          HOLogic.imp
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   324
        else if s = tptp_iff orelse s = tptp_equal then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   325
          HOLogic.eq_const dummyT
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   326
        else if s = tptp_not_iff orelse s = tptp_not_equal then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   327
          \<^term>\<open>\<lambda>x y. x \<noteq> y\<close>
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   328
        else if s = tptp_if then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   329
          \<^term>\<open>\<lambda>P Q. Q \<longrightarrow> P\<close>
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   330
        else if s = tptp_not_and then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   331
          \<^term>\<open>\<lambda>P Q. \<not> (P \<and> Q)\<close>
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   332
        else if s = tptp_not_or then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   333
          \<^term>\<open>\<lambda>P Q. \<not> (P \<or> Q)\<close>
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   334
        else if s = tptp_not then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   335
          HOLogic.Not
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   336
        else if s = tptp_ho_forall then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   337
          HOLogic.all_const dummyT
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   338
        else if s = tptp_ho_exists then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   339
          HOLogic.exists_const dummyT
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   340
        else if s = tptp_hilbert_choice then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   341
          HOLogic.choice_const dummyT
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   342
        else if s = tptp_hilbert_the then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   343
          \<^term>\<open>The\<close>
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   344
        else if String.isPrefix zip_internal_ite_prefix s then
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   345
          If_const dummyT
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   346
        else
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   347
          (case unprefix_and_unascii const_prefix s of
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   348
            SOME s' =>
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   349
            let
57547
677b07d777c3 don't generate TPTP THF 'Definition's, because they complicate reconstruction for AgsyHOL and Satallax
blanchet
parents: 57267
diff changeset
   350
              val ((s', _), mangled_us) = s' |> unmangled_const |>> `invert_const
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   351
              val num_ty_args = length us - the_default 0 (Symtab.lookup sym_tab s)
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   352
              val (type_us, term_us) = chop num_ty_args us |>> append mangled_us
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   353
              val term_ts = map (do_term NONE) term_us
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   354
              val Ts = map (typ_of_atp_type ctxt) tys @ map (typ_of_atp_term ctxt) type_us
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   355
              val T =
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   356
                (if not (null Ts) andalso robust_const_num_type_args thy s' = length Ts then
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   357
                   try (Sign.const_instance thy) (s', Ts)
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   358
                 else
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   359
                   NONE)
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   360
                |> (fn SOME T => T
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   361
                     | NONE =>
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   362
                       map slack_fastype_of term_ts --->
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   363
                       the_default (Type_Infer.anyT \<^sort>\<open>type\<close>) opt_T)
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   364
              val t = Const (unproxify_const s', T)
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   365
            in list_comb (t, term_ts) end
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   366
          | NONE => (* a free or schematic variable *)
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   367
            let
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   368
              val ts = map (do_term NONE) us
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   369
              val T =
58500
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   370
                (case tys of
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   371
                  [ty] => typ_of_atp_type ctxt ty
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   372
                | _ =>
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   373
                  map slack_fastype_of ts --->
58500
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   374
                  (case opt_T of
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   375
                    SOME T => T
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   376
                  | NONE => Type_Infer.anyT \<^sort>\<open>type\<close>))
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   377
              val t =
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   378
                (case unprefix_and_unascii fixed_var_prefix s of
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   379
                  SOME s => Free (s, T)
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   380
                | NONE =>
78697
8ca71c0ae31f avoid legacy binding errors in Sledgehammer Isar proofs
blanchet
parents: 78696
diff changeset
   381
                  if not (is_tptp_variable s) then Free (desymbolize_and_fresh_up ctxt s, T)
57789
a73255cffb5b don't rename variables which will be renamed later anyway
blanchet
parents: 57788
diff changeset
   382
                  else Var ((repair_var_name s, var_index), T))
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   383
            in list_comb (t, ts) end))
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   384
  in do_term end
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   385
56254
a2dd9200854d more antiquotations;
wenzelm
parents: 56104
diff changeset
   386
(* First-order translation. No types are known for variables. "Type_Infer.anyT @{sort type}"
a2dd9200854d more antiquotations;
wenzelm
parents: 56104
diff changeset
   387
   should allow them to be inferred. *)
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   388
fun term_of_atp_fo ctxt textual sym_tab =
36909
7d5587f6d5f7 made Sledgehammer's full-typed proof reconstruction work for the first time;
blanchet
parents: 36607
diff changeset
   389
  let
43135
8c32a0160b0d more uniform handling of tfree sort inference in ATP reconstruction code, based on what Metis always has done
blanchet
parents: 43131
diff changeset
   390
    val thy = Proof_Context.theory_of ctxt
54789
blanchet
parents: 54788
diff changeset
   391
    (* For Metis, we use 1 rather than 0 because variable references in clauses may otherwise
blanchet
parents: 54788
diff changeset
   392
       conflict with variable constraints in the goal. At least, type inference often fails
blanchet
parents: 54788
diff changeset
   393
       otherwise. See also "axiom_inference" in "Metis_Reconstruct". *)
57257
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   394
    val var_index = var_index_of_textual textual
57199
blanchet
parents: 56854
diff changeset
   395
43131
9e9420122f91 fixed interaction between type tags and hAPP in reconstruction code
blanchet
parents: 43130
diff changeset
   396
    fun do_term extra_ts opt_T u =
54789
blanchet
parents: 54788
diff changeset
   397
      (case u of
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   398
        ATerm ((s, tys), us) =>
74050
blanchet
parents: 72967
diff changeset
   399
        if s = "" (* special marker generated on parse error *) then
57199
blanchet
parents: 56854
diff changeset
   400
          error "Isar proof reconstruction failed because the ATP proof contains unparsable \
63692
1bc4bc2c9fd1 killed final stops in Sledgehammer and friends
blanchet
parents: 59582
diff changeset
   401
            \material"
51878
f11039b31bae handle dummy atp terms
smolkas
parents: 51192
diff changeset
   402
        else if String.isPrefix native_type_prefix s then
74379
9ea507f63bcb clarified antiquotations;
wenzelm
parents: 74050
diff changeset
   403
          \<^Const>\<open>True\<close> (* ignore TPTP type information (needed?) *)
44773
e701dabbfe37 perform mangling before computing symbol arity, to avoid needless "hAPP"s and "hBOOL"s
blanchet
parents: 44399
diff changeset
   404
        else if s = tptp_equal then
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   405
          list_comb (Const (\<^const_name>\<open>HOL.eq\<close>, Type_Infer.anyT \<^sort>\<open>type\<close>),
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   406
            map (do_term [] NONE) us)
54789
blanchet
parents: 54788
diff changeset
   407
        else
blanchet
parents: 54788
diff changeset
   408
          (case unprefix_and_unascii const_prefix s of
blanchet
parents: 54788
diff changeset
   409
            SOME s' =>
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   410
            let val ((s', s''), mangled_us) = s' |> unmangled_const |>> `invert_const in
54789
blanchet
parents: 54788
diff changeset
   411
              if s' = type_tag_name then
blanchet
parents: 54788
diff changeset
   412
                (case mangled_us @ us of
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   413
                  [typ_u, term_u] => do_term extra_ts (SOME (typ_of_atp_term ctxt typ_u)) term_u
54789
blanchet
parents: 54788
diff changeset
   414
                | _ => raise ATP_TERM us)
blanchet
parents: 54788
diff changeset
   415
              else if s' = predicator_name then
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   416
                do_term [] (SOME \<^typ>\<open>bool\<close>) (hd us)
54789
blanchet
parents: 54788
diff changeset
   417
              else if s' = app_op_name then
blanchet
parents: 54788
diff changeset
   418
                let val extra_t = do_term [] NONE (List.last us) in
blanchet
parents: 54788
diff changeset
   419
                  do_term (extra_t :: extra_ts)
57199
blanchet
parents: 56854
diff changeset
   420
                    (case opt_T of SOME T => SOME (slack_fastype_of extra_t --> T) | NONE => NONE)
blanchet
parents: 56854
diff changeset
   421
                    (nth us (length us - 2))
54789
blanchet
parents: 54788
diff changeset
   422
                end
blanchet
parents: 54788
diff changeset
   423
              else if s' = type_guard_name then
74379
9ea507f63bcb clarified antiquotations;
wenzelm
parents: 74050
diff changeset
   424
                \<^Const>\<open>True\<close> (* ignore type predicates *)
54789
blanchet
parents: 54788
diff changeset
   425
              else
blanchet
parents: 54788
diff changeset
   426
                let
blanchet
parents: 54788
diff changeset
   427
                  val new_skolem = String.isPrefix new_skolem_const_prefix s''
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   428
                  val num_ty_args = length us - the_default 0 (Symtab.lookup sym_tab s)
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   429
                  val (type_us, term_us) = chop num_ty_args us |>> append mangled_us
54789
blanchet
parents: 54788
diff changeset
   430
                  val term_ts = map (do_term [] NONE) term_us
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   431
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   432
                  val Ts = map (typ_of_atp_type ctxt) tys @ map (typ_of_atp_term ctxt) type_us
54789
blanchet
parents: 54788
diff changeset
   433
                  val T =
54818
a80bd631e573 honor SPASS-Pirate type arguments
blanchet
parents: 54811
diff changeset
   434
                    (if not (null Ts) andalso robust_const_num_type_args thy s' = length Ts then
57199
blanchet
parents: 56854
diff changeset
   435
                       if new_skolem then SOME (Type_Infer.paramify_vars (tl Ts ---> hd Ts))
blanchet
parents: 56854
diff changeset
   436
                       else if textual then try (Sign.const_instance thy) (s', Ts)
blanchet
parents: 56854
diff changeset
   437
                       else NONE
54789
blanchet
parents: 54788
diff changeset
   438
                     else
blanchet
parents: 54788
diff changeset
   439
                       NONE)
blanchet
parents: 54788
diff changeset
   440
                    |> (fn SOME T => T
blanchet
parents: 54788
diff changeset
   441
                         | NONE =>
56254
a2dd9200854d more antiquotations;
wenzelm
parents: 56104
diff changeset
   442
                           map slack_fastype_of term_ts --->
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   443
                           the_default (Type_Infer.anyT \<^sort>\<open>type\<close>) opt_T)
54789
blanchet
parents: 54788
diff changeset
   444
                  val t =
blanchet
parents: 54788
diff changeset
   445
                    if new_skolem then Var ((new_skolem_var_name_of_const s'', var_index), T)
blanchet
parents: 54788
diff changeset
   446
                    else Const (unproxify_const s', T)
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   447
                in
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   448
                  list_comb (t, term_ts @ extra_ts)
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   449
                end
54789
blanchet
parents: 54788
diff changeset
   450
            end
blanchet
parents: 54788
diff changeset
   451
          | NONE => (* a free or schematic variable *)
blanchet
parents: 54788
diff changeset
   452
            let
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   453
              val term_ts = map (do_term [] NONE) us |> is_reverse_skolem s ? rev
54789
blanchet
parents: 54788
diff changeset
   454
              val ts = term_ts @ extra_ts
blanchet
parents: 54788
diff changeset
   455
              val T =
58500
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   456
                (case tys of
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   457
                  [ty] => typ_of_atp_type ctxt ty
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   458
                | _ =>
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   459
                  (case opt_T of
430306aa03b1 proper types for applied variables, for typed formats (TFF0, DFG)
blanchet
parents: 58484
diff changeset
   460
                    SOME T => map slack_fastype_of term_ts ---> T
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   461
                  | NONE => map slack_fastype_of ts ---> Type_Infer.anyT \<^sort>\<open>type\<close>))
54789
blanchet
parents: 54788
diff changeset
   462
              val t =
blanchet
parents: 54788
diff changeset
   463
                (case unprefix_and_unascii fixed_var_prefix s of
blanchet
parents: 54788
diff changeset
   464
                  SOME s => Free (s, T)
36909
7d5587f6d5f7 made Sledgehammer's full-typed proof reconstruction work for the first time;
blanchet
parents: 36607
diff changeset
   465
                | NONE =>
55185
a0bd8d6414e6 centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
blanchet
parents: 54822
diff changeset
   466
                  if textual andalso not (is_tptp_variable s) then
78697
8ca71c0ae31f avoid legacy binding errors in Sledgehammer Isar proofs
blanchet
parents: 78696
diff changeset
   467
                    Free (desymbolize_and_fresh_up ctxt s, T)
55185
a0bd8d6414e6 centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
blanchet
parents: 54822
diff changeset
   468
                  else
57789
a73255cffb5b don't rename variables which will be renamed later anyway
blanchet
parents: 57788
diff changeset
   469
                    Var ((repair_var_name s, var_index), T))
54789
blanchet
parents: 54788
diff changeset
   470
            in list_comb (t, ts) end))
43093
blanchet
parents: 43085
diff changeset
   471
  in do_term [] end
21978
72c21698a055 Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
paulson
parents:
diff changeset
   472
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   473
fun term_of_atp ctxt (ATP_Problem.THF _) type_enc =
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   474
    if ATP_Problem_Generate.is_type_enc_higher_order type_enc then K (term_of_atp_ho ctxt)
63692
1bc4bc2c9fd1 killed final stops in Sledgehammer and friends
blanchet
parents: 59582
diff changeset
   475
    else error "Unsupported Isar reconstruction"
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   476
  | term_of_atp ctxt _ type_enc =
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   477
    if not (ATP_Problem_Generate.is_type_enc_higher_order type_enc) then term_of_atp_fo ctxt
63692
1bc4bc2c9fd1 killed final stops in Sledgehammer and friends
blanchet
parents: 59582
diff changeset
   478
    else error "Unsupported Isar reconstruction"
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   479
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   480
fun term_of_atom ctxt format type_enc textual sym_tab pos (u as ATerm ((s, _), _)) =
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   481
  if String.isPrefix class_prefix s then
52031
9a9238342963 tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents: 51878
diff changeset
   482
    add_type_constraint pos (type_constraint_of_term ctxt u)
74379
9ea507f63bcb clarified antiquotations;
wenzelm
parents: 74050
diff changeset
   483
    #> pair \<^Const>\<open>True\<close>
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   484
  else
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   485
    pair (term_of_atp ctxt format type_enc textual sym_tab (SOME \<^typ>\<open>bool\<close>) u)
36402
1b20805974c7 introduced direct proof reconstruction code, eliminating the need for the "neg_clausify" method;
blanchet
parents: 36396
diff changeset
   486
37991
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   487
(* Update schematic type variables with detected sort constraints. It's not
42563
e70ffe3846d0 improve helper type instantiation code
blanchet
parents: 42562
diff changeset
   488
   totally clear whether this code is necessary. *)
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   489
fun repair_tvar_sorts (t, tvar_tab) =
36909
7d5587f6d5f7 made Sledgehammer's full-typed proof reconstruction work for the first time;
blanchet
parents: 36607
diff changeset
   490
  let
37991
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   491
    fun do_type (Type (a, Ts)) = Type (a, map do_type Ts)
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   492
      | do_type (TVar (xi, s)) =
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   493
        TVar (xi, the_default s (Vartab.lookup tvar_tab xi))
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   494
      | do_type (TFree z) = TFree z
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   495
    fun do_term (Const (a, T)) = Const (a, do_type T)
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   496
      | do_term (Free (a, T)) = Free (a, do_type T)
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   497
      | do_term (Var (xi, T)) = Var (xi, do_type T)
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   498
      | do_term (t as Bound _) = t
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   499
      | do_term (Abs (a, T, t)) = Abs (a, do_type T, do_term t)
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   500
      | do_term (t1 $ t2) = do_term t1 $ do_term t2
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   501
  in t |> not (Vartab.is_empty tvar_tab) ? do_term end
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   502
54811
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   503
(* Interpret an ATP formula as a HOL term, extracting sort constraints as they appear in the
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   504
   formula. *)
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   505
fun prop_of_atp ctxt format type_enc textual sym_tab phi =
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   506
  let
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   507
    fun do_formula pos phi =
54789
blanchet
parents: 54788
diff changeset
   508
      (case phi of
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   509
        AQuant (_, [], phi) => do_formula pos phi
42526
46d485f8d144 added room for types in ATP quantifiers
blanchet
parents: 42451
diff changeset
   510
      | AQuant (q, (s, _) :: xs, phi') =>
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   511
        do_formula pos (AQuant (q, xs, phi'))
42526
46d485f8d144 added room for types in ATP quantifiers
blanchet
parents: 42451
diff changeset
   512
        (* FIXME: TFF *)
57257
0d5e34ba4d28 Correcting the type parser
fleury
parents: 57256
diff changeset
   513
        #>> quantify_over_var textual (case q of AForall => forall_of | AExists => exists_of)
57789
a73255cffb5b don't rename variables which will be renamed later anyway
blanchet
parents: 57788
diff changeset
   514
          (repair_var_name s) dummyT
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   515
      | AConn (ANot, [phi']) => do_formula (not pos) phi' #>> s_not
37991
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   516
      | AConn (c, [phi1, phi2]) =>
38014
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   517
        do_formula (pos |> c = AImplies ? not) phi1
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   518
        ##>> do_formula pos phi2
81c23d286f0c extract sort constraints from FOFs properly;
blanchet
parents: 38007
diff changeset
   519
        #>> (case c of
54811
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   520
              AAnd => s_conj
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   521
            | AOr => s_disj
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   522
            | AImplies => s_imp
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   523
            | AIff => s_iff
df56a01f5684 parse SPASS-Pirate types
blanchet
parents: 54799
diff changeset
   524
            | ANot => raise Fail "impossible connective")
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   525
      | AAtom tm => term_of_atom ctxt format type_enc textual sym_tab pos tm
54789
blanchet
parents: 54788
diff changeset
   526
      | _ => raise ATP_FORMULA [phi])
blanchet
parents: 54788
diff changeset
   527
  in
blanchet
parents: 54788
diff changeset
   528
    repair_tvar_sorts (do_formula true phi Vartab.empty)
blanchet
parents: 54788
diff changeset
   529
  end
37991
3093ab32f1e7 proof reconstruction for full FOF terms
blanchet
parents: 37962
diff changeset
   530
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   531
val unprefix_fact_number = space_implode "_" o tl o space_explode "_"
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   532
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   533
fun resolve_fact facts s =
54789
blanchet
parents: 54788
diff changeset
   534
  (case try (unprefix fact_prefix) s of
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   535
    SOME s' =>
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   536
    let val s' = s' |> unprefix_fact_number |> unascii_of in
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   537
      AList.lookup (op =) facts s' |> Option.map (pair s')
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   538
    end
54789
blanchet
parents: 54788
diff changeset
   539
  | NONE => NONE)
54506
blanchet
parents: 54505
diff changeset
   540
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   541
fun resolve_conjecture s =
54789
blanchet
parents: 54788
diff changeset
   542
  (case try (unprefix conjecture_prefix) s of
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   543
    SOME s' => Int.fromString s'
54789
blanchet
parents: 54788
diff changeset
   544
  | NONE => NONE)
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   545
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   546
fun resolve_facts facts = map_filter (resolve_fact facts)
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   547
val resolve_conjectures = map_filter resolve_conjecture
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   548
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   549
fun is_axiom_used_in_proof pred =
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   550
  exists (fn ((_, ss), _, _, _, []) => exists pred ss | _ => false)
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   551
77432
e51aa922079a tweaked Sledgehammer interaction
blanchet
parents: 77430
diff changeset
   552
val is_conjecture_used_in_proof = is_axiom_used_in_proof (is_some o resolve_conjecture)
e51aa922079a tweaked Sledgehammer interaction
blanchet
parents: 77430
diff changeset
   553
70940
ce3a05ad07b7 added support for Zipperposition on SystemOnTPTP
blanchet
parents: 69597
diff changeset
   554
fun add_fact ctxt facts ((num, ss), _, _, rule, deps) =
58653
4b44c227c0e0 improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
blanchet
parents: 58652
diff changeset
   555
  (if member (op =) [agsyhol_core_rule, leo2_extcnf_equal_neg_rule] rule orelse
4b44c227c0e0 improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
blanchet
parents: 58652
diff changeset
   556
      String.isPrefix satallax_tab_rule_prefix rule then
56104
fd6e132ee4fb correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
blanchet
parents: 55285
diff changeset
   557
     insert (op =) (short_thm_name ctxt ext, (Global, General))
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   558
   else
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   559
     I)
70940
ce3a05ad07b7 added support for Zipperposition on SystemOnTPTP
blanchet
parents: 69597
diff changeset
   560
  #> (if null deps then union (op =) (resolve_facts facts (num :: ss)) else I)
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   561
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   562
fun used_facts_in_atp_proof ctxt facts atp_proof =
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   563
  if null atp_proof then facts else fold (add_fact ctxt facts) atp_proof []
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   564
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   565
val ascii_of_lam_fact_prefix = ascii_of lam_fact_prefix
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   566
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   567
(* overapproximation (good enough) *)
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   568
fun is_lam_lifted s =
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   569
  String.isPrefix fact_prefix s andalso
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   570
  String.isSubstring ascii_of_lam_fact_prefix s
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   571
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   572
val is_combinator_def = String.isPrefix (helper_prefix ^ combinator_prefix)
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   573
55257
abfd7b90bba2 rationalized threading of 'metis' arguments
blanchet
parents: 55195
diff changeset
   574
fun atp_proof_prefers_lifting atp_proof =
abfd7b90bba2 rationalized threading of 'metis' arguments
blanchet
parents: 55195
diff changeset
   575
  (is_axiom_used_in_proof is_combinator_def atp_proof,
abfd7b90bba2 rationalized threading of 'metis' arguments
blanchet
parents: 55195
diff changeset
   576
   is_axiom_used_in_proof is_lam_lifted atp_proof) = (false, true)
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   577
81254
d3c0734059ee variable instantiation in Sledgehammer and Metis
blanchet
parents: 79734
diff changeset
   578
val is_lam_def_used_in_atp_proof =
d3c0734059ee variable instantiation in Sledgehammer and Metis
blanchet
parents: 79734
diff changeset
   579
  is_axiom_used_in_proof (is_combinator_def orf is_lam_lifted)
d3c0734059ee variable instantiation in Sledgehammer and Metis
blanchet
parents: 79734
diff changeset
   580
54500
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   581
val is_typed_helper_name =
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   582
  String.isPrefix helper_prefix andf String.isSuffix typed_helper_suffix
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   583
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   584
fun is_typed_helper_used_in_atp_proof atp_proof =
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   585
  is_axiom_used_in_proof is_typed_helper_name atp_proof
f625e0e79dd1 refactoring
blanchet
parents: 54499
diff changeset
   586
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   587
fun replace_one_dependency (old, new) dep = if is_same_atp_step dep old then new else [dep]
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   588
fun replace_dependencies_in_line old_new (name, role, t, rule, deps) =
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   589
  (name, role, t, rule, fold (union (op =) o replace_one_dependency old_new) deps [])
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   590
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   591
fun repair_name "$true" = "c_True"
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   592
  | repair_name "$false" = "c_False"
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   593
  | repair_name "$$e" = tptp_equal (* seen in Vampire proofs *)
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   594
  | repair_name s =
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   595
    if is_tptp_equal s orelse
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   596
       (* seen in Vampire proofs *)
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   597
       (String.isPrefix "sQ" s andalso String.isSuffix "_eqProxy" s) then
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   598
      tptp_equal
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   599
    else
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   600
      s
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   601
57699
a6cf197c1f1e also try 'metis' with 'full_types'
blanchet
parents: 57697
diff changeset
   602
fun set_var_index j = map_aterms (fn Var ((s, 0), T) => Var ((s, j), T) | t => t)
57635
97adb86619a4 more robust handling of types for skolems (modeled as Frees)
blanchet
parents: 57547
diff changeset
   603
57699
a6cf197c1f1e also try 'metis' with 'full_types'
blanchet
parents: 57697
diff changeset
   604
fun infer_formulas_types ctxt =
57635
97adb86619a4 more robust handling of types for skolems (modeled as Frees)
blanchet
parents: 57547
diff changeset
   605
  map_index (uncurry (fn j => set_var_index j #> Type.constraint HOLogic.boolT))
97adb86619a4 more robust handling of types for skolems (modeled as Frees)
blanchet
parents: 57547
diff changeset
   606
  #> Syntax.check_terms (Proof_Context.set_mode Proof_Context.mode_schematic ctxt)
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   607
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   608
val combinator_table =
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   609
  [(\<^const_name>\<open>Meson.COMBI\<close>, @{thm Meson.COMBI_def [abs_def]}),
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   610
   (\<^const_name>\<open>Meson.COMBK\<close>, @{thm Meson.COMBK_def [abs_def]}),
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   611
   (\<^const_name>\<open>Meson.COMBB\<close>, @{thm Meson.COMBB_def [abs_def]}),
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   612
   (\<^const_name>\<open>Meson.COMBC\<close>, @{thm Meson.COMBC_def [abs_def]}),
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   613
   (\<^const_name>\<open>Meson.COMBS\<close>, @{thm Meson.COMBS_def [abs_def]})]
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   614
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   615
fun uncombine_term thy =
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   616
  let
57717
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   617
    fun uncomb (t1 $ t2) = betapply (uncomb t1, uncomb t2)
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   618
      | uncomb (Abs (s, T, t)) = Abs (s, T, uncomb t)
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   619
      | uncomb (t as Const (x as (s, _))) =
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   620
        (case AList.lookup (op =) combinator_table s of
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59577
diff changeset
   621
          SOME thm => thm |> Thm.prop_of |> specialize_type thy x |> Logic.dest_equals |> snd
54756
blanchet
parents: 54507
diff changeset
   622
        | NONE => t)
57717
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   623
      | uncomb t = t
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   624
  in uncomb end
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   625
57717
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   626
fun unlift_aterm lifted (t as Const (s, _)) =
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   627
    if String.isPrefix lam_lifted_prefix s then
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   628
      (* FIXME: do something about the types *)
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   629
      (case AList.lookup (op =) lifted s of
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   630
        SOME t' => unlift_term lifted t'
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   631
      | NONE => t)
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   632
    else
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   633
      t
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   634
  | unlift_aterm _ t = t
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   635
and unlift_term lifted =
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   636
  map_aterms (unlift_aterm lifted)
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   637
57256
cf43583f9bb9 imported patch leo2_skolem_simplication
fleury
parents: 57255
diff changeset
   638
fun termify_line _ _ _ _ _ (_, Type_Role, _, _, _) = NONE
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   639
  | termify_line ctxt format type_enc lifted sym_tab (name, role, u, rule, deps) =
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   640
    let
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   641
      val thy = Proof_Context.theory_of ctxt
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   642
      val t = u
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   643
        |> prop_of_atp ctxt format type_enc true sym_tab
57717
949838aba487 unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
blanchet
parents: 57713
diff changeset
   644
        |> unlift_term lifted
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   645
        |> uncombine_term thy
57768
a63f14f1214c fine-tuned Isar reconstruction, esp. boolean simplifications
blanchet
parents: 57767
diff changeset
   646
        |> simplify_bool
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   647
    in
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   648
      SOME (name, role, t, rule, deps)
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   649
    end
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   650
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   651
val waldmeister_conjecture_num = "1.0.0.0"
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   652
54756
blanchet
parents: 54507
diff changeset
   653
fun repair_waldmeister_endgame proof =
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   654
  let
74379
9ea507f63bcb clarified antiquotations;
wenzelm
parents: 74050
diff changeset
   655
    fun repair_tail (name, _, \<^Const>\<open>Trueprop for t\<close>, rule, deps) =
9ea507f63bcb clarified antiquotations;
wenzelm
parents: 74050
diff changeset
   656
      (name, Negated_Conjecture, \<^Const>\<open>Trueprop for \<open>s_not t\<close>\<close>, rule, deps)
54756
blanchet
parents: 54507
diff changeset
   657
    fun repair_body [] = []
blanchet
parents: 54507
diff changeset
   658
      | repair_body ((line as ((num, _), _, _, _, _)) :: lines) =
blanchet
parents: 54507
diff changeset
   659
        if num = waldmeister_conjecture_num then map repair_tail (line :: lines)
blanchet
parents: 54507
diff changeset
   660
        else line :: repair_body lines
blanchet
parents: 54507
diff changeset
   661
  in
blanchet
parents: 54507
diff changeset
   662
    repair_body proof
blanchet
parents: 54507
diff changeset
   663
  end
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   664
57635
97adb86619a4 more robust handling of types for skolems (modeled as Frees)
blanchet
parents: 57547
diff changeset
   665
fun map_proof_terms f (lines : ('a * 'b * 'c * 'd * 'e) list) =
97adb86619a4 more robust handling of types for skolems (modeled as Frees)
blanchet
parents: 57547
diff changeset
   666
  map2 (fn c => fn (a, b, _, d, e) => (a, b, c, d, e)) (f (map #3 lines)) lines
97adb86619a4 more robust handling of types for skolems (modeled as Frees)
blanchet
parents: 57547
diff changeset
   667
57258
67d85a8aa6cc Moving the remote prefix deleting on Sledgehammer's side
fleury
parents: 57257
diff changeset
   668
fun termify_atp_proof ctxt local_prover format type_enc pool lifted sym_tab =
57267
8b87114357bd integrated new Waldmeister code with 'sledgehammer' command
blanchet
parents: 57263
diff changeset
   669
  nasty_atp_proof pool
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   670
  #> map_term_names_in_atp_proof repair_name
57255
488046fdda59 add support for Isar reconstruction for thf1 ATP provers like Leo-II.
fleury
parents: 57199
diff changeset
   671
  #> map_filter (termify_line ctxt format type_enc lifted sym_tab)
57699
a6cf197c1f1e also try 'metis' with 'full_types'
blanchet
parents: 57697
diff changeset
   672
  #> map_proof_terms (infer_formulas_types ctxt #> map HOLogic.mk_Trueprop)
57258
67d85a8aa6cc Moving the remote prefix deleting on Sledgehammer's side
fleury
parents: 57257
diff changeset
   673
  #> local_prover = waldmeisterN ? repair_waldmeister_endgame
54499
319f8659267d refactoring
blanchet
parents: 53586
diff changeset
   674
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   675
fun unskolemize_spass_term skos =
55192
b75b52c7cf94 unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
blanchet
parents: 55185
diff changeset
   676
  let
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   677
    val is_skolem_name = member (op =) skos
55192
b75b52c7cf94 unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
blanchet
parents: 55185
diff changeset
   678
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   679
    fun find_argless_skolem (Free _ $ Var _) = NONE
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   680
      | find_argless_skolem (Free (x as (s, _))) = if is_skolem_name s then SOME x else NONE
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   681
      | find_argless_skolem (t $ u) =
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   682
        (case find_argless_skolem t of NONE => find_argless_skolem u | sk => sk)
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   683
      | find_argless_skolem (Abs (_, _, t)) = find_argless_skolem t
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   684
      | find_argless_skolem _ = NONE
55192
b75b52c7cf94 unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
blanchet
parents: 55185
diff changeset
   685
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   686
    fun find_skolem_arg (Free (s, _) $ Var v) = if is_skolem_name s then SOME v else NONE
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   687
      | find_skolem_arg (t $ u) = (case find_skolem_arg t of NONE => find_skolem_arg u | v => v)
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   688
      | find_skolem_arg (Abs (_, _, t)) = find_skolem_arg t
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   689
      | find_skolem_arg _ = NONE
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   690
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   691
    fun kill_skolem_arg (t as Free (s, T) $ Var _) =
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   692
        if is_skolem_name s then Free (s, range_type T) else t
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   693
      | kill_skolem_arg (t $ u) = kill_skolem_arg t $ kill_skolem_arg u
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   694
      | kill_skolem_arg (Abs (s, T, t)) = Abs (s, T, kill_skolem_arg t)
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   695
      | kill_skolem_arg t = t
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   696
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   697
    fun find_var (Var v) = SOME v
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   698
      | find_var (t $ u) = (case find_var t of NONE => find_var u | v => v)
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   699
      | find_var (Abs (_, _, t)) = find_var t
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   700
      | find_var _ = NONE
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   701
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   702
    val safe_abstract_over = abstract_over o apsnd (incr_boundvars 1)
55192
b75b52c7cf94 unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
blanchet
parents: 55185
diff changeset
   703
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   704
    fun unskolem_inner t =
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   705
      (case find_argless_skolem t of
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   706
        SOME (x as (s, T)) =>
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   707
        HOLogic.exists_const T $ Abs (s, T, unskolem_inner (safe_abstract_over (Free x, t)))
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   708
      | NONE =>
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   709
        (case find_skolem_arg t of
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   710
          SOME (v as ((s, _), T)) =>
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   711
          let
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   712
            val (haves, have_nots) =
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   713
              HOLogic.disjuncts t
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   714
              |> List.partition (exists_subterm (curry (op =) (Var v)))
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   715
              |> apply2 (fn lits => fold (curry s_disj) lits \<^term>\<open>False\<close>)
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   716
          in
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   717
            s_disj (HOLogic.all_const T
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   718
                $ Abs (s, T, unskolem_inner (safe_abstract_over (Var v, kill_skolem_arg haves))),
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   719
              unskolem_inner have_nots)
58091
ecf5826ba234 reworked unskolemization for SPASS
blanchet
parents: 57820
diff changeset
   720
          end
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   721
        | NONE =>
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   722
          (case find_var t of
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   723
            SOME (v as ((s, _), T)) =>
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   724
            HOLogic.all_const T $ Abs (s, T, unskolem_inner (safe_abstract_over (Var v, t)))
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   725
          | NONE => t)))
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   726
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   727
    fun unskolem_outer (@{const Trueprop} $ t) = @{const Trueprop} $ unskolem_outer t
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   728
      | unskolem_outer t = unskolem_inner t
55195
067142c53c3b reverted unsound optimization
blanchet
parents: 55192
diff changeset
   729
  in
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   730
    unskolem_outer
55192
b75b52c7cf94 unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
blanchet
parents: 55185
diff changeset
   731
  end
b75b52c7cf94 unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
blanchet
parents: 55185
diff changeset
   732
57788
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   733
fun rename_skolem_args t =
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   734
  let
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   735
    fun add_skolem_args (Abs (_, _, t)) = add_skolem_args t
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   736
      | add_skolem_args t =
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   737
        (case strip_comb t of
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   738
          (Free (s, _), args as _ :: _) =>
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   739
          if is_spass_skolem s then insert (op =) (s, take_prefix is_Var args)
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   740
          else fold add_skolem_args args
57788
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   741
        | (u, args as _ :: _) => fold add_skolem_args (u :: args)
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   742
        | _ => I)
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   743
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   744
    fun subst_of_skolem (sk, args) =
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   745
      map_index (fn (j, Var (z, T)) => (z, Var ((sk ^ "_" ^ string_of_int j, 0), T))) args
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   746
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   747
    val subst = maps subst_of_skolem (add_skolem_args t [])
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   748
  in
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   749
    subst_vars ([], subst) t
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   750
  end
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   751
72401
2783779b7dd3 removed obsolete unmaintained experimental prover Pirate
blanchet
parents: 70940
diff changeset
   752
fun introduce_spass_skolems proof =
57787
blanchet
parents: 57785
diff changeset
   753
  let
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   754
    fun add_skolem (Free (s, _)) = is_spass_skolem s ? insert (op =) s
57788
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   755
      | add_skolem _ = I
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   756
57787
blanchet
parents: 57785
diff changeset
   757
    (* union-find would be faster *)
blanchet
parents: 57785
diff changeset
   758
    fun add_cycle [] = I
blanchet
parents: 57785
diff changeset
   759
      | add_cycle ss =
blanchet
parents: 57785
diff changeset
   760
        fold (fn s => Graph.default_node (s, ())) ss
blanchet
parents: 57785
diff changeset
   761
        #> fold Graph.add_edge (ss ~~ tl ss @ [hd ss])
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   762
57787
blanchet
parents: 57785
diff changeset
   763
    val (input_steps, other_steps) = List.partition (null o #5) proof
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   764
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   765
    (* The names of the formulas are added to the Skolem constants, to ensure that formulas giving
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   766
       rise to several clauses are skolemized together. *)
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   767
    val skoXss = map (fn ((_, ss), _, t, _, _) => Term.fold_aterms add_skolem t ss) input_steps
58601
85fa90262807 avoid creating needless skolemization steps for SPASS
blanchet
parents: 58600
diff changeset
   768
    val groups0 = Graph.strong_conn (fold add_cycle skoXss Graph.empty)
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   769
    val groups = filter (exists is_spass_skolem) groups0
58601
85fa90262807 avoid creating needless skolemization steps for SPASS
blanchet
parents: 58600
diff changeset
   770
85fa90262807 avoid creating needless skolemization steps for SPASS
blanchet
parents: 58600
diff changeset
   771
    val skoXss_input_steps = skoXss ~~ input_steps
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   772
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   773
    fun step_name_of_group skoXs = (implode skoXs, [])
57787
blanchet
parents: 57785
diff changeset
   774
    fun in_group group = member (op =) group o hd
58601
85fa90262807 avoid creating needless skolemization steps for SPASS
blanchet
parents: 58600
diff changeset
   775
    fun group_of skoX = find_first (fn group => in_group group skoX) groups
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   776
58652
da12763acd6b made SML/NJ happier
blanchet
parents: 58601
diff changeset
   777
    fun new_steps (skoXss_steps : (string list * (term, 'a) atp_step) list) group =
57787
blanchet
parents: 57785
diff changeset
   778
      let
blanchet
parents: 57785
diff changeset
   779
        val name = step_name_of_group group
blanchet
parents: 57785
diff changeset
   780
        val name0 = name |>> prefix "0"
57788
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   781
        val t =
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   782
          (case map (snd #> #3) skoXss_steps of
57788
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   783
            [t] => t
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   784
          | ts => ts
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   785
            |> map (HOLogic.dest_Trueprop #> rename_skolem_args)
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   786
            |> Library.foldr1 s_conj
0a38c47ebb69 normalize skolem argument variable names so that they coincide when taking the conjunction
blanchet
parents: 57787
diff changeset
   787
            |> HOLogic.mk_Trueprop)
79730
4031aafc2dda deal with new-style Vampire skolemization in reconstructed Isar proofs
blanchet
parents: 78697
diff changeset
   788
        val skos = fold (union (op =) o filter is_spass_skolem o fst) skoXss_steps []
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   789
        val deps = map (snd #> #1) skoXss_steps
57787
blanchet
parents: 57785
diff changeset
   790
      in
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   791
        [(name0, Unknown, unskolemize_spass_term skos t, spass_pre_skolemize_rule, deps),
57787
blanchet
parents: 57785
diff changeset
   792
         (name, Unknown, t, spass_skolemize_rule, [name0])]
blanchet
parents: 57785
diff changeset
   793
      end
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   794
57787
blanchet
parents: 57785
diff changeset
   795
    val sko_steps =
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   796
      maps (fn group => new_steps (filter (in_group group o fst) skoXss_input_steps) group) groups
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   797
57787
blanchet
parents: 57785
diff changeset
   798
    val old_news =
58601
85fa90262807 avoid creating needless skolemization steps for SPASS
blanchet
parents: 58600
diff changeset
   799
      map_filter (fn (skoXs, (name, _, _, _, _)) =>
85fa90262807 avoid creating needless skolemization steps for SPASS
blanchet
parents: 58600
diff changeset
   800
          Option.map (pair name o single o step_name_of_group) (group_of skoXs))
58597
21a741e96970 improved unskolemization of SPASS problems
blanchet
parents: 58500
diff changeset
   801
        skoXss_input_steps
57787
blanchet
parents: 57785
diff changeset
   802
    val repair_deps = fold replace_dependencies_in_line old_news
blanchet
parents: 57785
diff changeset
   803
  in
blanchet
parents: 57785
diff changeset
   804
    input_steps @ sko_steps @ map repair_deps other_steps
blanchet
parents: 57785
diff changeset
   805
  end
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   806
79734
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   807
fun regroup_zipperposition_skolems steps =
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   808
  let
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   809
    val contains_skolem =
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   810
      Term.exists_subterm (fn Free (sk, _) => is_zipperposition_skolem sk | _ => false)
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   811
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   812
    fun is_skolem_step (_, _, t, rule, _) =
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   813
      rule = zipperposition_cnf_rule andalso contains_skolem t
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   814
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   815
    val dep_to_skolem_steps = steps
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   816
      |> filter is_skolem_step
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   817
      |> map_filter (fn step as (_, _, _, _, [dep]) => SOME (fst dep, step)
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   818
        | _ => NONE)
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   819
      |> AList.group (op =)
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   820
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   821
    val prop_of_skolem_steps =
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   822
      map (#3 #> perhaps (try HOLogic.dest_Trueprop))
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   823
      #> Library.foldr1 HOLogic.mk_conj
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   824
      #> HOLogic.mk_Trueprop
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   825
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   826
    fun insert_back_regrouped_skolem_steps (step as (name, _, _, _, _)) =
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   827
      (case AList.lookup (op =) dep_to_skolem_steps (fst name) of
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   828
        SOME skolem_steps =>
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   829
        [step, ((fst name ^ pseudo_zipperposition_skolemization_suffix, []), Plain,
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   830
           prop_of_skolem_steps skolem_steps, zipperposition_cnf_rule, [name])]
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   831
      | NONE => [step])
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   832
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   833
    fun adjust_dependencies (step as (name, role, t, _, [dep])) =
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   834
        if is_skolem_step step then
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   835
          (name, role, t, pseudo_zipperposition_conjunct,
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   836
           [(fst dep ^ pseudo_zipperposition_skolemization_suffix, [])])
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   837
        else
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   838
          step
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   839
     | adjust_dependencies step = step
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   840
  in
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   841
    steps
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   842
    |> map adjust_dependencies
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   843
    |> maps insert_back_regrouped_skolem_steps
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   844
  end
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   845
78693
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   846
val zf_stmt_prefix = "zf_stmt_"
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   847
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   848
fun is_if_True_or_False_axiom true_or_false t =
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   849
  (case t of
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   850
    @{const Trueprop} $
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   851
     (Const (@{const_name HOL.eq}, _) $
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   852
       (Const (@{const_name If}, _) $ cond $ Var _ $ Var _) $
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   853
       Var _) =>
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   854
     cond aconv true_or_false
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   855
  | _ => false)
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   856
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   857
fun factify_atp_proof facts hyp_ts concl_t atp_proof =
54505
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   858
  let
57785
0388026060d1 deal with E definitions
blanchet
parents: 57768
diff changeset
   859
    fun factify_step ((num, ss), role, t, rule, deps) =
54505
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   860
      let
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   861
        val (ss', role', t') =
57263
2b6a96cc64c9 simplified code
blanchet
parents: 57258
diff changeset
   862
          (case resolve_conjectures ss of
54505
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   863
            [j] =>
58484
b4c0e2b00036 support hypotheses with schematics in Isar proofs
blanchet
parents: 58477
diff changeset
   864
            if j = length hyp_ts then ([], Conjecture, concl_t)
b4c0e2b00036 support hypotheses with schematics in Isar proofs
blanchet
parents: 58477
diff changeset
   865
            else ([], Hypothesis, close_form (nth hyp_ts j))
55185
a0bd8d6414e6 centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
blanchet
parents: 54822
diff changeset
   866
          | _ =>
70940
ce3a05ad07b7 added support for Zipperposition on SystemOnTPTP
blanchet
parents: 69597
diff changeset
   867
            (case resolve_facts facts (num :: ss) of
78693
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   868
              [] =>
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   869
              if role = Axiom andalso String.isPrefix zf_stmt_prefix num
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   870
                 andalso is_if_True_or_False_axiom @{const True} t then
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   871
                (["if_True"], Axiom, t)
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   872
              else if role = Axiom andalso String.isPrefix zf_stmt_prefix num
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   873
                 andalso is_if_True_or_False_axiom @{const False} t then
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   874
                (["if_False"], Axiom, t)
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   875
              else
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   876
                (ss,
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   877
                 if role = Definition then Definition
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   878
                 else if role = Lemma then Lemma
1c0576840bf4 reconstruct Zipperposition's if-then-else in Sledgehammer Isar proofs
blanchet
parents: 77602
diff changeset
   879
                 else Plain, t)
55185
a0bd8d6414e6 centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
blanchet
parents: 54822
diff changeset
   880
            | facts => (map fst facts, Axiom, t)))
54505
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   881
      in
79734
0fa4bebbdd75 support Zipperposition's skolemization in generated Isar proofs
blanchet
parents: 79730
diff changeset
   882
        ((num, ss' |> distinct (op =)), role', t', rule, deps)
54505
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   883
      end
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   884
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   885
    val atp_proof = map factify_step atp_proof
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   886
    val names = map #1 atp_proof
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   887
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   888
    fun repair_dep (num, ss) = (num, the_default ss (AList.lookup (op =) names num))
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   889
    fun repair_deps (name, role, t, rule, deps) = (name, role, t, rule, map repair_dep deps)
54772
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   890
  in
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   891
    map repair_deps atp_proof
f5fd4a34b0e8 handle Skolems gracefully for SPASS as well
blanchet
parents: 54770
diff changeset
   892
  end
54505
d023838eb252 more refactoring to accommodate SMT proofs
blanchet
parents: 54501
diff changeset
   893
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   894
fun termify_atp_abduce_candidate ctxt local_prover format type_enc pool lifted sym_tab phi =
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   895
  let
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   896
    val proof = [(("", []), Conjecture, mk_anot phi, "", [])]
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   897
    val new_proof = termify_atp_proof ctxt local_prover format type_enc pool lifted sym_tab proof
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   898
  in
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   899
    (case new_proof of
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   900
      [(_, _, phi', _, _)] => phi'
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   901
    | _ => error "Impossible case in termify_atp_abduce_candidate")
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   902
  end
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   903
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   904
fun sort_top n scored_items =
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   905
  if n <= 0 orelse null scored_items then
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   906
    []
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   907
  else
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   908
    let
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   909
      fun split_min accum [] (_, best_item) = (best_item, List.rev accum)
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   910
        | split_min accum ((score, item) :: scored_items) (best_score, best_item) =
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   911
          if score < best_score then
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   912
            split_min ((best_score, best_item) :: accum) scored_items (score, item)
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   913
          else
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   914
            split_min ((score, item) :: accum) scored_items (best_score, best_item)
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   915
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   916
      val (min_item, other_scored_items) = split_min [] (tl scored_items) (hd scored_items)
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   917
    in
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   918
      min_item :: sort_top (n - 1) (filter_out (equal min_item o snd) other_scored_items)
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   919
      |> distinct (op aconv)
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   920
    end
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   921
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   922
fun top_abduce_candidates max_candidates candidates =
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   923
  let
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   924
    (* We prefer free variables to other constructs, so that e.g. "x \<le> y" is
77576
80bcebe6cf33 require the presence of free variables to do abduction in Sledgehammer
blanchet
parents: 77432
diff changeset
   925
       prioritized over "x \<le> 5". *)
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   926
    fun score t =
77425
bde374587d93 tweaked abduction in Sledgehammer
blanchet
parents: 77421
diff changeset
   927
      Term.fold_aterms (fn t => fn score => score + (case t of Free _ => 1 | _ => 2)) t 0
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   928
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   929
    (* Equations of the form "x = ..." or "... = x" or similar are too specific
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   930
       to be useful. Quantified formulas are also filtered out. As for "True",
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   931
       it may seem an odd choice for abduction, but it sometimes arises in
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   932
       conjunction with type class constraints, which are removed by the
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   933
       termifier. *)
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   934
    fun maybe_score t =
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   935
      (case t of
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   936
        @{prop True} => NONE
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   937
      | @{const Trueprop} $ (Const (@{const_name HOL.eq}, _) $ Free _ $ _) => NONE
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   938
      | @{const Trueprop} $ (Const (@{const_name HOL.eq}, _) $ _ $ Free _) => NONE
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   939
      | @{const Trueprop} $ (@{const less(nat)} $ _ $ @{const zero_class.zero(nat)}) => NONE
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   940
      | @{const Trueprop} $ (@{const less_eq(nat)} $ _ $ @{const zero_class.zero(nat)}) => NONE
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   941
      | @{const Trueprop} $ (@{const less(nat)} $ _ $ @{const one_class.one(nat)}) => NONE
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   942
      | @{const Trueprop} $ (@{const Not} $
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   943
          (@{const less(nat)} $ @{const zero_class.zero(nat)} $ _)) => NONE
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   944
      | @{const Trueprop} $ (@{const Not} $
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   945
          (@{const less_eq(nat)} $ @{const zero_class.zero(nat)} $ _)) => NONE
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   946
      | @{const Trueprop} $ (@{const Not} $
77425
bde374587d93 tweaked abduction in Sledgehammer
blanchet
parents: 77421
diff changeset
   947
          (@{const less_eq(nat)} $ @{const one_class.one(nat)} $ _)) => NONE
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   948
      | @{const Trueprop} $ (Const (@{const_name All}, _) $ _) => NONE
77421
4e8a6354c54f improve ad hoc abduction in Sledgehammer
blanchet
parents: 77418
diff changeset
   949
      | @{const Trueprop} $ (Const (@{const_name Ex}, _) $ _) => NONE
77576
80bcebe6cf33 require the presence of free variables to do abduction in Sledgehammer
blanchet
parents: 77432
diff changeset
   950
      | _ =>
80bcebe6cf33 require the presence of free variables to do abduction in Sledgehammer
blanchet
parents: 77432
diff changeset
   951
        (* We require the presence of at least one free variable. A "missing
80bcebe6cf33 require the presence of free variables to do abduction in Sledgehammer
blanchet
parents: 77432
diff changeset
   952
           assumption" that does not talk about any free variable is likely
80bcebe6cf33 require the presence of free variables to do abduction in Sledgehammer
blanchet
parents: 77432
diff changeset
   953
           spurious. *)
80bcebe6cf33 require the presence of free variables to do abduction in Sledgehammer
blanchet
parents: 77432
diff changeset
   954
        if exists_subterm (fn Free _ => true | _ => false) t then SOME (score t, t)
80bcebe6cf33 require the presence of free variables to do abduction in Sledgehammer
blanchet
parents: 77432
diff changeset
   955
        else NONE)
77418
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   956
  in
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   957
    sort_top max_candidates (map_filter maybe_score candidates)
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   958
  end
a8458f0df4ee implemented ad hoc abduction in Sledgehammer with E
blanchet
parents: 77272
diff changeset
   959
77602
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   960
fun provability_status ctxt t =
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   961
  let
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   962
    val res = Timeout.apply (seconds 0.1)
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   963
      (Thm.term_of o Thm.rhs_of o Simplifier.full_rewrite ctxt) (Thm.cterm_of ctxt t)
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   964
  in
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   965
    if res aconv @{prop True} then SOME true
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   966
    else if res aconv @{prop False} then SOME false
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   967
    else NONE
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   968
  end
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   969
  handle Timeout.TIMEOUT _ => NONE
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   970
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   971
(* Put propositions that simplify to "True" first, and filter out propositions
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   972
   that simplify to "False". *)
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   973
fun sort_propositions_by_provability ctxt ts =
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   974
  let
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   975
    val statuses_ts = map (`(provability_status ctxt)) ts
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   976
  in
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   977
    maps (fn (SOME true, t) => [t] | _ => []) statuses_ts @
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   978
    maps (fn (NONE, t) => [t] | _ => []) statuses_ts
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   979
  end
7c25451ae2c1 use simplifier to classify the missing assumptions in Sledgehammer's abduction mechanism
blanchet
parents: 77576
diff changeset
   980
31038
immler@in.tum.de
parents: 31037
diff changeset
   981
end;