author | wenzelm |
Wed, 15 Feb 2012 23:19:30 +0100 | |
changeset 46497 | 89ccf66aa73d |
parent 45654 | cf10bde35973 |
child 51717 | 9e7d1c139569 |
permissions | -rw-r--r-- |
37744 | 1 |
(* Title: HOL/Decision_Procs/ferrante_rackoff.ML |
23466 | 2 |
Author: Amine Chaieb, TU Muenchen |
3 |
||
4 |
Ferrante and Rackoff's algorithm for quantifier elimination in dense |
|
5 |
linear orders. Proof-synthesis and tactic. |
|
6 |
*) |
|
7 |
||
23567 | 8 |
signature FERRANTE_RACKOFF = |
23466 | 9 |
sig |
23567 | 10 |
val dlo_conv: Proof.context -> conv |
23466 | 11 |
val dlo_tac: Proof.context -> int -> tactic |
12 |
end; |
|
13 |
||
14 |
structure FerranteRackoff: FERRANTE_RACKOFF = |
|
15 |
struct |
|
16 |
||
17 |
open Ferrante_Rackoff_Data; |
|
18 |
open Conv; |
|
19 |
||
23567 | 20 |
type entry = {minf: thm list, pinf: thm list, nmi: thm list, npi: thm list, |
23466 | 21 |
ld: thm list, qe: thm, atoms : cterm list} * |
23567 | 22 |
{isolate_conv: cterm list -> cterm -> thm, |
23466 | 23 |
whatis : cterm -> cterm -> ord, |
24 |
simpset : simpset}; |
|
25 |
||
23567 | 26 |
fun get_p1 th = |
27 |
funpow 2 (Thm.dest_arg o snd o Thm.dest_abs NONE) |
|
28 |
(funpow 2 Thm.dest_arg (cprop_of th)) |> Thm.dest_arg |
|
23466 | 29 |
|
30 |
fun ferrack_conv |
|
23567 | 31 |
(entr as ({minf = minf, pinf = pinf, nmi = nmi, npi = npi, |
23466 | 32 |
ld = ld, qe = qe, atoms = atoms}, |
23567 | 33 |
{isolate_conv = icv, whatis = wi, simpset = simpset}):entry) = |
34 |
let |
|
23466 | 35 |
fun uset (vars as (x::vs)) p = case term_of p of |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
36 |
Const(@{const_name HOL.conj}, _)$ _ $ _ => |
23567 | 37 |
let |
38 |
val ((b,l),r) = Thm.dest_comb p |>> Thm.dest_comb |
|
23466 | 39 |
val (lS,lth) = uset vars l val (rS, rth) = uset vars r |
23567 | 40 |
in (lS@rS, Drule.binop_cong_rule b lth rth) end |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
41 |
| Const(@{const_name HOL.disj}, _)$ _ $ _ => |
23567 | 42 |
let |
43 |
val ((b,l),r) = Thm.dest_comb p |>> Thm.dest_comb |
|
23466 | 44 |
val (lS,lth) = uset vars l val (rS, rth) = uset vars r |
23567 | 45 |
in (lS@rS, Drule.binop_cong_rule b lth rth) end |
46 |
| _ => |
|
47 |
let |
|
48 |
val th = icv vars p |
|
23466 | 49 |
val p' = Thm.rhs_of th |
50 |
val c = wi x p' |
|
23567 | 51 |
val S = (if member (op =) [Lt, Le, Eq] c then single o Thm.dest_arg |
52 |
else if member (op =) [Gt, Ge] c then single o Thm.dest_arg1 |
|
53 |
else if c = NEq then single o Thm.dest_arg o Thm.dest_arg |
|
23466 | 54 |
else K []) p' |
55 |
in (S,th) end |
|
56 |
||
23567 | 57 |
val ((p1_v,p2_v),(mp1_v,mp2_v)) = |
58 |
funpow 2 (Thm.dest_arg o snd o Thm.dest_abs NONE) |
|
59 |
(funpow 4 Thm.dest_arg (cprop_of (hd minf))) |
|
60 |
|> Thm.dest_binop |> pairself Thm.dest_binop |> apfst (pairself Thm.dest_fun) |
|
61 |
||
62 |
fun myfwd (th1, th2, th3, th4, th5) p1 p2 |
|
63 |
[(th_1,th_2,th_3,th_4,th_5), (th_1',th_2',th_3',th_4',th_5')] = |
|
23466 | 64 |
let |
65 |
val (mp1, mp2) = (get_p1 th_1, get_p1 th_1') |
|
66 |
val (pp1, pp2) = (get_p1 th_2, get_p1 th_2') |
|
23567 | 67 |
fun fw mi th th' th'' = |
68 |
let |
|
69 |
val th0 = if mi then |
|
43333
2bdec7f430d3
renamed Drule.instantiate to Drule.instantiate_normalize to emphasize its meaning as opposed to plain Thm.instantiate;
wenzelm
parents:
40314
diff
changeset
|
70 |
Drule.instantiate_normalize ([],[(p1_v, p1),(p2_v, p2),(mp1_v, mp1), (mp2_v, mp2)]) th |
2bdec7f430d3
renamed Drule.instantiate to Drule.instantiate_normalize to emphasize its meaning as opposed to plain Thm.instantiate;
wenzelm
parents:
40314
diff
changeset
|
71 |
else Drule.instantiate_normalize ([],[(p1_v, p1),(p2_v, p2),(mp1_v, pp1), (mp2_v, pp2)]) th |
36945 | 72 |
in Thm.implies_elim (Thm.implies_elim th0 th') th'' end |
23567 | 73 |
in (fw true th1 th_1 th_1', fw false th2 th_2 th_2', |
74 |
fw true th3 th_3 th_3', fw false th4 th_4 th_4', fw true th5 th_5 th_5') |
|
23466 | 75 |
end |
76 |
val U_v = (Thm.dest_arg o Thm.dest_arg o Thm.dest_arg1) (cprop_of qe) |
|
23567 | 77 |
fun main vs p = |
78 |
let |
|
79 |
val ((xn,ce),(x,fm)) = (case term_of p of |
|
38558 | 80 |
Const(@{const_name Ex},_)$Abs(xn,xT,_) => |
23466 | 81 |
Thm.dest_comb p ||> Thm.dest_abs (SOME xn) |>> pair xn |
23567 | 82 |
| _ => raise CTERM ("main QE only treats existential quantifiers!", [p])) |
23466 | 83 |
val cT = ctyp_of_term x |
84 |
val (u,nth) = uset (x::vs) fm |>> distinct (op aconvc) |
|
85 |
val nthx = Thm.abstract_rule xn x nth |
|
86 |
val q = Thm.rhs_of nth |
|
87 |
val qx = Thm.rhs_of nthx |
|
88 |
val enth = Drule.arg_cong_rule ce nthx |
|
89 |
val [th0,th1] = map (instantiate' [SOME cT] []) @{thms "finite.intros"} |
|
23567 | 90 |
fun ins x th = |
36945 | 91 |
Thm.implies_elim (instantiate' [] [(SOME o Thm.dest_arg o Thm.dest_arg) |
23466 | 92 |
(Thm.cprop_of th), SOME x] th1) th |
93 |
val fU = fold ins u th0 |
|
94 |
val cU = funpow 2 Thm.dest_arg (Thm.cprop_of fU) |
|
23567 | 95 |
local |
23466 | 96 |
val insI1 = instantiate' [SOME cT] [] @{thm "insertI1"} |
97 |
val insI2 = instantiate' [SOME cT] [] @{thm "insertI2"} |
|
98 |
in |
|
23567 | 99 |
fun provein x S = |
23466 | 100 |
case term_of S of |
32264
0be31453f698
Set.UNIV and Set.empty are mere abbreviations for top and bot
haftmann
parents:
32149
diff
changeset
|
101 |
Const(@{const_name Orderings.bot}, _) => raise CTERM ("provein : not a member!", [S]) |
30304
d8e4cd2ac2a1
set operations Int, Un, INTER, UNION, Inter, Union, empty, UNIV are now proper qualified constants with authentic syntax
haftmann
parents:
24584
diff
changeset
|
102 |
| Const(@{const_name insert}, _) $ y $_ => |
23466 | 103 |
let val (cy,S') = Thm.dest_binop S |
104 |
in if term_of x aconv y then instantiate' [] [SOME x, SOME S'] insI1 |
|
36945 | 105 |
else Thm.implies_elim (instantiate' [] [SOME x, SOME S', SOME cy] insI2) |
23466 | 106 |
(provein x S') |
107 |
end |
|
108 |
end |
|
23567 | 109 |
val tabU = fold (fn t => fn tab => Termtab.update (term_of t, provein t cU) tab) |
23466 | 110 |
u Termtab.empty |
23567 | 111 |
val U = the o Termtab.lookup tabU o term_of |
112 |
val [minf_conj, minf_disj, minf_eq, minf_neq, minf_lt, |
|
23466 | 113 |
minf_le, minf_gt, minf_ge, minf_P] = minf |
23567 | 114 |
val [pinf_conj, pinf_disj, pinf_eq, pinf_neq, pinf_lt, |
23466 | 115 |
pinf_le, pinf_gt, pinf_ge, pinf_P] = pinf |
23567 | 116 |
val [nmi_conj, nmi_disj, nmi_eq, nmi_neq, nmi_lt, |
43333
2bdec7f430d3
renamed Drule.instantiate to Drule.instantiate_normalize to emphasize its meaning as opposed to plain Thm.instantiate;
wenzelm
parents:
40314
diff
changeset
|
117 |
nmi_le, nmi_gt, nmi_ge, nmi_P] = map (Drule.instantiate_normalize ([],[(U_v,cU)])) nmi |
23567 | 118 |
val [npi_conj, npi_disj, npi_eq, npi_neq, npi_lt, |
43333
2bdec7f430d3
renamed Drule.instantiate to Drule.instantiate_normalize to emphasize its meaning as opposed to plain Thm.instantiate;
wenzelm
parents:
40314
diff
changeset
|
119 |
npi_le, npi_gt, npi_ge, npi_P] = map (Drule.instantiate_normalize ([],[(U_v,cU)])) npi |
23567 | 120 |
val [ld_conj, ld_disj, ld_eq, ld_neq, ld_lt, |
43333
2bdec7f430d3
renamed Drule.instantiate to Drule.instantiate_normalize to emphasize its meaning as opposed to plain Thm.instantiate;
wenzelm
parents:
40314
diff
changeset
|
121 |
ld_le, ld_gt, ld_ge, ld_P] = map (Drule.instantiate_normalize ([],[(U_v,cU)])) ld |
23567 | 122 |
|
123 |
fun decomp_mpinf fm = |
|
23466 | 124 |
case term_of fm of |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
125 |
Const(@{const_name HOL.conj},_)$_$_ => |
23567 | 126 |
let val (p,q) = Thm.dest_binop fm |
127 |
in ([p,q], myfwd (minf_conj,pinf_conj, nmi_conj, npi_conj,ld_conj) |
|
46497
89ccf66aa73d
renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in conformance with similar operations in structure Term and Logic;
wenzelm
parents:
45654
diff
changeset
|
128 |
(Thm.lambda x p) (Thm.lambda x q)) |
23466 | 129 |
end |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
130 |
| Const(@{const_name HOL.disj},_)$_$_ => |
23567 | 131 |
let val (p,q) = Thm.dest_binop fm |
23466 | 132 |
in ([p,q],myfwd (minf_disj, pinf_disj, nmi_disj, npi_disj,ld_disj) |
46497
89ccf66aa73d
renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in conformance with similar operations in structure Term and Logic;
wenzelm
parents:
45654
diff
changeset
|
133 |
(Thm.lambda x p) (Thm.lambda x q)) |
23466 | 134 |
end |
23567 | 135 |
| _ => |
23466 | 136 |
(let val c = wi x fm |
23567 | 137 |
val t = (if c=Nox then I |
138 |
else if member (op =) [Lt, Le, Eq] c then Thm.dest_arg |
|
139 |
else if member (op =) [Gt, Ge] c then Thm.dest_arg1 |
|
140 |
else if c = NEq then (Thm.dest_arg o Thm.dest_arg) |
|
40314
b5ec88d9ac03
replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
wenzelm
parents:
38864
diff
changeset
|
141 |
else raise Fail "decomp_mpinf: Impossible case!!") fm |
23567 | 142 |
val [mi_th, pi_th, nmi_th, npi_th, ld_th] = |
143 |
if c = Nox then map (instantiate' [] [SOME fm]) |
|
23466 | 144 |
[minf_P, pinf_P, nmi_P, npi_P, ld_P] |
23567 | 145 |
else |
146 |
let val [mi_th,pi_th,nmi_th,npi_th,ld_th] = |
|
23466 | 147 |
map (instantiate' [] [SOME t]) |
148 |
(case c of Lt => [minf_lt, pinf_lt, nmi_lt, npi_lt, ld_lt] |
|
149 |
| Le => [minf_le, pinf_le, nmi_le, npi_le, ld_le] |
|
150 |
| Gt => [minf_gt, pinf_gt, nmi_gt, npi_gt, ld_gt] |
|
151 |
| Ge => [minf_ge, pinf_ge, nmi_ge, npi_ge, ld_ge] |
|
152 |
| Eq => [minf_eq, pinf_eq, nmi_eq, npi_eq, ld_eq] |
|
153 |
| NEq => [minf_neq, pinf_neq, nmi_neq, npi_neq, ld_neq]) |
|
154 |
val tU = U t |
|
36945 | 155 |
fun Ufw th = Thm.implies_elim th tU |
23466 | 156 |
in [mi_th, pi_th, Ufw nmi_th, Ufw npi_th, Ufw ld_th] |
157 |
end |
|
158 |
in ([], K (mi_th, pi_th, nmi_th, npi_th, ld_th)) end) |
|
159 |
val (minf_th, pinf_th, nmi_th, npi_th, ld_th) = divide_and_conquer decomp_mpinf q |
|
23567 | 160 |
val qe_th = Drule.implies_elim_list |
161 |
((fconv_rule (Thm.beta_conversion true)) |
|
162 |
(instantiate' [] (map SOME [cU, qx, get_p1 minf_th, get_p1 pinf_th]) |
|
23466 | 163 |
qe)) |
23567 | 164 |
[fU, ld_th, nmi_th, npi_th, minf_th, pinf_th] |
165 |
val bex_conv = |
|
45654 | 166 |
Simplifier.rewrite (HOL_basic_ss addsimps @{thms simp_thms bex_simps(1-5)}) |
36945 | 167 |
val result_th = fconv_rule (arg_conv bex_conv) (Thm.transitive enth qe_th) |
23466 | 168 |
in result_th |
169 |
end |
|
170 |
||
171 |
in main |
|
172 |
end; |
|
173 |
||
23567 | 174 |
val grab_atom_bop = |
175 |
let |
|
23466 | 176 |
fun h bounds tm = |
177 |
(case term_of tm of |
|
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
178 |
Const (@{const_name HOL.eq}, T) $ _ $ _ => |
23567 | 179 |
if domain_type T = HOLogic.boolT then find_args bounds tm |
23466 | 180 |
else Thm.dest_fun2 tm |
38558 | 181 |
| Const (@{const_name Not}, _) $ _ => h bounds (Thm.dest_arg tm) |
182 |
| Const (@{const_name All}, _) $ _ => find_body bounds (Thm.dest_arg tm) |
|
183 |
| Const (@{const_name Ex}, _) $ _ => find_body bounds (Thm.dest_arg tm) |
|
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
184 |
| Const (@{const_name HOL.conj}, _) $ _ $ _ => find_args bounds tm |
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
185 |
| Const (@{const_name HOL.disj}, _) $ _ $ _ => find_args bounds tm |
38786
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
haftmann
parents:
38558
diff
changeset
|
186 |
| Const (@{const_name HOL.implies}, _) $ _ $ _ => find_args bounds tm |
23466 | 187 |
| Const ("==>", _) $ _ $ _ => find_args bounds tm |
188 |
| Const ("==", _) $ _ $ _ => find_args bounds tm |
|
36099 | 189 |
| Const ("all", _) $ _ => find_body bounds (Thm.dest_arg tm) |
38558 | 190 |
| Const (@{const_name Trueprop}, _) $ _ => h bounds (Thm.dest_arg tm) |
23466 | 191 |
| _ => Thm.dest_fun2 tm) |
23567 | 192 |
and find_args bounds tm = |
23466 | 193 |
(h bounds (Thm.dest_arg tm) handle CTERM _ => Thm.dest_arg1 tm) |
194 |
and find_body bounds b = |
|
195 |
let val (_, b') = Thm.dest_abs (SOME (Name.bound bounds)) b |
|
196 |
in h (bounds + 1) b' end; |
|
197 |
in h end; |
|
198 |
||
23567 | 199 |
fun raw_ferrack_qe_conv ctxt (thy, {isolate_conv, whatis, simpset}) tm = |
200 |
let |
|
23466 | 201 |
val ss = simpset |
23567 | 202 |
val ss' = |
45654 | 203 |
merge_ss (HOL_basic_ss addsimps @{thms simp_thms ex_simps all_simps |
204 |
not_all all_not_ex ex_disj_distrib}, ss) |
|
23567 | 205 |
|> Simplifier.inherit_context ss |
206 |
val pcv = Simplifier.rewrite ss' |
|
207 |
val postcv = Simplifier.rewrite ss |
|
208 |
val nnf = K (nnf_conv then_conv postcv) |
|
209 |
val qe_conv = Qelim.gen_qelim_conv pcv postcv pcv cons (Thm.add_cterm_frees tm []) |
|
23466 | 210 |
(isolate_conv ctxt) nnf |
23567 | 211 |
(fn vs => ferrack_conv (thy,{isolate_conv = isolate_conv ctxt, |
23466 | 212 |
whatis = whatis, simpset = simpset}) vs |
213 |
then_conv postcv) |
|
23486 | 214 |
in (Simplifier.rewrite ss then_conv qe_conv) tm end; |
23466 | 215 |
|
23567 | 216 |
fun dlo_instance ctxt tm = |
217 |
Ferrante_Rackoff_Data.match ctxt (grab_atom_bop 0 tm); |
|
23486 | 218 |
|
23567 | 219 |
fun dlo_conv ctxt tm = |
220 |
(case dlo_instance ctxt tm of |
|
221 |
NONE => raise CTERM ("ferrackqe_conv: no corresponding instance in context!", [tm]) |
|
222 |
| SOME instance => raw_ferrack_qe_conv ctxt instance tm); |
|
23466 | 223 |
|
23567 | 224 |
fun dlo_tac ctxt = CSUBGOAL (fn (p, i) => |
225 |
(case dlo_instance ctxt p of |
|
226 |
NONE => no_tac |
|
227 |
| SOME instance => |
|
35625 | 228 |
Object_Logic.full_atomize_tac i THEN |
23567 | 229 |
simp_tac (#simpset (snd instance)) i THEN (* FIXME already part of raw_ferrack_qe_conv? *) |
35625 | 230 |
CONVERSION (Object_Logic.judgment_conv (raw_ferrack_qe_conv ctxt instance)) i THEN |
32149
ef59550a55d3
renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;
wenzelm
parents:
30304
diff
changeset
|
231 |
simp_tac (simpset_of ctxt) i)); (* FIXME really? *) |
23466 | 232 |
|
233 |
end; |