author | wenzelm |
Tue, 27 Oct 2009 17:34:00 +0100 | |
changeset 33243 | 17014b1b9353 |
parent 33227 | 83322d668601 |
child 33305 | a103fa7c19cc |
permissions | -rw-r--r-- |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
1 |
(* Title: HOL/Tools/metis_tools.ML |
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
2 |
Author: Kong W. Susanto and Lawrence C. Paulson, CU Computer Laboratory |
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
3 |
Copyright Cambridge University 2007 |
23447 | 4 |
|
29266 | 5 |
HOL setup for the Metis prover. |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
6 |
*) |
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
7 |
|
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
8 |
signature METIS_TOOLS = |
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
9 |
sig |
32955 | 10 |
val trace: bool Unsynchronized.ref |
24309
01f3e1a43c24
turned type_lits into configuration option (with attribute);
wenzelm
parents:
24300
diff
changeset
|
11 |
val type_lits: bool Config.T |
24319 | 12 |
val metis_tac: Proof.context -> thm list -> int -> tactic |
13 |
val metisF_tac: Proof.context -> thm list -> int -> tactic |
|
32532
a0a54a51b15b
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
paulson
parents:
32530
diff
changeset
|
14 |
val metisFT_tac: Proof.context -> thm list -> int -> tactic |
24319 | 15 |
val setup: theory -> theory |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
16 |
end |
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
17 |
|
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
18 |
structure MetisTools: METIS_TOOLS = |
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
19 |
struct |
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
20 |
|
32956 | 21 |
val trace = Unsynchronized.ref false; |
22 |
fun trace_msg msg = if ! trace then tracing (msg ()) else (); |
|
32955 | 23 |
|
32956 | 24 |
val (type_lits, type_lits_setup) = Attrib.config_bool "metis_type_lits" true; |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
25 |
|
32956 | 26 |
datatype mode = FO | HO | FT (*first-order, higher-order, fully-typed*) |
32532
a0a54a51b15b
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
paulson
parents:
32530
diff
changeset
|
27 |
|
32956 | 28 |
(* ------------------------------------------------------------------------- *) |
29 |
(* Useful Theorems *) |
|
30 |
(* ------------------------------------------------------------------------- *) |
|
31 |
val EXCLUDED_MIDDLE = rotate_prems 1 (read_instantiate @{context} [(("R", 0), "False")] notE); |
|
32 |
val REFL_THM = incr_indexes 2 (Meson.make_meta_clause refl); (*Rename from 0,1*) |
|
33 |
val subst_em = zero_var_indexes (subst RS EXCLUDED_MIDDLE); |
|
34 |
val ssubst_em = read_instantiate @{context} [(("t", 0), "?s"), (("s", 0), "?t")] (sym RS subst_em); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
35 |
|
32956 | 36 |
(* ------------------------------------------------------------------------- *) |
37 |
(* Useful Functions *) |
|
38 |
(* ------------------------------------------------------------------------- *) |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
39 |
|
32956 | 40 |
(* match untyped terms*) |
41 |
fun untyped_aconv (Const(a,_)) (Const(b,_)) = (a=b) |
|
42 |
| untyped_aconv (Free(a,_)) (Free(b,_)) = (a=b) |
|
43 |
| untyped_aconv (Var((a,_),_)) (Var((b,_),_)) = (a=b) (*the index is ignored!*) |
|
44 |
| untyped_aconv (Bound i) (Bound j) = (i=j) |
|
45 |
| untyped_aconv (Abs(a,_,t)) (Abs(b,_,u)) = (a=b) andalso untyped_aconv t u |
|
46 |
| untyped_aconv (t1$t2) (u1$u2) = untyped_aconv t1 u1 andalso untyped_aconv t2 u2 |
|
47 |
| untyped_aconv _ _ = false; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
48 |
|
32956 | 49 |
(* Finding the relative location of an untyped term within a list of terms *) |
50 |
fun get_index lit = |
|
51 |
let val lit = Envir.eta_contract lit |
|
52 |
fun get n [] = raise Empty |
|
53 |
| get n (x::xs) = if untyped_aconv lit (Envir.eta_contract (HOLogic.dest_Trueprop x)) |
|
54 |
then n else get (n+1) xs |
|
55 |
in get 1 end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
56 |
|
32956 | 57 |
(* ------------------------------------------------------------------------- *) |
58 |
(* HOL to FOL (Isabelle to Metis) *) |
|
59 |
(* ------------------------------------------------------------------------- *) |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
60 |
|
32956 | 61 |
fun fn_isa_to_met "equal" = "=" |
62 |
| fn_isa_to_met x = x; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
63 |
|
32956 | 64 |
fun metis_lit b c args = (b, (c, args)); |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
65 |
|
32956 | 66 |
fun hol_type_to_fol (ResClause.AtomV x) = Metis.Term.Var x |
67 |
| hol_type_to_fol (ResClause.AtomF x) = Metis.Term.Fn(x,[]) |
|
68 |
| hol_type_to_fol (ResClause.Comp(tc,tps)) = Metis.Term.Fn(tc, map hol_type_to_fol tps); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
69 |
|
32956 | 70 |
(*These two functions insert type literals before the real literals. That is the |
71 |
opposite order from TPTP linkup, but maybe OK.*) |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
72 |
|
32956 | 73 |
fun hol_term_to_fol_FO tm = |
74 |
case ResHolClause.strip_comb tm of |
|
75 |
(ResHolClause.CombConst(c,_,tys), tms) => |
|
76 |
let val tyargs = map hol_type_to_fol tys |
|
77 |
val args = map hol_term_to_fol_FO tms |
|
78 |
in Metis.Term.Fn (c, tyargs @ args) end |
|
79 |
| (ResHolClause.CombVar(v,_), []) => Metis.Term.Var v |
|
80 |
| _ => error "hol_term_to_fol_FO"; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
81 |
|
32994 | 82 |
fun hol_term_to_fol_HO (ResHolClause.CombVar (a, _)) = Metis.Term.Var a |
83 |
| hol_term_to_fol_HO (ResHolClause.CombConst (a, _, tylist)) = |
|
84 |
Metis.Term.Fn (fn_isa_to_met a, map hol_type_to_fol tylist) |
|
85 |
| hol_term_to_fol_HO (ResHolClause.CombApp (tm1, tm2)) = |
|
86 |
Metis.Term.Fn (".", map hol_term_to_fol_HO [tm1, tm2]); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
87 |
|
32956 | 88 |
(*The fully-typed translation, to avoid type errors*) |
89 |
fun wrap_type (tm, ty) = Metis.Term.Fn("ti", [tm, hol_type_to_fol ty]); |
|
90 |
||
91 |
fun hol_term_to_fol_FT (ResHolClause.CombVar(a, ty)) = |
|
92 |
wrap_type (Metis.Term.Var a, ty) |
|
93 |
| hol_term_to_fol_FT (ResHolClause.CombConst(a, ty, _)) = |
|
94 |
wrap_type (Metis.Term.Fn(fn_isa_to_met a, []), ty) |
|
95 |
| hol_term_to_fol_FT (tm as ResHolClause.CombApp(tm1,tm2)) = |
|
96 |
wrap_type (Metis.Term.Fn(".", map hol_term_to_fol_FT [tm1,tm2]), |
|
97 |
ResHolClause.type_of_combterm tm); |
|
32532
a0a54a51b15b
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
paulson
parents:
32530
diff
changeset
|
98 |
|
32956 | 99 |
fun hol_literal_to_fol FO (ResHolClause.Literal (pol, tm)) = |
100 |
let val (ResHolClause.CombConst(p,_,tys), tms) = ResHolClause.strip_comb tm |
|
101 |
val tylits = if p = "equal" then [] else map hol_type_to_fol tys |
|
102 |
val lits = map hol_term_to_fol_FO tms |
|
103 |
in metis_lit pol (fn_isa_to_met p) (tylits @ lits) end |
|
104 |
| hol_literal_to_fol HO (ResHolClause.Literal (pol, tm)) = |
|
105 |
(case ResHolClause.strip_comb tm of |
|
106 |
(ResHolClause.CombConst("equal",_,_), tms) => |
|
107 |
metis_lit pol "=" (map hol_term_to_fol_HO tms) |
|
108 |
| _ => metis_lit pol "{}" [hol_term_to_fol_HO tm]) (*hBOOL*) |
|
109 |
| hol_literal_to_fol FT (ResHolClause.Literal (pol, tm)) = |
|
110 |
(case ResHolClause.strip_comb tm of |
|
111 |
(ResHolClause.CombConst("equal",_,_), tms) => |
|
112 |
metis_lit pol "=" (map hol_term_to_fol_FT tms) |
|
113 |
| _ => metis_lit pol "{}" [hol_term_to_fol_FT tm]) (*hBOOL*); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
114 |
|
32956 | 115 |
fun literals_of_hol_thm thy mode t = |
116 |
let val (lits, types_sorts) = ResHolClause.literals_of_term thy t |
|
117 |
in (map (hol_literal_to_fol mode) lits, types_sorts) end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
118 |
|
32956 | 119 |
(*Sign should be "true" for conjecture type constraints, "false" for type lits in clauses.*) |
120 |
fun metis_of_typeLit pos (ResClause.LTVar (s,x)) = metis_lit pos s [Metis.Term.Var x] |
|
121 |
| metis_of_typeLit pos (ResClause.LTFree (s,x)) = metis_lit pos s [Metis.Term.Fn(x,[])]; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
122 |
|
32994 | 123 |
fun default_sort _ (TVar _) = false |
33035 | 124 |
| default_sort ctxt (TFree (x, s)) = (s = the_default [] (Variable.def_sort ctxt (x, ~1))); |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
125 |
|
32956 | 126 |
fun metis_of_tfree tf = |
127 |
Metis.Thm.axiom (Metis.LiteralSet.singleton (metis_of_typeLit true tf)); |
|
24937
340523598914
context-based treatment of generalization; also handling TFrees in axiom clauses
paulson
parents:
24920
diff
changeset
|
128 |
|
32956 | 129 |
fun hol_thm_to_fol is_conjecture ctxt mode th = |
130 |
let val thy = ProofContext.theory_of ctxt |
|
131 |
val (mlits, types_sorts) = |
|
132 |
(literals_of_hol_thm thy mode o HOLogic.dest_Trueprop o prop_of) th |
|
133 |
in |
|
134 |
if is_conjecture then |
|
135 |
(Metis.Thm.axiom (Metis.LiteralSet.fromList mlits), ResClause.add_typs types_sorts) |
|
136 |
else |
|
137 |
let val tylits = ResClause.add_typs |
|
138 |
(filter (not o default_sort ctxt) types_sorts) |
|
139 |
val mtylits = if Config.get ctxt type_lits |
|
140 |
then map (metis_of_typeLit false) tylits else [] |
|
141 |
in |
|
142 |
(Metis.Thm.axiom (Metis.LiteralSet.fromList(mtylits @ mlits)), []) |
|
143 |
end |
|
144 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
145 |
|
32956 | 146 |
(* ARITY CLAUSE *) |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
147 |
|
32956 | 148 |
fun m_arity_cls (ResClause.TConsLit (c,t,args)) = |
149 |
metis_lit true (ResClause.make_type_class c) [Metis.Term.Fn(t, map Metis.Term.Var args)] |
|
150 |
| m_arity_cls (ResClause.TVarLit (c,str)) = |
|
151 |
metis_lit false (ResClause.make_type_class c) [Metis.Term.Var str]; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
152 |
|
32956 | 153 |
(*TrueI is returned as the Isabelle counterpart because there isn't any.*) |
154 |
fun arity_cls (ResClause.ArityClause{conclLit,premLits,...}) = |
|
155 |
(TrueI, |
|
156 |
Metis.Thm.axiom (Metis.LiteralSet.fromList (map m_arity_cls (conclLit :: premLits)))); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
157 |
|
32956 | 158 |
(* CLASSREL CLAUSE *) |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
159 |
|
32956 | 160 |
fun m_classrel_cls subclass superclass = |
161 |
[metis_lit false subclass [Metis.Term.Var "T"], metis_lit true superclass [Metis.Term.Var "T"]]; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
162 |
|
32994 | 163 |
fun classrel_cls (ResClause.ClassrelClause {subclass, superclass, ...}) = |
32956 | 164 |
(TrueI, Metis.Thm.axiom (Metis.LiteralSet.fromList (m_classrel_cls subclass superclass))); |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
165 |
|
32956 | 166 |
(* ------------------------------------------------------------------------- *) |
167 |
(* FOL to HOL (Metis to Isabelle) *) |
|
168 |
(* ------------------------------------------------------------------------- *) |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
169 |
|
32956 | 170 |
datatype term_or_type = Term of Term.term | Type of Term.typ; |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
171 |
|
32956 | 172 |
fun terms_of [] = [] |
173 |
| terms_of (Term t :: tts) = t :: terms_of tts |
|
174 |
| terms_of (Type _ :: tts) = terms_of tts; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
175 |
|
32956 | 176 |
fun types_of [] = [] |
32994 | 177 |
| types_of (Term (Term.Var ((a,idx), _)) :: tts) = |
32956 | 178 |
if String.isPrefix "_" a then |
179 |
(*Variable generated by Metis, which might have been a type variable.*) |
|
32994 | 180 |
TVar (("'" ^ a, idx), HOLogic.typeS) :: types_of tts |
32956 | 181 |
else types_of tts |
182 |
| types_of (Term _ :: tts) = types_of tts |
|
183 |
| types_of (Type T :: tts) = T :: types_of tts; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
184 |
|
32956 | 185 |
fun apply_list rator nargs rands = |
186 |
let val trands = terms_of rands |
|
187 |
in if length trands = nargs then Term (list_comb(rator, trands)) |
|
188 |
else error |
|
189 |
("apply_list: wrong number of arguments: " ^ Syntax.string_of_term_global Pure.thy rator ^ |
|
190 |
" expected " ^ Int.toString nargs ^ |
|
191 |
" received " ^ commas (map (Syntax.string_of_term_global Pure.thy) trands)) |
|
192 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
193 |
|
24500 | 194 |
fun infer_types ctxt = |
195 |
Syntax.check_terms (ProofContext.set_mode ProofContext.mode_pattern ctxt); |
|
25713 | 196 |
|
32956 | 197 |
(*We use 1 rather than 0 because variable references in clauses may otherwise conflict |
198 |
with variable constraints in the goal...at least, type inference often fails otherwise. |
|
199 |
SEE ALSO axiom_inf below.*) |
|
200 |
fun mk_var (w,T) = Term.Var((w,1), T); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
201 |
|
32956 | 202 |
(*include the default sort, if available*) |
203 |
fun mk_tfree ctxt w = |
|
204 |
let val ww = "'" ^ w |
|
33035 | 205 |
in TFree(ww, the_default HOLogic.typeS (Variable.def_sort ctxt (ww, ~1))) end; |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
206 |
|
32956 | 207 |
(*Remove the "apply" operator from an HO term*) |
208 |
fun strip_happ args (Metis.Term.Fn(".",[t,u])) = strip_happ (u::args) t |
|
209 |
| strip_happ args x = (x, args); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
210 |
|
32994 | 211 |
fun fol_type_to_isa _ (Metis.Term.Var v) = |
33227 | 212 |
(case ResReconstruct.strip_prefix ResClause.tvar_prefix v of |
213 |
SOME w => ResReconstruct.make_tvar w |
|
214 |
| NONE => ResReconstruct.make_tvar v) |
|
32956 | 215 |
| fol_type_to_isa ctxt (Metis.Term.Fn(x, tys)) = |
33227 | 216 |
(case ResReconstruct.strip_prefix ResClause.tconst_prefix x of |
217 |
SOME tc => Term.Type (ResReconstruct.invert_type_const tc, map (fol_type_to_isa ctxt) tys) |
|
32956 | 218 |
| NONE => |
33227 | 219 |
case ResReconstruct.strip_prefix ResClause.tfree_prefix x of |
32956 | 220 |
SOME tf => mk_tfree ctxt tf |
221 |
| NONE => error ("fol_type_to_isa: " ^ x)); |
|
32532
a0a54a51b15b
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
paulson
parents:
32530
diff
changeset
|
222 |
|
32956 | 223 |
(*Maps metis terms to isabelle terms*) |
224 |
fun fol_term_to_hol_RAW ctxt fol_tm = |
|
225 |
let val thy = ProofContext.theory_of ctxt |
|
226 |
val _ = trace_msg (fn () => "fol_term_to_hol: " ^ Metis.Term.toString fol_tm) |
|
227 |
fun tm_to_tt (Metis.Term.Var v) = |
|
33227 | 228 |
(case ResReconstruct.strip_prefix ResClause.tvar_prefix v of |
229 |
SOME w => Type (ResReconstruct.make_tvar w) |
|
32956 | 230 |
| NONE => |
33227 | 231 |
case ResReconstruct.strip_prefix ResClause.schematic_var_prefix v of |
32956 | 232 |
SOME w => Term (mk_var (w, HOLogic.typeT)) |
233 |
| NONE => Term (mk_var (v, HOLogic.typeT)) ) |
|
234 |
(*Var from Metis with a name like _nnn; possibly a type variable*) |
|
235 |
| tm_to_tt (Metis.Term.Fn ("{}", [arg])) = tm_to_tt arg (*hBOOL*) |
|
236 |
| tm_to_tt (t as Metis.Term.Fn (".",_)) = |
|
237 |
let val (rator,rands) = strip_happ [] t |
|
238 |
in case rator of |
|
239 |
Metis.Term.Fn(fname,ts) => applic_to_tt (fname, ts @ rands) |
|
240 |
| _ => case tm_to_tt rator of |
|
241 |
Term t => Term (list_comb(t, terms_of (map tm_to_tt rands))) |
|
242 |
| _ => error "tm_to_tt: HO application" |
|
243 |
end |
|
244 |
| tm_to_tt (Metis.Term.Fn (fname, args)) = applic_to_tt (fname,args) |
|
245 |
and applic_to_tt ("=",ts) = |
|
246 |
Term (list_comb(Const ("op =", HOLogic.typeT), terms_of (map tm_to_tt ts))) |
|
247 |
| applic_to_tt (a,ts) = |
|
33227 | 248 |
case ResReconstruct.strip_prefix ResClause.const_prefix a of |
32956 | 249 |
SOME b => |
33227 | 250 |
let val c = ResReconstruct.invert_const b |
251 |
val ntypes = ResReconstruct.num_typargs thy c |
|
32956 | 252 |
val nterms = length ts - ntypes |
253 |
val tts = map tm_to_tt ts |
|
254 |
val tys = types_of (List.take(tts,ntypes)) |
|
33227 | 255 |
val ntyargs = ResReconstruct.num_typargs thy c |
32956 | 256 |
in if length tys = ntyargs then |
257 |
apply_list (Const (c, dummyT)) nterms (List.drop(tts,ntypes)) |
|
258 |
else error ("Constant " ^ c ^ " expects " ^ Int.toString ntyargs ^ |
|
259 |
" but gets " ^ Int.toString (length tys) ^ |
|
260 |
" type arguments\n" ^ |
|
261 |
cat_lines (map (Syntax.string_of_typ ctxt) tys) ^ |
|
262 |
" the terms are \n" ^ |
|
263 |
cat_lines (map (Syntax.string_of_term ctxt) (terms_of tts))) |
|
264 |
end |
|
265 |
| NONE => (*Not a constant. Is it a type constructor?*) |
|
33227 | 266 |
case ResReconstruct.strip_prefix ResClause.tconst_prefix a of |
267 |
SOME b => |
|
268 |
Type (Term.Type (ResReconstruct.invert_type_const b, types_of (map tm_to_tt ts))) |
|
32956 | 269 |
| NONE => (*Maybe a TFree. Should then check that ts=[].*) |
33227 | 270 |
case ResReconstruct.strip_prefix ResClause.tfree_prefix a of |
32956 | 271 |
SOME b => Type (mk_tfree ctxt b) |
272 |
| NONE => (*a fixed variable? They are Skolem functions.*) |
|
33227 | 273 |
case ResReconstruct.strip_prefix ResClause.fixed_var_prefix a of |
32956 | 274 |
SOME b => |
275 |
let val opr = Term.Free(b, HOLogic.typeT) |
|
276 |
in apply_list opr (length ts) (map tm_to_tt ts) end |
|
277 |
| NONE => error ("unexpected metis function: " ^ a) |
|
278 |
in case tm_to_tt fol_tm of Term t => t | _ => error "fol_tm_to_tt: Term expected" end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
279 |
|
32956 | 280 |
(*Maps fully-typed metis terms to isabelle terms*) |
281 |
fun fol_term_to_hol_FT ctxt fol_tm = |
|
282 |
let val _ = trace_msg (fn () => "fol_term_to_hol_FT: " ^ Metis.Term.toString fol_tm) |
|
32994 | 283 |
fun cvt (Metis.Term.Fn ("ti", [Metis.Term.Var v, _])) = |
33227 | 284 |
(case ResReconstruct.strip_prefix ResClause.schematic_var_prefix v of |
32956 | 285 |
SOME w => mk_var(w, dummyT) |
286 |
| NONE => mk_var(v, dummyT)) |
|
32994 | 287 |
| cvt (Metis.Term.Fn ("ti", [Metis.Term.Fn ("=",[]), _])) = |
32956 | 288 |
Const ("op =", HOLogic.typeT) |
289 |
| cvt (Metis.Term.Fn ("ti", [Metis.Term.Fn (x,[]), ty])) = |
|
33227 | 290 |
(case ResReconstruct.strip_prefix ResClause.const_prefix x of |
291 |
SOME c => Const (ResReconstruct.invert_const c, dummyT) |
|
32956 | 292 |
| NONE => (*Not a constant. Is it a fixed variable??*) |
33227 | 293 |
case ResReconstruct.strip_prefix ResClause.fixed_var_prefix x of |
32956 | 294 |
SOME v => Free (v, fol_type_to_isa ctxt ty) |
295 |
| NONE => error ("fol_term_to_hol_FT bad constant: " ^ x)) |
|
296 |
| cvt (Metis.Term.Fn ("ti", [Metis.Term.Fn (".",[tm1,tm2]), _])) = |
|
297 |
cvt tm1 $ cvt tm2 |
|
298 |
| cvt (Metis.Term.Fn (".",[tm1,tm2])) = (*untyped application*) |
|
299 |
cvt tm1 $ cvt tm2 |
|
300 |
| cvt (Metis.Term.Fn ("{}", [arg])) = cvt arg (*hBOOL*) |
|
301 |
| cvt (Metis.Term.Fn ("=", [tm1,tm2])) = |
|
302 |
list_comb(Const ("op =", HOLogic.typeT), map cvt [tm1,tm2]) |
|
303 |
| cvt (t as Metis.Term.Fn (x, [])) = |
|
33227 | 304 |
(case ResReconstruct.strip_prefix ResClause.const_prefix x of |
305 |
SOME c => Const (ResReconstruct.invert_const c, dummyT) |
|
32956 | 306 |
| NONE => (*Not a constant. Is it a fixed variable??*) |
33227 | 307 |
case ResReconstruct.strip_prefix ResClause.fixed_var_prefix x of |
32956 | 308 |
SOME v => Free (v, dummyT) |
33227 | 309 |
| NONE => (trace_msg (fn () => "fol_term_to_hol_FT bad const: " ^ x); |
310 |
fol_term_to_hol_RAW ctxt t)) |
|
311 |
| cvt t = (trace_msg (fn () => "fol_term_to_hol_FT bad term: " ^ Metis.Term.toString t); |
|
312 |
fol_term_to_hol_RAW ctxt t) |
|
32956 | 313 |
in cvt fol_tm end; |
32532
a0a54a51b15b
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
paulson
parents:
32530
diff
changeset
|
314 |
|
32956 | 315 |
fun fol_term_to_hol ctxt FO = fol_term_to_hol_RAW ctxt |
316 |
| fol_term_to_hol ctxt HO = fol_term_to_hol_RAW ctxt |
|
317 |
| fol_term_to_hol ctxt FT = fol_term_to_hol_FT ctxt; |
|
32532
a0a54a51b15b
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
paulson
parents:
32530
diff
changeset
|
318 |
|
32956 | 319 |
fun fol_terms_to_hol ctxt mode fol_tms = |
320 |
let val ts = map (fol_term_to_hol ctxt mode) fol_tms |
|
321 |
val _ = trace_msg (fn () => " calling type inference:") |
|
322 |
val _ = app (fn t => trace_msg (fn () => Syntax.string_of_term ctxt t)) ts |
|
323 |
val ts' = infer_types ctxt ts; |
|
324 |
val _ = app (fn t => trace_msg |
|
325 |
(fn () => " final term: " ^ Syntax.string_of_term ctxt t ^ |
|
326 |
" of type " ^ Syntax.string_of_typ ctxt (type_of t))) |
|
327 |
ts' |
|
328 |
in ts' end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
329 |
|
32956 | 330 |
fun mk_not (Const ("Not", _) $ b) = b |
331 |
| mk_not b = HOLogic.mk_not b; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
332 |
|
32956 | 333 |
val metis_eq = Metis.Term.Fn ("=", []); |
32532
a0a54a51b15b
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
paulson
parents:
32530
diff
changeset
|
334 |
|
32956 | 335 |
(* ------------------------------------------------------------------------- *) |
336 |
(* FOL step Inference Rules *) |
|
337 |
(* ------------------------------------------------------------------------- *) |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
338 |
|
32956 | 339 |
(*for debugging only*) |
340 |
fun print_thpair (fth,th) = |
|
341 |
(trace_msg (fn () => "============================================="); |
|
342 |
trace_msg (fn () => "Metis: " ^ Metis.Thm.toString fth); |
|
343 |
trace_msg (fn () => "Isabelle: " ^ Display.string_of_thm_without_context th)); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
344 |
|
32956 | 345 |
fun lookth thpairs (fth : Metis.Thm.thm) = |
33035 | 346 |
the (AList.lookup (uncurry Metis.Thm.equal) thpairs fth) |
32956 | 347 |
handle Option => error ("Failed to find a Metis theorem " ^ Metis.Thm.toString fth); |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
348 |
|
32956 | 349 |
fun is_TrueI th = Thm.eq_thm(TrueI,th); |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
350 |
|
32956 | 351 |
fun cterm_incr_types thy idx = cterm_of thy o (map_types (Logic.incr_tvar idx)); |
24974 | 352 |
|
32956 | 353 |
fun inst_excluded_middle thy i_atm = |
354 |
let val th = EXCLUDED_MIDDLE |
|
355 |
val [vx] = Term.add_vars (prop_of th) [] |
|
356 |
val substs = [(cterm_of thy (Var vx), cterm_of thy i_atm)] |
|
357 |
in cterm_instantiate substs th end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
358 |
|
32956 | 359 |
(* INFERENCE RULE: AXIOM *) |
32994 | 360 |
fun axiom_inf thpairs th = incr_indexes 1 (lookth thpairs th); |
32956 | 361 |
(*This causes variables to have an index of 1 by default. SEE ALSO mk_var above.*) |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
362 |
|
32956 | 363 |
(* INFERENCE RULE: ASSUME *) |
364 |
fun assume_inf ctxt mode atm = |
|
365 |
inst_excluded_middle |
|
366 |
(ProofContext.theory_of ctxt) |
|
367 |
(singleton (fol_terms_to_hol ctxt mode) (Metis.Term.Fn atm)); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
368 |
|
32956 | 369 |
(* INFERENCE RULE: INSTANTIATE (Subst). Type instantiations are ignored. Trying to reconstruct |
370 |
them admits new possibilities of errors, e.g. concerning sorts. Instead we try to arrange |
|
371 |
that new TVars are distinct and that types can be inferred from terms.*) |
|
372 |
fun inst_inf ctxt mode thpairs fsubst th = |
|
373 |
let val thy = ProofContext.theory_of ctxt |
|
374 |
val i_th = lookth thpairs th |
|
375 |
val i_th_vars = Term.add_vars (prop_of i_th) [] |
|
33035 | 376 |
fun find_var x = the (List.find (fn ((a,_),_) => a=x) i_th_vars) |
32956 | 377 |
fun subst_translation (x,y) = |
378 |
let val v = find_var x |
|
379 |
val t = fol_term_to_hol ctxt mode y (*we call infer_types below*) |
|
380 |
in SOME (cterm_of thy (Var v), t) end |
|
381 |
handle Option => |
|
382 |
(trace_msg (fn() => "List.find failed for the variable " ^ x ^ |
|
383 |
" in " ^ Display.string_of_thm ctxt i_th); |
|
384 |
NONE) |
|
385 |
fun remove_typeinst (a, t) = |
|
33227 | 386 |
case ResReconstruct.strip_prefix ResClause.schematic_var_prefix a of |
32956 | 387 |
SOME b => SOME (b, t) |
33227 | 388 |
| NONE => case ResReconstruct.strip_prefix ResClause.tvar_prefix a of |
32956 | 389 |
SOME _ => NONE (*type instantiations are forbidden!*) |
390 |
| NONE => SOME (a,t) (*internal Metis var?*) |
|
391 |
val _ = trace_msg (fn () => " isa th: " ^ Display.string_of_thm ctxt i_th) |
|
392 |
val substs = map_filter remove_typeinst (Metis.Subst.toList fsubst) |
|
393 |
val (vars,rawtms) = ListPair.unzip (map_filter subst_translation substs) |
|
394 |
val tms = infer_types ctxt rawtms; |
|
395 |
val ctm_of = cterm_incr_types thy (1 + Thm.maxidx_of i_th) |
|
396 |
val substs' = ListPair.zip (vars, map ctm_of tms) |
|
397 |
val _ = trace_msg (fn () => |
|
398 |
cat_lines ("subst_translations:" :: |
|
399 |
(substs' |> map (fn (x, y) => |
|
400 |
Syntax.string_of_term ctxt (term_of x) ^ " |-> " ^ |
|
401 |
Syntax.string_of_term ctxt (term_of y))))); |
|
402 |
in cterm_instantiate substs' i_th |
|
403 |
handle THM (msg, _, _) => error ("metis error (inst_inf): " ^ msg) |
|
404 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
405 |
|
32956 | 406 |
(* INFERENCE RULE: RESOLVE *) |
25713 | 407 |
|
32956 | 408 |
(*Like RSN, but we rename apart only the type variables. Vars here typically have an index |
409 |
of 1, and the use of RSN would increase this typically to 3. Instantiations of those Vars |
|
410 |
could then fail. See comment on mk_var.*) |
|
411 |
fun resolve_inc_tyvars(tha,i,thb) = |
|
412 |
let val tha = Drule.incr_type_indexes (1 + Thm.maxidx_of thb) tha |
|
413 |
val ths = Seq.list_of (Thm.bicompose false (false,tha,nprems_of tha) i thb) |
|
414 |
in |
|
415 |
case distinct Thm.eq_thm ths of |
|
416 |
[th] => th |
|
417 |
| _ => raise THM ("resolve_inc_tyvars: unique result expected", i, [tha,thb]) |
|
418 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
419 |
|
32956 | 420 |
fun resolve_inf ctxt mode thpairs atm th1 th2 = |
421 |
let |
|
422 |
val i_th1 = lookth thpairs th1 and i_th2 = lookth thpairs th2 |
|
423 |
val _ = trace_msg (fn () => " isa th1 (pos): " ^ Display.string_of_thm ctxt i_th1) |
|
424 |
val _ = trace_msg (fn () => " isa th2 (neg): " ^ Display.string_of_thm ctxt i_th2) |
|
425 |
in |
|
426 |
if is_TrueI i_th1 then i_th2 (*Trivial cases where one operand is type info*) |
|
427 |
else if is_TrueI i_th2 then i_th1 |
|
428 |
else |
|
429 |
let |
|
430 |
val i_atm = singleton (fol_terms_to_hol ctxt mode) (Metis.Term.Fn atm) |
|
431 |
val _ = trace_msg (fn () => " atom: " ^ Syntax.string_of_term ctxt i_atm) |
|
432 |
val prems_th1 = prems_of i_th1 |
|
433 |
val prems_th2 = prems_of i_th2 |
|
434 |
val index_th1 = get_index (mk_not i_atm) prems_th1 |
|
435 |
handle Empty => error "Failed to find literal in th1" |
|
436 |
val _ = trace_msg (fn () => " index_th1: " ^ Int.toString index_th1) |
|
437 |
val index_th2 = get_index i_atm prems_th2 |
|
438 |
handle Empty => error "Failed to find literal in th2" |
|
439 |
val _ = trace_msg (fn () => " index_th2: " ^ Int.toString index_th2) |
|
440 |
in resolve_inc_tyvars (Meson.select_literal index_th1 i_th1, index_th2, i_th2) end |
|
441 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
442 |
|
32956 | 443 |
(* INFERENCE RULE: REFL *) |
444 |
val refl_x = cterm_of @{theory} (Var (hd (Term.add_vars (prop_of REFL_THM) []))); |
|
445 |
val refl_idx = 1 + Thm.maxidx_of REFL_THM; |
|
25713 | 446 |
|
32956 | 447 |
fun refl_inf ctxt mode t = |
448 |
let val thy = ProofContext.theory_of ctxt |
|
449 |
val i_t = singleton (fol_terms_to_hol ctxt mode) t |
|
450 |
val _ = trace_msg (fn () => " term: " ^ Syntax.string_of_term ctxt i_t) |
|
451 |
val c_t = cterm_incr_types thy refl_idx i_t |
|
452 |
in cterm_instantiate [(refl_x, c_t)] REFL_THM end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
453 |
|
32994 | 454 |
fun get_ty_arg_size _ (Const ("op =", _)) = 0 (*equality has no type arguments*) |
33227 | 455 |
| get_ty_arg_size thy (Const (c, _)) = (ResReconstruct.num_typargs thy c handle TYPE _ => 0) |
32994 | 456 |
| get_ty_arg_size _ _ = 0; |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
457 |
|
32956 | 458 |
(* INFERENCE RULE: EQUALITY *) |
32994 | 459 |
fun equality_inf ctxt mode (pos, atm) fp fr = |
32956 | 460 |
let val thy = ProofContext.theory_of ctxt |
461 |
val m_tm = Metis.Term.Fn atm |
|
462 |
val [i_atm,i_tm] = fol_terms_to_hol ctxt mode [m_tm, fr] |
|
463 |
val _ = trace_msg (fn () => "sign of the literal: " ^ Bool.toString pos) |
|
32994 | 464 |
fun replace_item_list lx 0 (_::ls) = lx::ls |
32956 | 465 |
| replace_item_list lx i (l::ls) = l :: replace_item_list lx (i-1) ls |
466 |
fun path_finder_FO tm [] = (tm, Term.Bound 0) |
|
467 |
| path_finder_FO tm (p::ps) = |
|
468 |
let val (tm1,args) = Term.strip_comb tm |
|
469 |
val adjustment = get_ty_arg_size thy tm1 |
|
470 |
val p' = if adjustment > p then p else p-adjustment |
|
471 |
val tm_p = List.nth(args,p') |
|
472 |
handle Subscript => error ("equality_inf: " ^ Int.toString p ^ " adj " ^ |
|
473 |
Int.toString adjustment ^ " term " ^ Syntax.string_of_term ctxt tm) |
|
474 |
val _ = trace_msg (fn () => "path_finder: " ^ Int.toString p ^ |
|
475 |
" " ^ Syntax.string_of_term ctxt tm_p) |
|
476 |
val (r,t) = path_finder_FO tm_p ps |
|
477 |
in |
|
478 |
(r, list_comb (tm1, replace_item_list t p' args)) |
|
479 |
end |
|
480 |
fun path_finder_HO tm [] = (tm, Term.Bound 0) |
|
481 |
| path_finder_HO (t$u) (0::ps) = (fn(x,y) => (x, y$u)) (path_finder_HO t ps) |
|
32994 | 482 |
| path_finder_HO (t$u) (_::ps) = (fn(x,y) => (x, t$y)) (path_finder_HO u ps) |
32956 | 483 |
fun path_finder_FT tm [] _ = (tm, Term.Bound 0) |
32994 | 484 |
| path_finder_FT tm (0::ps) (Metis.Term.Fn ("ti", [t1, _])) = |
32956 | 485 |
path_finder_FT tm ps t1 |
32994 | 486 |
| path_finder_FT (t$u) (0::ps) (Metis.Term.Fn (".", [t1, _])) = |
32956 | 487 |
(fn(x,y) => (x, y$u)) (path_finder_FT t ps t1) |
32994 | 488 |
| path_finder_FT (t$u) (1::ps) (Metis.Term.Fn (".", [_, t2])) = |
32956 | 489 |
(fn(x,y) => (x, t$y)) (path_finder_FT u ps t2) |
490 |
| path_finder_FT tm ps t = error ("equality_inf, path_finder_FT: path = " ^ |
|
491 |
space_implode " " (map Int.toString ps) ^ |
|
492 |
" isa-term: " ^ Syntax.string_of_term ctxt tm ^ |
|
493 |
" fol-term: " ^ Metis.Term.toString t) |
|
494 |
fun path_finder FO tm ps _ = path_finder_FO tm ps |
|
495 |
| path_finder HO (tm as Const("op =",_) $ _ $ _) (p::ps) _ = |
|
496 |
(*equality: not curried, as other predicates are*) |
|
497 |
if p=0 then path_finder_HO tm (0::1::ps) (*select first operand*) |
|
498 |
else path_finder_HO tm (p::ps) (*1 selects second operand*) |
|
32994 | 499 |
| path_finder HO tm (_ :: ps) (Metis.Term.Fn ("{}", [_])) = |
32956 | 500 |
path_finder_HO tm ps (*if not equality, ignore head to skip hBOOL*) |
501 |
| path_finder FT (tm as Const("op =",_) $ _ $ _) (p::ps) |
|
502 |
(Metis.Term.Fn ("=", [t1,t2])) = |
|
503 |
(*equality: not curried, as other predicates are*) |
|
504 |
if p=0 then path_finder_FT tm (0::1::ps) |
|
505 |
(Metis.Term.Fn (".", [Metis.Term.Fn (".", [metis_eq,t1]), t2])) |
|
506 |
(*select first operand*) |
|
507 |
else path_finder_FT tm (p::ps) |
|
508 |
(Metis.Term.Fn (".", [metis_eq,t2])) |
|
509 |
(*1 selects second operand*) |
|
32994 | 510 |
| path_finder FT tm (_ :: ps) (Metis.Term.Fn ("{}", [t1])) = path_finder_FT tm ps t1 |
32956 | 511 |
(*if not equality, ignore head to skip the hBOOL predicate*) |
512 |
| path_finder FT tm ps t = path_finder_FT tm ps t (*really an error case!*) |
|
513 |
fun path_finder_lit ((nt as Term.Const ("Not", _)) $ tm_a) idx = |
|
514 |
let val (tm, tm_rslt) = path_finder mode tm_a idx m_tm |
|
515 |
in (tm, nt $ tm_rslt) end |
|
516 |
| path_finder_lit tm_a idx = path_finder mode tm_a idx m_tm |
|
517 |
val (tm_subst, body) = path_finder_lit i_atm fp |
|
518 |
val tm_abs = Term.Abs("x", Term.type_of tm_subst, body) |
|
519 |
val _ = trace_msg (fn () => "abstraction: " ^ Syntax.string_of_term ctxt tm_abs) |
|
520 |
val _ = trace_msg (fn () => "i_tm: " ^ Syntax.string_of_term ctxt i_tm) |
|
521 |
val _ = trace_msg (fn () => "located term: " ^ Syntax.string_of_term ctxt tm_subst) |
|
522 |
val imax = maxidx_of_term (i_tm $ tm_abs $ tm_subst) (*ill typed but gives right max*) |
|
523 |
val subst' = incr_indexes (imax+1) (if pos then subst_em else ssubst_em) |
|
524 |
val _ = trace_msg (fn () => "subst' " ^ Display.string_of_thm ctxt subst') |
|
525 |
val eq_terms = map (pairself (cterm_of thy)) |
|
33227 | 526 |
(ListPair.zip (OldTerm.term_vars (prop_of subst'), [tm_abs, tm_subst, i_tm])) |
32956 | 527 |
in cterm_instantiate eq_terms subst' end; |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
528 |
|
32956 | 529 |
val factor = Seq.hd o distinct_subgoals_tac; |
28528
0cf2749e8ef7
The result of the equality inference rule no longer undergoes factoring.
paulson
parents:
28262
diff
changeset
|
530 |
|
32994 | 531 |
fun step _ _ thpairs (fol_th, Metis.Proof.Axiom _) = factor (axiom_inf thpairs fol_th) |
532 |
| step ctxt mode _ (_, Metis.Proof.Assume f_atm) = assume_inf ctxt mode f_atm |
|
533 |
| step ctxt mode thpairs (_, Metis.Proof.Subst (f_subst, f_th1)) = |
|
32956 | 534 |
factor (inst_inf ctxt mode thpairs f_subst f_th1) |
32994 | 535 |
| step ctxt mode thpairs (_, Metis.Proof.Resolve(f_atm, f_th1, f_th2)) = |
32956 | 536 |
factor (resolve_inf ctxt mode thpairs f_atm f_th1 f_th2) |
32994 | 537 |
| step ctxt mode _ (_, Metis.Proof.Refl f_tm) = refl_inf ctxt mode f_tm |
538 |
| step ctxt mode _ (_, Metis.Proof.Equality (f_lit, f_p, f_r)) = |
|
539 |
equality_inf ctxt mode f_lit f_p f_r; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
540 |
|
32994 | 541 |
fun real_literal (_, (c, _)) = not (String.isPrefix ResClause.class_prefix c); |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
542 |
|
32994 | 543 |
fun translate _ _ thpairs [] = thpairs |
32956 | 544 |
| translate mode ctxt thpairs ((fol_th, inf) :: infpairs) = |
545 |
let val _ = trace_msg (fn () => "=============================================") |
|
546 |
val _ = trace_msg (fn () => "METIS THM: " ^ Metis.Thm.toString fol_th) |
|
547 |
val _ = trace_msg (fn () => "INFERENCE: " ^ Metis.Proof.inferenceToString inf) |
|
548 |
val th = Meson.flexflex_first_order (step ctxt mode thpairs (fol_th, inf)) |
|
549 |
val _ = trace_msg (fn () => "ISABELLE THM: " ^ Display.string_of_thm ctxt th) |
|
550 |
val _ = trace_msg (fn () => "=============================================") |
|
32994 | 551 |
val n_metis_lits = |
552 |
length (filter real_literal (Metis.LiteralSet.toList (Metis.Thm.clause fol_th))) |
|
32956 | 553 |
in |
554 |
if nprems_of th = n_metis_lits then () |
|
555 |
else error "Metis: proof reconstruction has gone wrong"; |
|
556 |
translate mode ctxt ((fol_th, th) :: thpairs) infpairs |
|
557 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
558 |
|
32956 | 559 |
(*Determining which axiom clauses are actually used*) |
560 |
fun used_axioms axioms (th, Metis.Proof.Axiom _) = SOME (lookth axioms th) |
|
32994 | 561 |
| used_axioms _ _ = NONE; |
24855 | 562 |
|
32956 | 563 |
(* ------------------------------------------------------------------------- *) |
564 |
(* Translation of HO Clauses *) |
|
565 |
(* ------------------------------------------------------------------------- *) |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
566 |
|
32956 | 567 |
fun cnf_th thy th = hd (ResAxioms.cnf_axiom thy th); |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
568 |
|
32956 | 569 |
val equal_imp_fequal' = cnf_th @{theory} @{thm equal_imp_fequal}; |
570 |
val fequal_imp_equal' = cnf_th @{theory} @{thm fequal_imp_equal}; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
571 |
|
32956 | 572 |
val comb_I = cnf_th @{theory} ResHolClause.comb_I; |
573 |
val comb_K = cnf_th @{theory} ResHolClause.comb_K; |
|
574 |
val comb_B = cnf_th @{theory} ResHolClause.comb_B; |
|
575 |
val comb_C = cnf_th @{theory} ResHolClause.comb_C; |
|
576 |
val comb_S = cnf_th @{theory} ResHolClause.comb_S; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
577 |
|
32956 | 578 |
fun type_ext thy tms = |
579 |
let val subs = ResAtp.tfree_classes_of_terms tms |
|
580 |
val supers = ResAtp.tvar_classes_of_terms tms |
|
581 |
and tycons = ResAtp.type_consts_of_terms thy tms |
|
32994 | 582 |
val (supers', arity_clauses) = ResClause.make_arity_clauses thy tycons supers |
32956 | 583 |
val classrel_clauses = ResClause.make_classrel_clauses thy subs supers' |
584 |
in map classrel_cls classrel_clauses @ map arity_cls arity_clauses |
|
585 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
586 |
|
32956 | 587 |
(* ------------------------------------------------------------------------- *) |
588 |
(* Logic maps manage the interface between HOL and first-order logic. *) |
|
589 |
(* ------------------------------------------------------------------------- *) |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
590 |
|
32956 | 591 |
type logic_map = |
33243 | 592 |
{axioms : (Metis.Thm.thm * thm) list, |
32956 | 593 |
tfrees : ResClause.type_literal list}; |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
594 |
|
32994 | 595 |
fun const_in_metis c (pred, tm_list) = |
32956 | 596 |
let |
32994 | 597 |
fun in_mterm (Metis.Term.Var _) = false |
32956 | 598 |
| in_mterm (Metis.Term.Fn (".", tm_list)) = exists in_mterm tm_list |
599 |
| in_mterm (Metis.Term.Fn (nm, tm_list)) = c=nm orelse exists in_mterm tm_list |
|
32994 | 600 |
in c = pred orelse exists in_mterm tm_list end; |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
601 |
|
32956 | 602 |
(*Extract TFree constraints from context to include as conjecture clauses*) |
603 |
fun init_tfrees ctxt = |
|
604 |
let fun add ((a,i),s) Ts = if i = ~1 then TFree(a,s) :: Ts else Ts |
|
605 |
in ResClause.add_typs (Vartab.fold add (#2 (Variable.constraints_of ctxt)) []) end; |
|
24937
340523598914
context-based treatment of generalization; also handling TFrees in axiom clauses
paulson
parents:
24920
diff
changeset
|
606 |
|
32956 | 607 |
(*transform isabelle type / arity clause to metis clause *) |
608 |
fun add_type_thm [] lmap = lmap |
|
609 |
| add_type_thm ((ith, mth) :: cls) {axioms, tfrees} = |
|
610 |
add_type_thm cls {axioms = (mth, ith) :: axioms, |
|
611 |
tfrees = tfrees} |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
612 |
|
32956 | 613 |
(*Insert non-logical axioms corresponding to all accumulated TFrees*) |
614 |
fun add_tfrees {axioms, tfrees} : logic_map = |
|
615 |
{axioms = (map (fn tf => (metis_of_tfree tf, TrueI)) (distinct op= tfrees)) @ axioms, |
|
616 |
tfrees = tfrees}; |
|
25713 | 617 |
|
32956 | 618 |
fun string_of_mode FO = "FO" |
619 |
| string_of_mode HO = "HO" |
|
620 |
| string_of_mode FT = "FT" |
|
32532
a0a54a51b15b
My umpteenth attempt to commit the method metisFT, a fully-typed version of metis
paulson
parents:
32530
diff
changeset
|
621 |
|
32956 | 622 |
(* Function to generate metis clauses, including comb and type clauses *) |
623 |
fun build_map mode0 ctxt cls ths = |
|
624 |
let val thy = ProofContext.theory_of ctxt |
|
625 |
(*The modes FO and FT are sticky. HO can be downgraded to FO.*) |
|
626 |
fun set_mode FO = FO |
|
627 |
| set_mode HO = if forall (Meson.is_fol_term thy o prop_of) (cls@ths) then FO else HO |
|
628 |
| set_mode FT = FT |
|
629 |
val mode = set_mode mode0 |
|
630 |
(*transform isabelle clause to metis clause *) |
|
631 |
fun add_thm is_conjecture (ith, {axioms, tfrees}) : logic_map = |
|
632 |
let val (mth, tfree_lits) = hol_thm_to_fol is_conjecture ctxt mode ith |
|
633 |
in |
|
634 |
{axioms = (mth, Meson.make_meta_clause ith) :: axioms, |
|
33042 | 635 |
tfrees = union (op =) tfree_lits tfrees} |
32956 | 636 |
end; |
637 |
val lmap0 = List.foldl (add_thm true) |
|
638 |
{axioms = [], tfrees = init_tfrees ctxt} cls |
|
639 |
val lmap = List.foldl (add_thm false) (add_tfrees lmap0) ths |
|
640 |
val clause_lists = map (Metis.Thm.clause o #1) (#axioms lmap) |
|
32994 | 641 |
fun used c = exists (Metis.LiteralSet.exists (const_in_metis c o #2)) clause_lists |
32956 | 642 |
(*Now check for the existence of certain combinators*) |
643 |
val thI = if used "c_COMBI" then [comb_I] else [] |
|
644 |
val thK = if used "c_COMBK" then [comb_K] else [] |
|
645 |
val thB = if used "c_COMBB" then [comb_B] else [] |
|
646 |
val thC = if used "c_COMBC" then [comb_C] else [] |
|
647 |
val thS = if used "c_COMBS" then [comb_S] else [] |
|
648 |
val thEQ = if used "c_fequal" then [fequal_imp_equal', equal_imp_fequal'] else [] |
|
649 |
val lmap' = if mode=FO then lmap |
|
650 |
else List.foldl (add_thm false) lmap (thEQ @ thS @ thC @ thB @ thK @ thI) |
|
651 |
in |
|
652 |
(mode, add_type_thm (type_ext thy (map prop_of (cls @ ths))) lmap') |
|
653 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
654 |
|
32956 | 655 |
fun refute cls = |
656 |
Metis.Resolution.loop (Metis.Resolution.new Metis.Resolution.default cls); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
657 |
|
32956 | 658 |
fun is_false t = t aconv (HOLogic.mk_Trueprop HOLogic.false_const); |
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
659 |
|
32956 | 660 |
fun common_thm ths1 ths2 = exists (member Thm.eq_thm ths1) (map Meson.make_meta_clause ths2); |
24855 | 661 |
|
32956 | 662 |
exception METIS of string; |
28233
f14f34194f63
The metis method now fails in the usual manner, rather than raising an exception,
paulson
parents:
28175
diff
changeset
|
663 |
|
32956 | 664 |
(* Main function to start metis prove and reconstruction *) |
665 |
fun FOL_SOLVE mode ctxt cls ths0 = |
|
666 |
let val thy = ProofContext.theory_of ctxt |
|
667 |
val th_cls_pairs = map (fn th => (Thm.get_name_hint th, ResAxioms.cnf_axiom thy th)) ths0 |
|
668 |
val ths = maps #2 th_cls_pairs |
|
669 |
val _ = trace_msg (fn () => "FOL_SOLVE: CONJECTURE CLAUSES") |
|
670 |
val _ = app (fn th => trace_msg (fn () => Display.string_of_thm ctxt th)) cls |
|
671 |
val _ = trace_msg (fn () => "THEOREM CLAUSES") |
|
672 |
val _ = app (fn th => trace_msg (fn () => Display.string_of_thm ctxt th)) ths |
|
673 |
val (mode, {axioms,tfrees}) = build_map mode ctxt cls ths |
|
674 |
val _ = if null tfrees then () |
|
675 |
else (trace_msg (fn () => "TFREE CLAUSES"); |
|
676 |
app (fn tf => trace_msg (fn _ => ResClause.tptp_of_typeLit true tf)) tfrees) |
|
677 |
val _ = trace_msg (fn () => "CLAUSES GIVEN TO METIS") |
|
678 |
val thms = map #1 axioms |
|
679 |
val _ = app (fn th => trace_msg (fn () => Metis.Thm.toString th)) thms |
|
680 |
val _ = trace_msg (fn () => "mode = " ^ string_of_mode mode) |
|
681 |
val _ = trace_msg (fn () => "START METIS PROVE PROCESS") |
|
682 |
in |
|
683 |
case List.filter (is_false o prop_of) cls of |
|
684 |
false_th::_ => [false_th RS @{thm FalseE}] |
|
685 |
| [] => |
|
686 |
case refute thms of |
|
687 |
Metis.Resolution.Contradiction mth => |
|
688 |
let val _ = trace_msg (fn () => "METIS RECONSTRUCTION START: " ^ |
|
689 |
Metis.Thm.toString mth) |
|
690 |
val ctxt' = fold Variable.declare_constraints (map prop_of cls) ctxt |
|
691 |
(*add constraints arising from converting goal to clause form*) |
|
692 |
val proof = Metis.Proof.proof mth |
|
693 |
val result = translate mode ctxt' axioms proof |
|
694 |
and used = map_filter (used_axioms axioms) proof |
|
695 |
val _ = trace_msg (fn () => "METIS COMPLETED...clauses actually used:") |
|
696 |
val _ = app (fn th => trace_msg (fn () => Display.string_of_thm ctxt th)) used |
|
32994 | 697 |
val unused = filter (fn (_, cls) => not (common_thm used cls)) th_cls_pairs |
32956 | 698 |
in |
699 |
if null unused then () |
|
700 |
else warning ("Metis: unused theorems " ^ commas_quote (map #1 unused)); |
|
701 |
case result of |
|
702 |
(_,ith)::_ => |
|
703 |
(trace_msg (fn () => "success: " ^ Display.string_of_thm ctxt ith); |
|
704 |
[ith]) |
|
705 |
| _ => (trace_msg (fn () => "Metis: no result"); |
|
706 |
[]) |
|
707 |
end |
|
708 |
| Metis.Resolution.Satisfiable _ => |
|
709 |
(trace_msg (fn () => "Metis: No first-order proof with the lemmas supplied"); |
|
710 |
[]) |
|
711 |
end; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
712 |
|
32956 | 713 |
fun metis_general_tac mode ctxt ths i st0 = |
714 |
let val _ = trace_msg (fn () => |
|
715 |
"Metis called with theorems " ^ cat_lines (map (Display.string_of_thm ctxt) ths)) |
|
716 |
in |
|
717 |
if exists_type ResAxioms.type_has_empty_sort (prop_of st0) |
|
718 |
then (warning "Proof state contains the empty sort"; Seq.empty) |
|
719 |
else |
|
720 |
(Meson.MESON ResAxioms.neg_clausify |
|
721 |
(fn cls => resolve_tac (FOL_SOLVE mode ctxt cls ths) 1) ctxt i |
|
722 |
THEN ResAxioms.expand_defs_tac st0) st0 |
|
723 |
end |
|
724 |
handle METIS s => (warning ("Metis: " ^ s); Seq.empty); |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
725 |
|
32956 | 726 |
val metis_tac = metis_general_tac HO; |
727 |
val metisF_tac = metis_general_tac FO; |
|
728 |
val metisFT_tac = metis_general_tac FT; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
729 |
|
32956 | 730 |
fun method name mode comment = Method.setup name (Attrib.thms >> (fn ths => fn ctxt => |
731 |
SIMPLE_METHOD' (CHANGED_PROP o metis_general_tac mode ctxt ths))) comment; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
732 |
|
32956 | 733 |
val setup = |
734 |
type_lits_setup #> |
|
735 |
method @{binding metis} HO "METIS for FOL & HOL problems" #> |
|
736 |
method @{binding metisF} FO "METIS for FOL problems" #> |
|
737 |
method @{binding metisFT} FT "METIS With-fully typed translation" #> |
|
738 |
Method.setup @{binding finish_clausify} |
|
739 |
(Scan.succeed (K (SIMPLE_METHOD (ResAxioms.expand_defs_tac refl)))) |
|
740 |
"cleanup after conversion to clauses"; |
|
23442
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
741 |
|
028e39e5e8f3
The Metis prover (slightly modified version from Larry);
wenzelm
parents:
diff
changeset
|
742 |
end; |