| author | fleury | 
| Wed, 30 Jul 2014 14:03:12 +0200 | |
| changeset 57707 | 0242e9578828 | 
| parent 57703 | fefe3ea75289 | 
| child 57709 | 9cda0c64c37a | 
| permissions | -rw-r--r-- | 
| 46320 | 1  | 
(* Title: HOL/Tools/ATP/atp_proof_reconstruct.ML  | 
| 38027 | 2  | 
Author: Lawrence C. Paulson, Cambridge University Computer Laboratory  | 
3  | 
Author: Claire Quigley, Cambridge University Computer Laboratory  | 
|
| 36392 | 4  | 
Author: Jasmin Blanchette, TU Muenchen  | 
| 
21978
 
72c21698a055
Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
 
paulson 
parents:  
diff
changeset
 | 
5  | 
|
| 49914 | 6  | 
Basic proof reconstruction from ATP proofs.  | 
| 33310 | 7  | 
*)  | 
8  | 
||
| 46320 | 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 | 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 | 14  | 
type stature = ATP_Problem_Generate.stature  | 
| 54772 | 15  | 
type atp_step_name = ATP_Proof.atp_step_name  | 
| 54499 | 16  | 
  type ('a, 'b) atp_step = ('a, 'b) ATP_Proof.atp_step
 | 
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 | 29  | 
val default_metis_lam_trans : string  | 
| 54772 | 30  | 
|
| 
49983
 
33e18e9916a8
use metaquantification when possible in Isar proofs
 
blanchet 
parents: 
49914 
diff
changeset
 | 
31  | 
val forall_of : term -> term -> term  | 
| 
 
33e18e9916a8
use metaquantification when possible in Isar proofs
 
blanchet 
parents: 
49914 
diff
changeset
 | 
32  | 
val exists_of : term -> term -> term  | 
| 55285 | 33  | 
val type_enc_aliases : (string * string list) list  | 
| 
45519
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
34  | 
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
 | 
35  | 
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
 | 
36  | 
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
 | 
37  | 
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
 | 
38  | 
bool -> int Symtab.table ->  | 
| 54811 | 39  | 
(string, string, (string, string atp_type) atp_term, string) atp_formula -> term  | 
| 54499 | 40  | 
|
| 57263 | 41  | 
val used_facts_in_atp_proof : Proof.context -> (string * stature) list -> string atp_proof ->  | 
42  | 
(string * stature) list  | 
|
43  | 
val used_facts_in_unsound_atp_proof : Proof.context -> (string * stature) list -> 'a atp_proof ->  | 
|
44  | 
string list option  | 
|
| 55257 | 45  | 
val atp_proof_prefers_lifting : string atp_proof -> bool  | 
| 54500 | 46  | 
val is_typed_helper_used_in_atp_proof : string atp_proof -> bool  | 
| 54772 | 47  | 
  val replace_dependencies_in_line : atp_step_name * atp_step_name list -> ('a, 'b) atp_step ->
 | 
48  | 
    ('a, 'b) atp_step
 | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
49  | 
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
 | 
50  | 
ATP_Problem_Generate.type_enc -> string Symtab.table -> (string * term) list ->  | 
| 54499 | 51  | 
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
 | 
52  | 
val repair_waldmeister_endgame : (term, 'a) atp_step list -> (term, 'a) atp_step list  | 
| 57699 | 53  | 
val infer_formulas_types : Proof.context -> term list -> term list  | 
| 54772 | 54  | 
val introduce_spass_skolem : (term, string) atp_step list -> (term, string) atp_step list  | 
| 57263 | 55  | 
val factify_atp_proof : (string * 'a) list -> term list -> term -> (term, string) atp_step list ->  | 
56  | 
(term, string) atp_step list  | 
|
| 
24425
 
ca97c6f3d9cd
Returning both a "one-line" proof and a structured proof
 
paulson 
parents: 
24387 
diff
changeset
 | 
57  | 
end;  | 
| 
21978
 
72c21698a055
Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
 
paulson 
parents:  
diff
changeset
 | 
58  | 
|
| 46320 | 59  | 
structure ATP_Proof_Reconstruct : ATP_PROOF_RECONSTRUCT =  | 
| 
21978
 
72c21698a055
Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
 
paulson 
parents:  
diff
changeset
 | 
60  | 
struct  | 
| 
 
72c21698a055
Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
 
paulson 
parents:  
diff
changeset
 | 
61  | 
|
| 
43085
 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 
blanchet 
parents: 
43062 
diff
changeset
 | 
62  | 
open ATP_Util  | 
| 38028 | 63  | 
open ATP_Problem  | 
| 39452 | 64  | 
open ATP_Proof  | 
| 46320 | 65  | 
open ATP_Problem_Generate  | 
| 
21978
 
72c21698a055
Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
 
paulson 
parents:  
diff
changeset
 | 
66  | 
|
| 
45519
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
67  | 
val metisN = "metis"  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
68  | 
|
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
69  | 
val full_typesN = "full_types"  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
70  | 
val partial_typesN = "partial_types"  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
71  | 
val no_typesN = "no_types"  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
72  | 
|
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
73  | 
val really_full_type_enc = "mono_tags"  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
74  | 
val full_type_enc = "poly_guards_query"  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
75  | 
val partial_type_enc = "poly_args"  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
76  | 
val no_type_enc = "erased"  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
77  | 
|
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
78  | 
val full_type_encs = [full_type_enc, really_full_type_enc]  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
79  | 
val partial_type_encs = partial_type_enc :: full_type_encs  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
80  | 
|
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
81  | 
val type_enc_aliases =  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
82  | 
[(full_typesN, full_type_encs),  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
83  | 
(partial_typesN, partial_type_encs),  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
84  | 
(no_typesN, [no_type_enc])]  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
85  | 
|
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
86  | 
fun unalias_type_enc s =  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
87  | 
AList.lookup (op =) type_enc_aliases s |> the_default [s]  | 
| 
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
88  | 
|
| 54500 | 89  | 
val default_metis_lam_trans = combsN  | 
| 
45519
 
cd6e78cb6ee8
make metis reconstruction handling more flexible
 
blanchet 
parents: 
45511 
diff
changeset
 | 
90  | 
|
| 
50670
 
eaa540986291
properly take the existential closure of skolems
 
blanchet 
parents: 
49983 
diff
changeset
 | 
91  | 
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
 | 
92  | 
| term_name' _ = ""  | 
| 
50670
 
eaa540986291
properly take the existential closure of skolems
 
blanchet 
parents: 
49983 
diff
changeset
 | 
93  | 
|
| 
 
eaa540986291
properly take the existential closure of skolems
 
blanchet 
parents: 
49983 
diff
changeset
 | 
94  | 
fun lambda' v = Term.lambda_name (term_name' v, v)  | 
| 
 
eaa540986291
properly take the existential closure of skolems
 
blanchet 
parents: 
49983 
diff
changeset
 | 
95  | 
|
| 
 
eaa540986291
properly take the existential closure of skolems
 
blanchet 
parents: 
49983 
diff
changeset
 | 
96  | 
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
 | 
97  | 
fun exists_of v t = HOLogic.exists_const (fastype_of v) $ lambda' v t  | 
| 39425 | 98  | 
|
| 
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
 | 
99  | 
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
 | 
100  | 
let val ww = "'" ^ w in  | 
| 56254 | 101  | 
    TFree (ww, the_default @{sort type} (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
 | 
102  | 
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
 | 
103  | 
|
| 54820 | 104  | 
exception ATP_CLASS of string list  | 
| 54818 | 105  | 
exception ATP_TYPE of string atp_type list  | 
| 54811 | 106  | 
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
 | 
107  | 
exception ATP_FORMULA of  | 
| 54811 | 108  | 
(string, string, (string, string atp_type) atp_term, string) atp_formula list  | 
| 37991 | 109  | 
exception SAME of unit  | 
| 
21978
 
72c21698a055
Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
 
paulson 
parents:  
diff
changeset
 | 
110  | 
|
| 54820 | 111  | 
fun class_of_atp_class cls =  | 
112  | 
(case unprefix_and_unascii class_prefix cls of  | 
|
113  | 
SOME s => s  | 
|
114  | 
| NONE => raise ATP_CLASS [cls])  | 
|
115  | 
||
| 54811 | 116  | 
(* Type variables are given the basic sort "HOL.type". Some will later be constrained by information  | 
117  | 
from type literals, or by type inference. *)  | 
|
| 54820 | 118  | 
fun typ_of_atp_type ctxt (ty as AType ((a, clss), tys)) =  | 
| 
57697
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
119  | 
let val Ts = map (typ_of_atp_type ctxt) tys in  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
120  | 
(case unprefix_and_unascii type_const_prefix a of  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
121  | 
SOME b => Type (invert_const b, Ts)  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
122  | 
| NONE =>  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
123  | 
if not (null tys) then  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
124  | 
raise ATP_TYPE [ty] (* only "tconst"s have type arguments *)  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
125  | 
else  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
126  | 
(case unprefix_and_unascii tfree_prefix a of  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
127  | 
SOME b => make_tfree ctxt b  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
128  | 
| NONE =>  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
129  | 
(* The term could be an Isabelle variable or a variable from the ATP, say "X1" or "_5018".  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
130  | 
Sometimes variables from the ATP are indistinguishable from Isabelle variables, which  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
131  | 
forces us to use a type parameter in all cases. *)  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
132  | 
            Type_Infer.param 0 ("'" ^ perhaps (unprefix_and_unascii tvar_prefix) a,
 | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
133  | 
              (if null clss then @{sort type} else map class_of_atp_class clss))))
 | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
134  | 
end  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
135  | 
| typ_of_atp_type ctxt (AFun (ty1, ty2)) = typ_of_atp_type ctxt ty1 --> typ_of_atp_type ctxt ty2  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
136  | 
|
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
137  | 
fun atp_type_of_atp_term (ATerm ((s, _), us)) =  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
138  | 
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
 | 
139  | 
if s = tptp_fun_type then  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
140  | 
(case tys of  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
141  | 
[ty1, ty2] => AFun (ty1, ty2)  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
142  | 
| _ => raise ATP_TYPE tys)  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
143  | 
else  | 
| 
 
44341963ade3
correctly translate THF functions from terms to types
 
blanchet 
parents: 
57635 
diff
changeset
 | 
144  | 
AType ((s, []), tys)  | 
| 37991 | 145  | 
end  | 
| 54818 | 146  | 
|
147  | 
fun typ_of_atp_term ctxt = typ_of_atp_type ctxt o atp_type_of_atp_term  | 
|
148  | 
||
| 54789 | 149  | 
(* 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
 | 
150  | 
fun type_constraint_of_term ctxt (u as ATerm ((a, _), us)) =  | 
| 54818 | 151  | 
(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
 | 
152  | 
(SOME b, [T]) => (b, T)  | 
| 54789 | 153  | 
| _ => raise ATP_TERM [u])  | 
| 38014 | 154  | 
|
| 
43907
 
073ab5379842
pass type arguments to lambda-lifted Frees, to account for polymorphism
 
blanchet 
parents: 
43863 
diff
changeset
 | 
155  | 
(* 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
 | 
156  | 
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
 | 
157  | 
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
 | 
158  | 
| 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
 | 
159  | 
| add_type_constraint _ _ = I  | 
| 38014 | 160  | 
|
| 
55185
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
161  | 
fun repair_var_name_raw s =  | 
| 
36486
 
c2d7e2dff59e
support Vampire definitions of constants as "let" constructs in Isar proofs
 
blanchet 
parents: 
36485 
diff
changeset
 | 
162  | 
let  | 
| 
 
c2d7e2dff59e
support Vampire definitions of constants as "let" constructs in Isar proofs
 
blanchet 
parents: 
36485 
diff
changeset
 | 
163  | 
fun subscript_name s n = s ^ nat_subscript n  | 
| 50704 | 164  | 
val s = s |> String.map Char.toLower  | 
| 
36486
 
c2d7e2dff59e
support Vampire definitions of constants as "let" constructs in Isar proofs
 
blanchet 
parents: 
36485 
diff
changeset
 | 
165  | 
in  | 
| 54789 | 166  | 
(case space_explode "_" s of  | 
167  | 
[_] =>  | 
|
168  | 
(case take_suffix Char.isDigit (String.explode s) of  | 
|
169  | 
(cs1 as _ :: _, cs2 as _ :: _) =>  | 
|
170  | 
subscript_name (String.implode cs1) (the (Int.fromString (String.implode cs2)))  | 
|
171  | 
| (_, _) => s)  | 
|
172  | 
| [s1, s2] => (case Int.fromString s2 of SOME n => subscript_name s1 n | NONE => s)  | 
|
173  | 
| _ => s)  | 
|
| 
36486
 
c2d7e2dff59e
support Vampire definitions of constants as "let" constructs in Isar proofs
 
blanchet 
parents: 
36485 
diff
changeset
 | 
174  | 
end  | 
| 
43182
 
649bada59658
slacker version of "fastype_of", in case a function has dummy type
 
blanchet 
parents: 
43176 
diff
changeset
 | 
175  | 
|
| 
55185
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
176  | 
fun repair_var_name textual s =  | 
| 
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
177  | 
(case unprefix_and_unascii schematic_var_prefix s of  | 
| 
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
178  | 
SOME s => s  | 
| 
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
179  | 
| NONE => s |> textual ? repair_var_name_raw)  | 
| 
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
180  | 
|
| 54789 | 181  | 
(* The number of type arguments of a constant, zero if it's monomorphic. For (instances of) Skolem  | 
182  | 
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
 | 
183  | 
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
 | 
184  | 
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
 | 
185  | 
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
 | 
186  | 
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
 | 
187  | 
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
 | 
188  | 
else  | 
| 
 
073ab5379842
pass type arguments to lambda-lifted Frees, to account for polymorphism
 
blanchet 
parents: 
43863 
diff
changeset
 | 
189  | 
(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
 | 
190  | 
|
| 56254 | 191  | 
fun slack_fastype_of t = fastype_of t handle TERM _ => Type_Infer.anyT @{sort type}
 | 
| 
43182
 
649bada59658
slacker version of "fastype_of", in case a function has dummy type
 
blanchet 
parents: 
43176 
diff
changeset
 | 
192  | 
|
| 
51192
 
4dc6bb65c3c3
slacker comparison for Skolems, to avoid trivial equations
 
blanchet 
parents: 
50704 
diff
changeset
 | 
193  | 
(* Cope with "tt(X) = X" atoms, where "X" is existentially quantified. *)  | 
| 
 
4dc6bb65c3c3
slacker comparison for Skolems, to avoid trivial equations
 
blanchet 
parents: 
50704 
diff
changeset
 | 
194  | 
fun loose_aconv (Free (s, _), Free (s', _)) = s = s'  | 
| 
 
4dc6bb65c3c3
slacker comparison for Skolems, to avoid trivial equations
 
blanchet 
parents: 
50704 
diff
changeset
 | 
195  | 
| loose_aconv (t, t') = t aconv t'  | 
| 
 
4dc6bb65c3c3
slacker comparison for Skolems, to avoid trivial equations
 
blanchet 
parents: 
50704 
diff
changeset
 | 
196  | 
|
| 54772 | 197  | 
val spass_skolem_prefix = "sk" (* "skc" or "skf" *)  | 
198  | 
val vampire_skolem_prefix = "sK"  | 
|
| 
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
 | 
199  | 
|
| 57257 | 200  | 
fun var_index_of_textual textual = if textual then 0 else 1  | 
201  | 
||
202  | 
fun quantify_over_var textual quant_of var_s var_T t =  | 
|
203  | 
let  | 
|
204  | 
val vars = ((var_s, var_index_of_textual textual), var_T) ::  | 
|
205  | 
filter (fn ((s, _), _) => s = var_s) (Term.add_vars t [])  | 
|
206  | 
val normTs = vars |> AList.group (op =) |> map (apsnd hd)  | 
|
207  | 
fun norm_var_types (Var (x, T)) =  | 
|
208  | 
Var (x, the_default T (AList.lookup (op =) normTs x))  | 
|
209  | 
| norm_var_types t = t  | 
|
210  | 
in t |> map_aterms norm_var_types |> fold_rev quant_of (map Var normTs) end  | 
|
211  | 
||
212  | 
||
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
213  | 
(* Higher-order translation. Variables are typed (although we don't use that information). Lambdas  | 
| 57256 | 214  | 
are typed.  | 
215  | 
||
216  | 
The code is similar to term_of_atp_fo. *)  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
217  | 
fun term_of_atp_ho ctxt textual sym_tab =  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
218  | 
let  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
219  | 
val thy = Proof_Context.theory_of ctxt  | 
| 57257 | 220  | 
val var_index = var_index_of_textual textual  | 
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
221  | 
|
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
222  | 
fun do_term opt_T u =  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
223  | 
(case u of  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
224  | 
AAbs(((var, ty), term), []) =>  | 
| 57257 | 225  | 
let  | 
226  | 
val typ = typ_of_atp_type ctxt ty  | 
|
227  | 
val var_name = repair_var_name textual var  | 
|
228  | 
val tm = do_term NONE term  | 
|
229  | 
in quantify_over_var textual lambda' var_name typ tm end  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
230  | 
| ATerm ((s, tys), us) =>  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
231  | 
if s = ""  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
232  | 
then error "Isar proof reconstruction failed because the ATP proof \  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
233  | 
\contains unparsable material."  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
234  | 
else if s = tptp_equal then  | 
| 57703 | 235  | 
let  | 
236  | 
val ts = map (do_term NONE) us  | 
|
237  | 
fun equal_term ts =  | 
|
238  | 
                list_comb (Const (@{const_name HOL.eq}, Type_Infer.anyT @{sort type}), ts)
 | 
|
239  | 
in  | 
|
240  | 
if textual then  | 
|
241  | 
(case ts of  | 
|
242  | 
[fst, lst] =>  | 
|
243  | 
if loose_aconv (fst, lst) then  | 
|
244  | 
                  @{const True}
 | 
|
245  | 
                else if Term.aconv_untyped (lst, @{const True}) then
 | 
|
246  | 
fst  | 
|
247  | 
                else if Term.aconv_untyped (fst, @{const True}) then
 | 
|
248  | 
lst  | 
|
249  | 
else  | 
|
250  | 
equal_term ts  | 
|
251  | 
| _ => equal_term ts)  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
252  | 
else  | 
| 57703 | 253  | 
equal_term ts  | 
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
254  | 
end  | 
| 57256 | 255  | 
else if not (null us) then  | 
256  | 
let  | 
|
257  | 
val args = List.map (do_term NONE) us  | 
|
258  | 
val opt_T' = SOME (map slack_fastype_of args ---> the_default dummyT opt_T)  | 
|
259  | 
val func = do_term opt_T' (ATerm ((s, tys), []))  | 
|
260  | 
in foldl1 (op $) (func :: args) end  | 
|
261  | 
else if s = tptp_or then HOLogic.disj  | 
|
262  | 
else if s = tptp_and then HOLogic.conj  | 
|
263  | 
else if s = tptp_implies then HOLogic.imp  | 
|
264  | 
else if s = tptp_iff orelse s = tptp_equal then HOLogic.eq_const dummyT  | 
|
265  | 
        else if s = tptp_not_iff orelse s = tptp_not_equal then @{term "% P Q. Q ~= P"}
 | 
|
266  | 
        else if s = tptp_if then @{term "% P Q. Q --> P"}
 | 
|
267  | 
        else if s = tptp_not_and then @{term "% P Q. ~ (P & Q)"}
 | 
|
268  | 
        else if s = tptp_not_or then @{term "% P Q. ~ (P | Q)"}
 | 
|
269  | 
else if s = tptp_not then HOLogic.Not  | 
|
270  | 
else if s = tptp_ho_forall then HOLogic.all_const dummyT  | 
|
271  | 
else if s = tptp_ho_exists then HOLogic.exists_const dummyT  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
272  | 
else  | 
| 57256 | 273  | 
(case unprefix_and_unascii const_prefix s of  | 
274  | 
SOME s' =>  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
275  | 
let  | 
| 
57547
 
677b07d777c3
don't generate TPTP THF 'Definition's, because they complicate reconstruction for AgsyHOL and Satallax
 
blanchet 
parents: 
57267 
diff
changeset
 | 
276  | 
val ((s', _), mangled_us) = s' |> unmangled_const |>> `invert_const  | 
| 57256 | 277  | 
val num_ty_args = length us - the_default 0 (Symtab.lookup sym_tab s)  | 
278  | 
val (type_us, term_us) = chop num_ty_args us |>> append mangled_us  | 
|
279  | 
val term_ts = map (do_term NONE) term_us  | 
|
280  | 
val Ts = map (typ_of_atp_type ctxt) tys @ map (typ_of_atp_term ctxt) type_us  | 
|
281  | 
val T =  | 
|
282  | 
(if not (null Ts) andalso robust_const_num_type_args thy s' = length Ts then  | 
|
283  | 
if textual then try (Sign.const_instance thy) (s', Ts) else NONE  | 
|
284  | 
else  | 
|
285  | 
NONE)  | 
|
286  | 
|> (fn SOME T => T  | 
|
287  | 
| NONE =>  | 
|
288  | 
map slack_fastype_of term_ts --->  | 
|
289  | 
                       the_default (Type_Infer.anyT @{sort type}) opt_T)
 | 
|
290  | 
val t = Const (unproxify_const s', T)  | 
|
291  | 
in list_comb (t, term_ts) end  | 
|
292  | 
| NONE => (* a free or schematic variable *)  | 
|
293  | 
let  | 
|
294  | 
fun fresh_up s =  | 
|
295  | 
[(s, ())] |> Variable.variant_frees ctxt [] |> hd |> fst  | 
|
296  | 
val ts = map (do_term NONE) us  | 
|
297  | 
val T =  | 
|
298  | 
(case opt_T of  | 
|
299  | 
SOME T => map slack_fastype_of ts ---> T  | 
|
300  | 
| NONE =>  | 
|
301  | 
map slack_fastype_of ts --->  | 
|
302  | 
(case tys of  | 
|
303  | 
[ty] => typ_of_atp_type ctxt ty  | 
|
304  | 
                    | _ => Type_Infer.anyT @{sort type}))
 | 
|
305  | 
val t =  | 
|
306  | 
(case unprefix_and_unascii fixed_var_prefix s of  | 
|
307  | 
SOME s => Free (s, T)  | 
|
308  | 
| NONE =>  | 
|
309  | 
if textual andalso not (is_tptp_variable s) then  | 
|
310  | 
Free (s |> textual ? (repair_var_name_raw #> fresh_up), T)  | 
|
311  | 
else  | 
|
312  | 
Var ((repair_var_name textual s, var_index), T))  | 
|
313  | 
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
 | 
314  | 
in do_term end  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
315  | 
|
| 56254 | 316  | 
(* First-order translation. No types are known for variables. "Type_Infer.anyT @{sort type}"
 | 
317  | 
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
 | 
318  | 
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
 | 
319  | 
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
 | 
320  | 
val thy = Proof_Context.theory_of ctxt  | 
| 54789 | 321  | 
(* For Metis, we use 1 rather than 0 because variable references in clauses may otherwise  | 
322  | 
conflict with variable constraints in the goal. At least, type inference often fails  | 
|
323  | 
otherwise. See also "axiom_inference" in "Metis_Reconstruct". *)  | 
|
| 57257 | 324  | 
val var_index = var_index_of_textual textual  | 
| 57199 | 325  | 
|
| 
43131
 
9e9420122f91
fixed interaction between type tags and hAPP in reconstruction code
 
blanchet 
parents: 
43130 
diff
changeset
 | 
326  | 
fun do_term extra_ts opt_T u =  | 
| 54789 | 327  | 
(case u of  | 
| 54818 | 328  | 
ATerm ((s, tys), us) =>  | 
| 57199 | 329  | 
if s = "" then  | 
330  | 
error "Isar proof reconstruction failed because the ATP proof contains unparsable \  | 
|
331  | 
\material."  | 
|
| 51878 | 332  | 
else if String.isPrefix native_type_prefix s then  | 
| 
42962
 
3b50fdeb6cfc
started adding support for THF output (but no lambdas)
 
blanchet 
parents: 
42943 
diff
changeset
 | 
333  | 
          @{const True} (* ignore TPTP type information *)
 | 
| 
44773
 
e701dabbfe37
perform mangling before computing symbol arity, to avoid needless "hAPP"s and "hBOOL"s
 
blanchet 
parents: 
44399 
diff
changeset
 | 
334  | 
else if s = tptp_equal then  | 
| 43093 | 335  | 
let val ts = map (do_term [] NONE) us in  | 
| 54822 | 336  | 
if textual andalso length ts = 2 andalso loose_aconv (hd ts, List.last ts) then  | 
| 39106 | 337  | 
              @{const True}
 | 
338  | 
else  | 
|
| 56254 | 339  | 
              list_comb (Const (@{const_name HOL.eq}, Type_Infer.anyT @{sort type}), ts)
 | 
| 39106 | 340  | 
end  | 
| 54789 | 341  | 
else  | 
342  | 
(case unprefix_and_unascii const_prefix s of  | 
|
343  | 
SOME s' =>  | 
|
| 54818 | 344  | 
let val ((s', s''), mangled_us) = s' |> unmangled_const |>> `invert_const in  | 
| 54789 | 345  | 
if s' = type_tag_name then  | 
346  | 
(case mangled_us @ us of  | 
|
| 54818 | 347  | 
[typ_u, term_u] => do_term extra_ts (SOME (typ_of_atp_term ctxt typ_u)) term_u  | 
| 54789 | 348  | 
| _ => raise ATP_TERM us)  | 
349  | 
else if s' = predicator_name then  | 
|
350  | 
                do_term [] (SOME @{typ bool}) (hd us)
 | 
|
351  | 
else if s' = app_op_name then  | 
|
352  | 
let val extra_t = do_term [] NONE (List.last us) in  | 
|
353  | 
do_term (extra_t :: extra_ts)  | 
|
| 57199 | 354  | 
(case opt_T of SOME T => SOME (slack_fastype_of extra_t --> T) | NONE => NONE)  | 
355  | 
(nth us (length us - 2))  | 
|
| 54789 | 356  | 
end  | 
357  | 
else if s' = type_guard_name then  | 
|
358  | 
                @{const True} (* ignore type predicates *)
 | 
|
359  | 
else  | 
|
360  | 
let  | 
|
361  | 
val new_skolem = String.isPrefix new_skolem_const_prefix s''  | 
|
| 54818 | 362  | 
val num_ty_args = length us - the_default 0 (Symtab.lookup sym_tab s)  | 
363  | 
val (type_us, term_us) = chop num_ty_args us |>> append mangled_us  | 
|
| 54789 | 364  | 
val term_ts = map (do_term [] NONE) term_us  | 
| 54818 | 365  | 
|
366  | 
val Ts = map (typ_of_atp_type ctxt) tys @ map (typ_of_atp_term ctxt) type_us  | 
|
| 54789 | 367  | 
val T =  | 
| 54818 | 368  | 
(if not (null Ts) andalso robust_const_num_type_args thy s' = length Ts then  | 
| 57199 | 369  | 
if new_skolem then SOME (Type_Infer.paramify_vars (tl Ts ---> hd Ts))  | 
370  | 
else if textual then try (Sign.const_instance thy) (s', Ts)  | 
|
371  | 
else NONE  | 
|
| 54789 | 372  | 
else  | 
373  | 
NONE)  | 
|
374  | 
|> (fn SOME T => T  | 
|
375  | 
| NONE =>  | 
|
| 56254 | 376  | 
map slack_fastype_of term_ts --->  | 
| 57199 | 377  | 
                           the_default (Type_Infer.anyT @{sort type}) opt_T)
 | 
| 54789 | 378  | 
val t =  | 
379  | 
if new_skolem then Var ((new_skolem_var_name_of_const s'', var_index), T)  | 
|
380  | 
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
 | 
381  | 
in  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
382  | 
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
 | 
383  | 
end  | 
| 54789 | 384  | 
end  | 
385  | 
| NONE => (* a free or schematic variable *)  | 
|
386  | 
let  | 
|
387  | 
(* This assumes that distinct names are mapped to distinct names by  | 
|
| 54822 | 388  | 
"Variable.variant_frees". This does not hold in general but should hold for  | 
389  | 
ATP-generated Skolem function names, since these end with a digit and  | 
|
390  | 
"variant_frees" appends letters. *)  | 
|
| 57199 | 391  | 
fun fresh_up s = [(s, ())] |> Variable.variant_frees ctxt [] |> hd |> fst  | 
392  | 
||
| 54789 | 393  | 
val term_ts =  | 
394  | 
map (do_term [] NONE) us  | 
|
395  | 
(* SPASS (3.8ds) and Vampire (2.6) pass arguments to Skolem functions in reverse  | 
|
| 57699 | 396  | 
order, which is incompatible with "metis"'s new skolemizer. *)  | 
| 54789 | 397  | 
|> exists (fn pre => String.isPrefix pre s)  | 
398  | 
[spass_skolem_prefix, vampire_skolem_prefix] ? rev  | 
|
399  | 
val ts = term_ts @ extra_ts  | 
|
400  | 
val T =  | 
|
401  | 
(case opt_T of  | 
|
402  | 
SOME T => map slack_fastype_of term_ts ---> T  | 
|
| 54822 | 403  | 
| NONE =>  | 
404  | 
map slack_fastype_of ts --->  | 
|
| 56254 | 405  | 
                  (case tys of [ty] => typ_of_atp_type ctxt ty | _ => Type_Infer.anyT @{sort type}))
 | 
| 54789 | 406  | 
val t =  | 
407  | 
(case unprefix_and_unascii fixed_var_prefix s of  | 
|
408  | 
SOME s => Free (s, T)  | 
|
| 
36909
 
7d5587f6d5f7
made Sledgehammer's full-typed proof reconstruction work for the first time;
 
blanchet 
parents: 
36607 
diff
changeset
 | 
409  | 
| NONE =>  | 
| 
55185
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
410  | 
if textual andalso not (is_tptp_variable s) then  | 
| 
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
411  | 
Free (s |> textual ? (repair_var_name_raw #> fresh_up), T)  | 
| 
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
412  | 
else  | 
| 
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
413  | 
Var ((repair_var_name textual s, var_index), T))  | 
| 54789 | 414  | 
in list_comb (t, ts) end))  | 
| 43093 | 415  | 
in do_term [] end  | 
| 
21978
 
72c21698a055
Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
 
paulson 
parents:  
diff
changeset
 | 
416  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
417  | 
fun term_of_atp ctxt (ATP_Problem.THF _) type_enc =  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
418  | 
if ATP_Problem_Generate.is_type_enc_higher_order type_enc  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
419  | 
then term_of_atp_ho ctxt  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
420  | 
else error "Unsupported Isar reconstruction."  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
421  | 
| term_of_atp ctxt _ type_enc =  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
422  | 
if not (ATP_Problem_Generate.is_type_enc_higher_order type_enc)  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
423  | 
then term_of_atp_fo ctxt  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
424  | 
else error "Unsupported Isar reconstruction."  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
425  | 
|
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
426  | 
fun term_of_atom ctxt format type_enc textual sym_tab pos (u as ATerm ((s, _), _)) =  | 
| 38014 | 427  | 
if String.isPrefix class_prefix s then  | 
| 
52031
 
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
 
blanchet 
parents: 
51878 
diff
changeset
 | 
428  | 
add_type_constraint pos (type_constraint_of_term ctxt u)  | 
| 38014 | 429  | 
    #> pair @{const True}
 | 
430  | 
else  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
431  | 
    pair (term_of_atp ctxt format type_enc textual sym_tab (SOME @{typ bool}) u)
 | 
| 
36402
 
1b20805974c7
introduced direct proof reconstruction code, eliminating the need for the "neg_clausify" method;
 
blanchet 
parents: 
36396 
diff
changeset
 | 
432  | 
|
| 37991 | 433  | 
(* Update schematic type variables with detected sort constraints. It's not  | 
| 42563 | 434  | 
totally clear whether this code is necessary. *)  | 
| 38014 | 435  | 
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
 | 
436  | 
let  | 
| 37991 | 437  | 
fun do_type (Type (a, Ts)) = Type (a, map do_type Ts)  | 
438  | 
| do_type (TVar (xi, s)) =  | 
|
439  | 
TVar (xi, the_default s (Vartab.lookup tvar_tab xi))  | 
|
440  | 
| do_type (TFree z) = TFree z  | 
|
441  | 
fun do_term (Const (a, T)) = Const (a, do_type T)  | 
|
442  | 
| do_term (Free (a, T)) = Free (a, do_type T)  | 
|
443  | 
| do_term (Var (xi, T)) = Var (xi, do_type T)  | 
|
444  | 
| do_term (t as Bound _) = t  | 
|
445  | 
| do_term (Abs (a, T, t)) = Abs (a, do_type T, do_term t)  | 
|
446  | 
| do_term (t1 $ t2) = do_term t1 $ do_term t2  | 
|
447  | 
in t |> not (Vartab.is_empty tvar_tab) ? do_term end  | 
|
448  | 
||
| 54811 | 449  | 
(* Interpret an ATP formula as a HOL term, extracting sort constraints as they appear in the  | 
450  | 
formula. *)  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
451  | 
fun prop_of_atp ctxt format type_enc textual sym_tab phi =  | 
| 38014 | 452  | 
let  | 
453  | 
fun do_formula pos phi =  | 
|
| 54789 | 454  | 
(case phi of  | 
| 38014 | 455  | 
AQuant (_, [], phi) => do_formula pos phi  | 
| 42526 | 456  | 
| AQuant (q, (s, _) :: xs, phi') =>  | 
| 38014 | 457  | 
do_formula pos (AQuant (q, xs, phi'))  | 
| 42526 | 458  | 
(* FIXME: TFF *)  | 
| 57257 | 459  | 
#>> quantify_over_var textual (case q of AForall => forall_of | AExists => exists_of)  | 
460  | 
(repair_var_name textual s) dummyT  | 
|
| 38014 | 461  | 
| AConn (ANot, [phi']) => do_formula (not pos) phi' #>> s_not  | 
| 37991 | 462  | 
| AConn (c, [phi1, phi2]) =>  | 
| 38014 | 463  | 
do_formula (pos |> c = AImplies ? not) phi1  | 
464  | 
##>> do_formula pos phi2  | 
|
465  | 
#>> (case c of  | 
|
| 54811 | 466  | 
AAnd => s_conj  | 
467  | 
| AOr => s_disj  | 
|
468  | 
| AImplies => s_imp  | 
|
469  | 
| AIff => s_iff  | 
|
470  | 
| ANot => raise Fail "impossible connective")  | 
|
| 
57255
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
471  | 
| AAtom tm => term_of_atom ctxt format type_enc textual sym_tab pos tm  | 
| 54789 | 472  | 
| _ => raise ATP_FORMULA [phi])  | 
473  | 
in  | 
|
474  | 
repair_tvar_sorts (do_formula true phi Vartab.empty)  | 
|
475  | 
end  | 
|
| 37991 | 476  | 
|
| 54500 | 477  | 
val unprefix_fact_number = space_implode "_" o tl o space_explode "_"  | 
478  | 
||
| 57263 | 479  | 
fun resolve_fact facts s =  | 
| 54789 | 480  | 
(case try (unprefix fact_prefix) s of  | 
| 54500 | 481  | 
SOME s' =>  | 
482  | 
let val s' = s' |> unprefix_fact_number |> unascii_of in  | 
|
| 57263 | 483  | 
AList.lookup (op =) facts s' |> Option.map (pair s')  | 
| 54500 | 484  | 
end  | 
| 54789 | 485  | 
| NONE => NONE)  | 
| 54506 | 486  | 
|
| 57263 | 487  | 
fun resolve_conjecture s =  | 
| 54789 | 488  | 
(case try (unprefix conjecture_prefix) s of  | 
| 54500 | 489  | 
SOME s' => Int.fromString s'  | 
| 54789 | 490  | 
| NONE => NONE)  | 
| 54500 | 491  | 
|
| 57263 | 492  | 
fun resolve_facts facts = map_filter (resolve_fact facts)  | 
493  | 
val resolve_conjectures = map_filter resolve_conjecture  | 
|
| 54500 | 494  | 
|
495  | 
fun is_axiom_used_in_proof pred =  | 
|
496  | 
exists (fn ((_, ss), _, _, _, []) => exists pred ss | _ => false)  | 
|
497  | 
||
498  | 
val leo2_extcnf_equal_neg_rule = "extcnf_equal_neg"  | 
|
499  | 
||
| 57263 | 500  | 
fun add_fact ctxt facts ((_, ss), _, _, rule, deps) =  | 
| 
57707
 
0242e9578828
imported patch satallax_proof_support_Sledgehammer
 
fleury 
parents: 
57703 
diff
changeset
 | 
501  | 
(if member (op =) [agsyhol_core_rule, leo2_extcnf_equal_neg_rule] rule then  | 
| 
56104
 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 
blanchet 
parents: 
55285 
diff
changeset
 | 
502  | 
insert (op =) (short_thm_name ctxt ext, (Global, General))  | 
| 54500 | 503  | 
else  | 
504  | 
I)  | 
|
| 57263 | 505  | 
#> (if null deps then union (op =) (resolve_facts facts ss) else I)  | 
| 54500 | 506  | 
|
| 57263 | 507  | 
fun used_facts_in_atp_proof ctxt facts atp_proof =  | 
508  | 
if null atp_proof then facts else fold (add_fact ctxt facts) atp_proof []  | 
|
| 54500 | 509  | 
|
510  | 
fun used_facts_in_unsound_atp_proof _ _ [] = NONE  | 
|
| 57263 | 511  | 
| used_facts_in_unsound_atp_proof ctxt facts atp_proof =  | 
512  | 
let val used_facts = used_facts_in_atp_proof ctxt facts atp_proof in  | 
|
| 54500 | 513  | 
if forall (fn (_, (sc, _)) => sc = Global) used_facts andalso  | 
| 57263 | 514  | 
not (is_axiom_used_in_proof (is_some o resolve_conjecture) atp_proof) then  | 
| 54500 | 515  | 
SOME (map fst used_facts)  | 
516  | 
else  | 
|
517  | 
NONE  | 
|
518  | 
end  | 
|
519  | 
||
520  | 
val ascii_of_lam_fact_prefix = ascii_of lam_fact_prefix  | 
|
521  | 
||
522  | 
(* overapproximation (good enough) *)  | 
|
523  | 
fun is_lam_lifted s =  | 
|
524  | 
String.isPrefix fact_prefix s andalso  | 
|
525  | 
String.isSubstring ascii_of_lam_fact_prefix s  | 
|
526  | 
||
527  | 
val is_combinator_def = String.isPrefix (helper_prefix ^ combinator_prefix)  | 
|
528  | 
||
| 55257 | 529  | 
fun atp_proof_prefers_lifting atp_proof =  | 
530  | 
(is_axiom_used_in_proof is_combinator_def atp_proof,  | 
|
531  | 
is_axiom_used_in_proof is_lam_lifted atp_proof) = (false, true)  | 
|
| 54500 | 532  | 
|
533  | 
val is_typed_helper_name =  | 
|
534  | 
String.isPrefix helper_prefix andf String.isSuffix typed_helper_suffix  | 
|
535  | 
||
536  | 
fun is_typed_helper_used_in_atp_proof atp_proof =  | 
|
537  | 
is_axiom_used_in_proof is_typed_helper_name atp_proof  | 
|
538  | 
||
| 54772 | 539  | 
fun replace_one_dependency (old, new) dep = if is_same_atp_step dep old then new else [dep]  | 
540  | 
fun replace_dependencies_in_line old_new (name, role, t, rule, deps) =  | 
|
541  | 
(name, role, t, rule, fold (union (op =) o replace_one_dependency old_new) deps [])  | 
|
542  | 
||
| 54499 | 543  | 
fun repair_name "$true" = "c_True"  | 
544  | 
| repair_name "$false" = "c_False"  | 
|
545  | 
| repair_name "$$e" = tptp_equal (* seen in Vampire proofs *)  | 
|
546  | 
| repair_name s =  | 
|
547  | 
if is_tptp_equal s orelse  | 
|
548  | 
(* seen in Vampire proofs *)  | 
|
549  | 
(String.isPrefix "sQ" s andalso String.isSuffix "_eqProxy" s) then  | 
|
550  | 
tptp_equal  | 
|
551  | 
else  | 
|
552  | 
s  | 
|
553  | 
||
| 57699 | 554  | 
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
 | 
555  | 
|
| 57699 | 556  | 
fun infer_formulas_types ctxt =  | 
| 
57635
 
97adb86619a4
more robust handling of types for skolems (modeled as Frees)
 
blanchet 
parents: 
57547 
diff
changeset
 | 
557  | 
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
 | 
558  | 
#> Syntax.check_terms (Proof_Context.set_mode Proof_Context.mode_schematic ctxt)  | 
| 
 
97adb86619a4
more robust handling of types for skolems (modeled as Frees)
 
blanchet 
parents: 
57547 
diff
changeset
 | 
559  | 
#> map (set_var_index 0)  | 
| 54499 | 560  | 
|
561  | 
val combinator_table =  | 
|
562  | 
  [(@{const_name Meson.COMBI}, @{thm Meson.COMBI_def [abs_def]}),
 | 
|
563  | 
   (@{const_name Meson.COMBK}, @{thm Meson.COMBK_def [abs_def]}),
 | 
|
564  | 
   (@{const_name Meson.COMBB}, @{thm Meson.COMBB_def [abs_def]}),
 | 
|
565  | 
   (@{const_name Meson.COMBC}, @{thm Meson.COMBC_def [abs_def]}),
 | 
|
566  | 
   (@{const_name Meson.COMBS}, @{thm Meson.COMBS_def [abs_def]})]
 | 
|
567  | 
||
568  | 
fun uncombine_term thy =  | 
|
569  | 
let  | 
|
570  | 
fun aux (t1 $ t2) = betapply (pairself aux (t1, t2))  | 
|
571  | 
| aux (Abs (s, T, t')) = Abs (s, T, aux t')  | 
|
572  | 
| aux (t as Const (x as (s, _))) =  | 
|
573  | 
(case AList.lookup (op =) combinator_table s of  | 
|
| 54756 | 574  | 
SOME thm => thm |> prop_of |> specialize_type thy x |> Logic.dest_equals |> snd  | 
575  | 
| NONE => t)  | 
|
| 54499 | 576  | 
| aux t = t  | 
577  | 
in aux end  | 
|
578  | 
||
579  | 
fun unlift_term lifted =  | 
|
580  | 
map_aterms (fn t as Const (s, _) =>  | 
|
581  | 
if String.isPrefix lam_lifted_prefix s then  | 
|
| 54756 | 582  | 
(* FIXME: do something about the types *)  | 
583  | 
(case AList.lookup (op =) lifted s of  | 
|
584  | 
SOME t => unlift_term lifted t  | 
|
585  | 
| NONE => t)  | 
|
| 54499 | 586  | 
else  | 
587  | 
t  | 
|
588  | 
| t => t)  | 
|
589  | 
||
| 57256 | 590  | 
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
 | 
591  | 
| 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
 | 
592  | 
let  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
593  | 
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
 | 
594  | 
val t = u  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
595  | 
|> prop_of_atp ctxt format type_enc true sym_tab  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
596  | 
|> uncombine_term thy  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
597  | 
|> unlift_term lifted  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
598  | 
in  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
599  | 
SOME (name, role, t, rule, deps)  | 
| 
 
488046fdda59
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
 
fleury 
parents: 
57199 
diff
changeset
 | 
600  | 
end  | 
| 54499 | 601  | 
|
602  | 
val waldmeister_conjecture_num = "1.0.0.0"  | 
|
603  | 
||
| 54756 | 604  | 
fun repair_waldmeister_endgame proof =  | 
| 54499 | 605  | 
let  | 
| 56854 | 606  | 
    fun repair_tail (name, _, @{const Trueprop} $ t, rule, deps) =
 | 
607  | 
      (name, Negated_Conjecture, @{const Trueprop} $ s_not t, rule, deps)
 | 
|
| 54756 | 608  | 
fun repair_body [] = []  | 
609  | 
| repair_body ((line as ((num, _), _, _, _, _)) :: lines) =  | 
|
610  | 
if num = waldmeister_conjecture_num then map repair_tail (line :: lines)  | 
|
611  | 
else line :: repair_body lines  | 
|
612  | 
in  | 
|
613  | 
repair_body proof  | 
|
614  | 
end  | 
|
| 54499 | 615  | 
|
| 
57635
 
97adb86619a4
more robust handling of types for skolems (modeled as Frees)
 
blanchet 
parents: 
57547 
diff
changeset
 | 
616  | 
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
 | 
617  | 
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
 | 
618  | 
|
| 
57258
 
67d85a8aa6cc
Moving the remote prefix deleting on Sledgehammer's side
 
fleury 
parents: 
57257 
diff
changeset
 | 
619  | 
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
 | 
620  | 
nasty_atp_proof pool  | 
| 54499 | 621  | 
#> 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
 | 
622  | 
#> map_filter (termify_line ctxt format type_enc lifted sym_tab)  | 
| 57699 | 623  | 
#> 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
 | 
624  | 
#> local_prover = waldmeisterN ? repair_waldmeister_endgame  | 
| 54499 | 625  | 
|
| 
55192
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
626  | 
fun take_distinct_vars seen ((t as Var _) :: ts) =  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
627  | 
if member (op aconv) seen t then rev seen else take_distinct_vars (t :: seen) ts  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
628  | 
| take_distinct_vars seen _ = rev seen  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
629  | 
|
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
630  | 
fun unskolemize_term skos t =  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
631  | 
let  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
632  | 
val is_sko = member (op =) skos  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
633  | 
|
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
634  | 
fun find_args args (t $ u) = find_args (u :: args) t #> find_args [] u  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
635  | 
| find_args _ (Abs (_, _, t)) = find_args [] t  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
636  | 
| find_args args (Free (s, _)) =  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
637  | 
if is_sko s then  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
638  | 
let val new = take_distinct_vars [] args in  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
639  | 
(fn [] => new | old => if length new < length old then new else old)  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
640  | 
end  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
641  | 
else  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
642  | 
I  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
643  | 
| find_args _ _ = I  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
644  | 
|
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
645  | 
val alls = find_args [] t []  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
646  | 
val num_alls = length alls  | 
| 55195 | 647  | 
|
648  | 
fun fix_skos args (t $ u) = fix_skos (fix_skos [] u :: args) t  | 
|
649  | 
| fix_skos args (t as Free (s, T)) =  | 
|
650  | 
if is_sko s then list_comb (Free (s, funpow num_alls body_type T), drop num_alls args)  | 
|
651  | 
else list_comb (t, args)  | 
|
652  | 
| fix_skos [] (Abs (s, T, t)) = Abs (s, T, fix_skos [] t)  | 
|
653  | 
| fix_skos [] t = t  | 
|
654  | 
| fix_skos args t = list_comb (fix_skos [] t, args)  | 
|
655  | 
||
656  | 
val t' = fix_skos [] t  | 
|
| 
55192
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
657  | 
|
| 55195 | 658  | 
fun add_sko (t as Free (s, _)) = is_sko s ? insert (op aconv) t  | 
659  | 
| add_sko _ = I  | 
|
| 
55192
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
660  | 
|
| 55195 | 661  | 
val exs = Term.fold_aterms add_sko t' []  | 
662  | 
in  | 
|
663  | 
t'  | 
|
664  | 
|> HOLogic.dest_Trueprop  | 
|
665  | 
|> fold exists_of exs |> Term.map_abs_vars (K Name.uu)  | 
|
666  | 
|> fold_rev forall_of alls  | 
|
667  | 
|> HOLogic.mk_Trueprop  | 
|
| 
55192
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
668  | 
end  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
669  | 
|
| 54772 | 670  | 
fun introduce_spass_skolem [] = []  | 
671  | 
| introduce_spass_skolem (proof as (_, _, _, rule1, _) :: _) =  | 
|
672  | 
if rule1 = spass_input_rule then  | 
|
673  | 
let  | 
|
674  | 
fun add_sko (Free (s, _)) = String.isPrefix spass_skolem_prefix s ? insert (op =) s  | 
|
675  | 
| add_sko _ = I  | 
|
676  | 
||
677  | 
(* union-find would be faster *)  | 
|
| 54799 | 678  | 
fun add_cycle [] = I  | 
679  | 
| add_cycle ss =  | 
|
| 54772 | 680  | 
fold (fn s => Graph.default_node (s, ())) ss  | 
681  | 
#> fold Graph.add_edge (ss ~~ tl ss @ [hd ss])  | 
|
682  | 
||
683  | 
val (input_steps, other_steps) = List.partition (null o #5) proof  | 
|
684  | 
||
685  | 
val skoss = map (fn (_, _, t, _, _) => Term.fold_aterms add_sko t []) input_steps  | 
|
686  | 
val skoss_input_steps = filter_out (null o fst) (skoss ~~ input_steps)  | 
|
| 54799 | 687  | 
val groups = Graph.strong_conn (fold add_cycle skoss Graph.empty)  | 
| 54772 | 688  | 
|
689  | 
fun step_name_of_group skos = (implode skos, [])  | 
|
690  | 
fun in_group group = member (op =) group o hd  | 
|
691  | 
fun group_of sko = the (find_first (fn group => in_group group sko) groups)  | 
|
692  | 
||
| 
55192
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
693  | 
fun new_steps (skoss_steps : (string list * (term, 'a) atp_step) list) group =  | 
| 54772 | 694  | 
let  | 
| 
55192
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
695  | 
val name = step_name_of_group group  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
696  | 
val name0 = name |>> prefix "0"  | 
| 54772 | 697  | 
val t =  | 
698  | 
skoss_steps  | 
|
699  | 
|> map (snd #> #3 #> HOLogic.dest_Trueprop)  | 
|
700  | 
|> Library.foldr1 s_conj  | 
|
701  | 
|> HOLogic.mk_Trueprop  | 
|
| 
55192
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
702  | 
val skos = fold (union (op =) o fst) skoss_steps []  | 
| 54772 | 703  | 
val deps = map (snd #> #1) skoss_steps  | 
704  | 
in  | 
|
| 55195 | 705  | 
[(name0, Unknown, unskolemize_term skos t, spass_pre_skolemize_rule, deps),  | 
706  | 
(name, Unknown, t, spass_skolemize_rule, [name0])]  | 
|
| 54772 | 707  | 
end  | 
708  | 
||
709  | 
val sko_steps =  | 
|
| 
55192
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
710  | 
maps (fn group => new_steps (filter (in_group group o fst) skoss_input_steps) group)  | 
| 
 
b75b52c7cf94
unskolemize SPASS formula to ensure that the variables are in the right order for 'metis's skolemizer
 
blanchet 
parents: 
55185 
diff
changeset
 | 
711  | 
groups  | 
| 54772 | 712  | 
|
713  | 
val old_news =  | 
|
714  | 
map (fn (skos, (name, _, _, _, _)) => (name, [step_name_of_group (group_of skos)]))  | 
|
715  | 
skoss_input_steps  | 
|
716  | 
val repair_deps = fold replace_dependencies_in_line old_news  | 
|
717  | 
in  | 
|
718  | 
input_steps @ sko_steps @ map repair_deps other_steps  | 
|
719  | 
end  | 
|
720  | 
else  | 
|
721  | 
proof  | 
|
722  | 
||
| 57263 | 723  | 
fun factify_atp_proof facts hyp_ts concl_t atp_proof =  | 
| 54505 | 724  | 
let  | 
| 54799 | 725  | 
fun factify_step ((num, ss), _, t, rule, deps) =  | 
| 54505 | 726  | 
let  | 
727  | 
val (ss', role', t') =  | 
|
| 57263 | 728  | 
(case resolve_conjectures ss of  | 
| 54505 | 729  | 
[j] =>  | 
730  | 
if j = length hyp_ts then ([], Conjecture, concl_t) else ([], Hypothesis, nth hyp_ts j)  | 
|
| 
55185
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
731  | 
| _ =>  | 
| 57263 | 732  | 
(case resolve_facts facts ss of  | 
| 
55185
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
733  | 
[] => (ss, Plain, t)  | 
| 
 
a0bd8d6414e6
centralized & repaired handling of bound variables in intermediate data structure (viva de Bruijn)
 
blanchet 
parents: 
54822 
diff
changeset
 | 
734  | 
| facts => (map fst facts, Axiom, t)))  | 
| 54505 | 735  | 
in  | 
736  | 
((num, ss'), role', t', rule, deps)  | 
|
737  | 
end  | 
|
738  | 
||
739  | 
val atp_proof = map factify_step atp_proof  | 
|
740  | 
val names = map #1 atp_proof  | 
|
741  | 
||
742  | 
fun repair_dep (num, ss) = (num, the_default ss (AList.lookup (op =) names num))  | 
|
743  | 
fun repair_deps (name, role, t, rule, deps) = (name, role, t, rule, map repair_dep deps)  | 
|
| 54772 | 744  | 
in  | 
745  | 
map repair_deps atp_proof  | 
|
746  | 
end  | 
|
| 54505 | 747  | 
|
| 31038 | 748  | 
end;  |