author | haftmann |
Fri, 24 Feb 2012 22:46:16 +0100 | |
changeset 46663 | 7fe029e818c2 |
parent 46218 | ecf6375e2abb |
child 46803 | f8875c15cbe1 |
permissions | -rw-r--r-- |
14620
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14518
diff
changeset
|
1 |
(* Title: HOL/Import/shuffler.ML |
14516 | 2 |
Author: Sebastian Skalberg, TU Muenchen |
3 |
||
4 |
Package for proving two terms equal by normalizing (hence the |
|
5 |
"shuffler" name). Uses the simplifier for the normalization. |
|
6 |
*) |
|
7 |
||
8 |
signature Shuffler = |
|
9 |
sig |
|
32740 | 10 |
val debug : bool Unsynchronized.ref |
14516 | 11 |
|
12 |
val norm_term : theory -> term -> thm |
|
13 |
val make_equal : theory -> term -> term -> thm option |
|
14 |
val set_prop : theory -> term -> (string * thm) list -> (string * thm) option |
|
15 |
||
16 |
val find_potential: theory -> term -> (string * thm) list |
|
17 |
||
31241 | 18 |
val gen_shuffle_tac: Proof.context -> bool -> (string * thm) list -> int -> tactic |
19 |
val shuffle_tac: Proof.context -> thm list -> int -> tactic |
|
20 |
val search_tac : Proof.context -> int -> tactic |
|
14516 | 21 |
|
22 |
val print_shuffles: theory -> unit |
|
23 |
||
24 |
val add_shuffle_rule: thm -> theory -> theory |
|
18728 | 25 |
val shuffle_attr: attribute |
14516 | 26 |
|
18708 | 27 |
val setup : theory -> theory |
14516 | 28 |
end |
29 |
||
30 |
structure Shuffler :> Shuffler = |
|
31 |
struct |
|
32 |
||
32740 | 33 |
val debug = Unsynchronized.ref false |
14516 | 34 |
|
35 |
fun if_debug f x = if !debug then f x else () |
|
36 |
val message = if_debug writeln |
|
37 |
||
37146
f652333bbf8e
renamed structure PrintMode to Print_Mode, keeping the old name as legacy alias for some time;
wenzelm
parents:
36945
diff
changeset
|
38 |
val string_of_thm = Print_Mode.setmp [] Display.string_of_thm_without_context; |
14516 | 39 |
|
33522 | 40 |
structure ShuffleData = Theory_Data |
22846 | 41 |
( |
42 |
type T = thm list |
|
43 |
val empty = [] |
|
44 |
val extend = I |
|
33522 | 45 |
val merge = Thm.merge_thms |
22846 | 46 |
) |
14516 | 47 |
|
22846 | 48 |
fun print_shuffles thy = |
49 |
Pretty.writeln (Pretty.big_list "Shuffle theorems:" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
31945
diff
changeset
|
50 |
(map (Display.pretty_thm_global thy) (ShuffleData.get thy))) |
14516 | 51 |
|
52 |
val weaken = |
|
53 |
let |
|
26424 | 54 |
val cert = cterm_of Pure.thy |
21588 | 55 |
val P = Free("P",propT) |
56 |
val Q = Free("Q",propT) |
|
57 |
val PQ = Logic.mk_implies(P,Q) |
|
58 |
val PPQ = Logic.mk_implies(P,PQ) |
|
59 |
val cP = cert P |
|
60 |
val cQ = cert Q |
|
61 |
val cPQ = cert PQ |
|
62 |
val cPPQ = cert PPQ |
|
36945 | 63 |
val th1 = Thm.assume cPQ |> implies_intr_list [cPQ,cP] |
64 |
val th3 = Thm.assume cP |
|
65 |
val th4 = implies_elim_list (Thm.assume cPPQ) [th3,th3] |
|
21588 | 66 |
|> implies_intr_list [cPPQ,cP] |
14516 | 67 |
in |
36945 | 68 |
Thm.equal_intr th4 th1 |> Drule.export_without_context |
14516 | 69 |
end |
70 |
||
71 |
val imp_comm = |
|
72 |
let |
|
26424 | 73 |
val cert = cterm_of Pure.thy |
21588 | 74 |
val P = Free("P",propT) |
75 |
val Q = Free("Q",propT) |
|
76 |
val R = Free("R",propT) |
|
77 |
val PQR = Logic.mk_implies(P,Logic.mk_implies(Q,R)) |
|
78 |
val QPR = Logic.mk_implies(Q,Logic.mk_implies(P,R)) |
|
79 |
val cP = cert P |
|
80 |
val cQ = cert Q |
|
81 |
val cPQR = cert PQR |
|
82 |
val cQPR = cert QPR |
|
36945 | 83 |
val th1 = implies_elim_list (Thm.assume cPQR) [Thm.assume cP,Thm.assume cQ] |
21588 | 84 |
|> implies_intr_list [cPQR,cQ,cP] |
36945 | 85 |
val th2 = implies_elim_list (Thm.assume cQPR) [Thm.assume cQ,Thm.assume cP] |
21588 | 86 |
|> implies_intr_list [cQPR,cP,cQ] |
14516 | 87 |
in |
36945 | 88 |
Thm.equal_intr th1 th2 |> Drule.export_without_context |
14516 | 89 |
end |
90 |
||
91 |
val all_comm = |
|
92 |
let |
|
26424 | 93 |
val cert = cterm_of Pure.thy |
21588 | 94 |
val xT = TFree("'a",[]) |
95 |
val yT = TFree("'b",[]) |
|
27330 | 96 |
val x = Free("x",xT) |
97 |
val y = Free("y",yT) |
|
21588 | 98 |
val P = Free("P",xT-->yT-->propT) |
27330 | 99 |
val lhs = Logic.all x (Logic.all y (P $ x $ y)) |
100 |
val rhs = Logic.all y (Logic.all x (P $ x $ y)) |
|
21588 | 101 |
val cl = cert lhs |
102 |
val cr = cert rhs |
|
27330 | 103 |
val cx = cert x |
104 |
val cy = cert y |
|
36945 | 105 |
val th1 = Thm.assume cr |
21588 | 106 |
|> forall_elim_list [cy,cx] |
107 |
|> forall_intr_list [cx,cy] |
|
36945 | 108 |
|> Thm.implies_intr cr |
109 |
val th2 = Thm.assume cl |
|
21588 | 110 |
|> forall_elim_list [cx,cy] |
111 |
|> forall_intr_list [cy,cx] |
|
36945 | 112 |
|> Thm.implies_intr cl |
14516 | 113 |
in |
36945 | 114 |
Thm.equal_intr th1 th2 |> Drule.export_without_context |
14516 | 115 |
end |
116 |
||
117 |
val equiv_comm = |
|
118 |
let |
|
26424 | 119 |
val cert = cterm_of Pure.thy |
21588 | 120 |
val T = TFree("'a",[]) |
121 |
val t = Free("t",T) |
|
122 |
val u = Free("u",T) |
|
123 |
val ctu = cert (Logic.mk_equals(t,u)) |
|
124 |
val cut = cert (Logic.mk_equals(u,t)) |
|
36945 | 125 |
val th1 = Thm.assume ctu |> Thm.symmetric |> Thm.implies_intr ctu |
126 |
val th2 = Thm.assume cut |> Thm.symmetric |> Thm.implies_intr cut |
|
14516 | 127 |
in |
36945 | 128 |
Thm.equal_intr th1 th2 |> Drule.export_without_context |
14516 | 129 |
end |
130 |
||
131 |
(* This simplification procedure rewrites !!x y. P x y |
|
132 |
deterministicly, in order for the normalization function, defined |
|
133 |
below, to handle nested quantifiers robustly *) |
|
134 |
||
135 |
local |
|
136 |
||
137 |
exception RESULT of int |
|
138 |
||
139 |
fun find_bound n (Bound i) = if i = n then raise RESULT 0 |
|
21588 | 140 |
else if i = n+1 then raise RESULT 1 |
141 |
else () |
|
14516 | 142 |
| find_bound n (t $ u) = (find_bound n t; find_bound n u) |
143 |
| find_bound n (Abs(_,_,t)) = find_bound (n+1) t |
|
144 |
| find_bound _ _ = () |
|
145 |
||
146 |
fun swap_bound n (Bound i) = if i = n then Bound (n+1) |
|
21588 | 147 |
else if i = n+1 then Bound n |
148 |
else Bound i |
|
14516 | 149 |
| swap_bound n (t $ u) = (swap_bound n t $ swap_bound n u) |
150 |
| swap_bound n (Abs(x,xT,t)) = Abs(x,xT,swap_bound (n+1) t) |
|
151 |
| swap_bound n t = t |
|
152 |
||
21078 | 153 |
fun rew_th thy (xv as (x,xT)) (yv as (y,yT)) t = |
14516 | 154 |
let |
46218
ecf6375e2abb
renamed Term.list_all to Logic.list_all, in accordance to HOLogic.list_all;
wenzelm
parents:
46201
diff
changeset
|
155 |
val lhs = Logic.list_all ([xv,yv],t) |
ecf6375e2abb
renamed Term.list_all to Logic.list_all, in accordance to HOLogic.list_all;
wenzelm
parents:
46201
diff
changeset
|
156 |
val rhs = Logic.list_all ([yv,xv],swap_bound 0 t) |
21588 | 157 |
val rew = Logic.mk_equals (lhs,rhs) |
36945 | 158 |
val init = Thm.trivial (cterm_of thy rew) |
14516 | 159 |
in |
37778
87b5dfe00387
do not intercept ML exceptions -- printing exception positions/text is the job of the Isar/ML toplevel;
wenzelm
parents:
37146
diff
changeset
|
160 |
all_comm RS init |
14516 | 161 |
end |
162 |
||
46201 | 163 |
fun quant_rewrite thy _ (t as Const("all",T1) $ (Abs(x,xT,Const("all",T2) $ Abs(y,yT,body)))) = |
14516 | 164 |
let |
21588 | 165 |
val res = (find_bound 0 body;2) handle RESULT i => i |
14516 | 166 |
in |
21588 | 167 |
case res of |
168 |
0 => SOME (rew_th thy (x,xT) (y,yT) body) |
|
169 |
| 1 => if string_ord(y,x) = LESS |
|
170 |
then |
|
171 |
let |
|
172 |
val newt = Const("all",T1) $ (Abs(y,xT,Const("all",T2) $ Abs(x,yT,body))) |
|
36945 | 173 |
val t_th = Thm.reflexive (cterm_of thy t) |
174 |
val newt_th = Thm.reflexive (cterm_of thy newt) |
|
21588 | 175 |
in |
36945 | 176 |
SOME (Thm.transitive t_th newt_th) |
21588 | 177 |
end |
178 |
else NONE |
|
179 |
| _ => error "norm_term (quant_rewrite) internal error" |
|
14516 | 180 |
end |
15531 | 181 |
| quant_rewrite _ _ _ = (warning "quant_rewrite: Unknown lhs"; NONE) |
14516 | 182 |
|
183 |
fun freeze_thaw_term t = |
|
184 |
let |
|
44121 | 185 |
val tvars = Misc_Legacy.term_tvars t |
186 |
val tfree_names = Misc_Legacy.add_term_tfree_names(t,[]) |
|
21588 | 187 |
val (type_inst,_) = |
33245 | 188 |
fold (fn (w as (v,_), S) => fn (inst, used) => |
21588 | 189 |
let |
43324
2b47822868e4
discontinued Name.variant to emphasize that this is old-style / indirect;
wenzelm
parents:
42368
diff
changeset
|
190 |
val v' = singleton (Name.variant_list used) v |
21588 | 191 |
in |
192 |
((w,TFree(v',S))::inst,v'::used) |
|
193 |
end) |
|
33245 | 194 |
tvars ([], tfree_names) |
21588 | 195 |
val t' = subst_TVars type_inst t |
14516 | 196 |
in |
33245 | 197 |
(t', map (fn (w,TFree(v,S)) => (v,TVar(w,S)) |
21588 | 198 |
| _ => error "Internal error in Shuffler.freeze_thaw") type_inst) |
14516 | 199 |
end |
200 |
||
21078 | 201 |
fun inst_tfrees thy [] thm = thm |
21588 | 202 |
| inst_tfrees thy ((name,U)::rest) thm = |
14516 | 203 |
let |
21588 | 204 |
val cU = ctyp_of thy U |
44121 | 205 |
val tfrees = Misc_Legacy.add_term_tfrees (prop_of thm,[]) |
35845
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
wenzelm
parents:
35408
diff
changeset
|
206 |
val (rens, thm') = Thm.varifyT_global' |
20951
868120282837
gen_rem(s) abandoned in favour of remove / subtract
haftmann
parents:
20897
diff
changeset
|
207 |
(remove (op = o apsnd fst) name tfrees) thm |
21588 | 208 |
val mid = |
209 |
case rens of |
|
210 |
[] => thm' |
|
43333
2bdec7f430d3
renamed Drule.instantiate to Drule.instantiate_normalize to emphasize its meaning as opposed to plain Thm.instantiate;
wenzelm
parents:
43324
diff
changeset
|
211 |
| [((_, S), idx)] => Drule.instantiate_normalize |
21078 | 212 |
([(ctyp_of thy (TVar (idx, S)), cU)], []) thm' |
21588 | 213 |
| _ => error "Shuffler.inst_tfrees internal error" |
14516 | 214 |
in |
21588 | 215 |
inst_tfrees thy rest mid |
14516 | 216 |
end |
217 |
||
218 |
fun is_Abs (Abs _) = true |
|
219 |
| is_Abs _ = false |
|
220 |
||
221 |
fun eta_redex (t $ Bound 0) = |
|
222 |
let |
|
21588 | 223 |
fun free n (Bound i) = i = n |
224 |
| free n (t $ u) = free n t orelse free n u |
|
225 |
| free n (Abs(_,_,t)) = free (n+1) t |
|
226 |
| free n _ = false |
|
14516 | 227 |
in |
21588 | 228 |
not (free 0 t) |
14516 | 229 |
end |
230 |
| eta_redex _ = false |
|
231 |
||
46201 | 232 |
fun eta_contract thy _ origt = |
14516 | 233 |
let |
21588 | 234 |
val (typet,Tinst) = freeze_thaw_term origt |
36945 | 235 |
val (init,thaw) = Drule.legacy_freeze_thaw (Thm.reflexive (cterm_of thy typet)) |
21588 | 236 |
val final = inst_tfrees thy Tinst o thaw |
237 |
val t = #1 (Logic.dest_equals (prop_of init)) |
|
238 |
val _ = |
|
239 |
let |
|
240 |
val lhs = #1 (Logic.dest_equals (prop_of (final init))) |
|
241 |
in |
|
242 |
if not (lhs aconv origt) |
|
32432
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
243 |
then |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
244 |
writeln (cat_lines |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
245 |
(["Something is utterly wrong: (orig, lhs, frozen type, t, tinst)", |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
246 |
Syntax.string_of_term_global thy origt, |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
247 |
Syntax.string_of_term_global thy lhs, |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
248 |
Syntax.string_of_term_global thy typet, |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
249 |
Syntax.string_of_term_global thy t] @ |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
250 |
map (fn (n, T) => n ^ ": " ^ Syntax.string_of_typ_global thy T) Tinst)) |
21588 | 251 |
else () |
252 |
end |
|
14516 | 253 |
in |
21588 | 254 |
case t of |
46201 | 255 |
Const("all",_) $ (Abs(x,xT,Const("==",_) $ P $ Q)) => |
37778
87b5dfe00387
do not intercept ML exceptions -- printing exception positions/text is the job of the Isar/ML toplevel;
wenzelm
parents:
37146
diff
changeset
|
256 |
(if eta_redex P andalso eta_redex Q |
21588 | 257 |
then |
258 |
let |
|
259 |
val cert = cterm_of thy |
|
43324
2b47822868e4
discontinued Name.variant to emphasize that this is old-style / indirect;
wenzelm
parents:
42368
diff
changeset
|
260 |
val v = Free (singleton (Name.variant_list (Term.add_free_names t [])) "v", xT) |
21588 | 261 |
val cv = cert v |
262 |
val ct = cert t |
|
36945 | 263 |
val th = (Thm.assume ct) |
264 |
|> Thm.forall_elim cv |
|
265 |
|> Thm.abstract_rule x cv |
|
266 |
val ext_th = Thm.eta_conversion (cert (Abs(x,xT,P))) |
|
267 |
val th' = Thm.transitive (Thm.symmetric ext_th) th |
|
21588 | 268 |
val cu = cert (prop_of th') |
36945 | 269 |
val uth = Thm.combination (Thm.assume cu) (Thm.reflexive cv) |
270 |
val uth' = (Thm.beta_conversion false (cert (Abs(x,xT,Q) $ v))) |
|
271 |
|> Thm.transitive uth |
|
272 |
|> Thm.forall_intr cv |
|
273 |
|> Thm.implies_intr cu |
|
274 |
val rew_th = Thm.equal_intr (th' |> Thm.implies_intr ct) uth' |
|
21588 | 275 |
val res = final rew_th |
276 |
in |
|
277 |
SOME res |
|
278 |
end |
|
279 |
else NONE) |
|
280 |
| _ => NONE |
|
17440
df77edc4f5d0
fixed HOL-light/Isabelle syntax incompatability via more protect_xxx functions
obua
parents:
17188
diff
changeset
|
281 |
end |
14516 | 282 |
|
46201 | 283 |
fun eta_expand thy _ origt = |
14516 | 284 |
let |
21588 | 285 |
val (typet,Tinst) = freeze_thaw_term origt |
36945 | 286 |
val (init,thaw) = Drule.legacy_freeze_thaw (Thm.reflexive (cterm_of thy typet)) |
21588 | 287 |
val final = inst_tfrees thy Tinst o thaw |
288 |
val t = #1 (Logic.dest_equals (prop_of init)) |
|
289 |
val _ = |
|
290 |
let |
|
291 |
val lhs = #1 (Logic.dest_equals (prop_of (final init))) |
|
292 |
in |
|
293 |
if not (lhs aconv origt) |
|
32432
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
294 |
then |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
295 |
writeln (cat_lines |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
296 |
(["Something is utterly wrong: (orig, lhs, frozen type, t, tinst)", |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
297 |
Syntax.string_of_term_global thy origt, |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
298 |
Syntax.string_of_term_global thy lhs, |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
299 |
Syntax.string_of_term_global thy typet, |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
300 |
Syntax.string_of_term_global thy t] @ |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
301 |
map (fn (n, T) => n ^ ": " ^ Syntax.string_of_typ_global thy T) Tinst)) |
21588 | 302 |
else () |
303 |
end |
|
14516 | 304 |
in |
21588 | 305 |
case t of |
306 |
Const("==",T) $ P $ Q => |
|
307 |
if is_Abs P orelse is_Abs Q |
|
308 |
then (case domain_type T of |
|
309 |
Type("fun",[aT,bT]) => |
|
310 |
let |
|
311 |
val cert = cterm_of thy |
|
43324
2b47822868e4
discontinued Name.variant to emphasize that this is old-style / indirect;
wenzelm
parents:
42368
diff
changeset
|
312 |
val vname = singleton (Name.variant_list (Term.add_free_names t [])) "v" |
21588 | 313 |
val v = Free(vname,aT) |
314 |
val cv = cert v |
|
315 |
val ct = cert t |
|
36945 | 316 |
val th1 = (Thm.combination (Thm.assume ct) (Thm.reflexive cv)) |
317 |
|> Thm.forall_intr cv |
|
318 |
|> Thm.implies_intr ct |
|
21588 | 319 |
val concl = cert (concl_of th1) |
36945 | 320 |
val th2 = (Thm.assume concl) |
321 |
|> Thm.forall_elim cv |
|
322 |
|> Thm.abstract_rule vname cv |
|
21588 | 323 |
val (lhs,rhs) = Logic.dest_equals (prop_of th2) |
36945 | 324 |
val elhs = Thm.eta_conversion (cert lhs) |
325 |
val erhs = Thm.eta_conversion (cert rhs) |
|
326 |
val th2' = Thm.transitive |
|
327 |
(Thm.transitive (Thm.symmetric elhs) th2) |
|
21588 | 328 |
erhs |
36945 | 329 |
val res = Thm.equal_intr th1 (th2' |> Thm.implies_intr concl) |
21588 | 330 |
val res' = final res |
331 |
in |
|
332 |
SOME res' |
|
333 |
end |
|
334 |
| _ => NONE) |
|
335 |
else NONE |
|
32432
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
336 |
| _ => error ("Bad eta_expand argument" ^ Syntax.string_of_term_global thy t) |
64f30bdd3ba1
modernized messages -- eliminated ctyp/cterm operations;
wenzelm
parents:
32091
diff
changeset
|
337 |
end; |
14516 | 338 |
|
14854 | 339 |
fun mk_tfree s = TFree("'"^s,[]) |
20326 | 340 |
fun mk_free s t = Free (s,t) |
14516 | 341 |
val xT = mk_tfree "a" |
342 |
val yT = mk_tfree "b" |
|
27330 | 343 |
val x = Free ("x", xT) |
344 |
val y = Free ("y", yT) |
|
20326 | 345 |
val P = mk_free "P" (xT-->yT-->propT) |
346 |
val Q = mk_free "Q" (xT-->yT) |
|
347 |
val R = mk_free "R" (xT-->yT) |
|
348 |
val S = mk_free "S" xT |
|
349 |
val S' = mk_free "S'" xT |
|
14516 | 350 |
in |
17188 | 351 |
|
38715
6513ea67d95d
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
wenzelm
parents:
38558
diff
changeset
|
352 |
fun quant_simproc thy = Simplifier.simproc_global_i |
21588 | 353 |
thy |
354 |
"Ordered rewriting of nested quantifiers" |
|
27330 | 355 |
[Logic.all x (Logic.all y (P $ x $ y))] |
21588 | 356 |
quant_rewrite |
38715
6513ea67d95d
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
wenzelm
parents:
38558
diff
changeset
|
357 |
fun eta_expand_simproc thy = Simplifier.simproc_global_i |
21588 | 358 |
thy |
359 |
"Smart eta-expansion by equivalences" |
|
360 |
[Logic.mk_equals(Q,R)] |
|
361 |
eta_expand |
|
38715
6513ea67d95d
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
wenzelm
parents:
38558
diff
changeset
|
362 |
fun eta_contract_simproc thy = Simplifier.simproc_global_i |
21588 | 363 |
thy |
364 |
"Smart handling of eta-contractions" |
|
27330 | 365 |
[Logic.all x (Logic.mk_equals (Q $ x, R $ x))] |
21588 | 366 |
eta_contract |
14516 | 367 |
end |
368 |
||
369 |
(* Disambiguates the names of bound variables in a term, returning t |
|
370 |
== t' where all the names of bound variables in t' are unique *) |
|
371 |
||
21078 | 372 |
fun disamb_bound thy t = |
14516 | 373 |
let |
21588 | 374 |
|
375 |
fun F (t $ u,idx) = |
|
376 |
let |
|
377 |
val (t',idx') = F (t,idx) |
|
378 |
val (u',idx'') = F (u,idx') |
|
379 |
in |
|
380 |
(t' $ u',idx'') |
|
381 |
end |
|
382 |
| F (Abs(x,xT,t),idx) = |
|
383 |
let |
|
41491 | 384 |
val x' = "x" ^ string_of_int idx |
21588 | 385 |
val (t',idx') = F (t,idx+1) |
386 |
in |
|
387 |
(Abs(x',xT,t'),idx') |
|
388 |
end |
|
389 |
| F arg = arg |
|
390 |
val (t',_) = F (t,0) |
|
391 |
val ct = cterm_of thy t |
|
392 |
val ct' = cterm_of thy t' |
|
36945 | 393 |
val res = Thm.transitive (Thm.reflexive ct) (Thm.reflexive ct') |
21588 | 394 |
val _ = message ("disamb_term: " ^ (string_of_thm res)) |
14516 | 395 |
in |
21588 | 396 |
res |
14516 | 397 |
end |
398 |
||
399 |
(* Transforms a term t to some normal form t', returning the theorem t |
|
400 |
== t'. This is originally a help function for make_equal, but might |
|
401 |
be handy in its own right, for example for indexing terms. *) |
|
402 |
||
403 |
fun norm_term thy t = |
|
404 |
let |
|
21588 | 405 |
val norms = ShuffleData.get thy |
35232
f588e1169c8b
renamed Simplifier.theory_context to Simplifier.global_context to emphasize that this is not the real thing;
wenzelm
parents:
35021
diff
changeset
|
406 |
val ss = Simplifier.global_context thy empty_ss |
21588 | 407 |
addsimps (map (Thm.transfer thy) norms) |
21078 | 408 |
addsimprocs [quant_simproc thy, eta_expand_simproc thy,eta_contract_simproc thy] |
21588 | 409 |
fun chain f th = |
410 |
let |
|
22902
ac833b4bb7ee
moved some Drule operations to Thm (see more_thm.ML);
wenzelm
parents:
22846
diff
changeset
|
411 |
val rhs = Thm.rhs_of th |
21588 | 412 |
in |
36945 | 413 |
Thm.transitive th (f rhs) |
21588 | 414 |
end |
415 |
val th = |
|
21078 | 416 |
t |> disamb_bound thy |
21588 | 417 |
|> chain (Simplifier.full_rewrite ss) |
36945 | 418 |
|> chain Thm.eta_conversion |
36614
b6c031ad3690
minor tuning of Thm.strip_shyps -- no longer pervasive;
wenzelm
parents:
36543
diff
changeset
|
419 |
|> Thm.strip_shyps |
21588 | 420 |
val _ = message ("norm_term: " ^ (string_of_thm th)) |
14516 | 421 |
in |
21588 | 422 |
th |
17463 | 423 |
end |
14516 | 424 |
|
425 |
||
426 |
(* Closes a theorem with respect to free and schematic variables (does |
|
427 |
not touch type variables, though). *) |
|
428 |
||
429 |
fun close_thm th = |
|
430 |
let |
|
22578 | 431 |
val thy = Thm.theory_of_thm th |
21588 | 432 |
val c = prop_of th |
44121 | 433 |
val vars = Misc_Legacy.add_term_frees (c, Misc_Legacy.add_term_vars(c,[])) |
14516 | 434 |
in |
21588 | 435 |
Drule.forall_intr_list (map (cterm_of thy) vars) th |
14516 | 436 |
end |
37778
87b5dfe00387
do not intercept ML exceptions -- printing exception positions/text is the job of the Isar/ML toplevel;
wenzelm
parents:
37146
diff
changeset
|
437 |
|
14516 | 438 |
|
439 |
(* Normalizes a theorem's conclusion using norm_term. *) |
|
440 |
||
441 |
fun norm_thm thy th = |
|
442 |
let |
|
21588 | 443 |
val c = prop_of th |
14516 | 444 |
in |
36945 | 445 |
Thm.equal_elim (norm_term thy c) th |
14516 | 446 |
end |
447 |
||
21078 | 448 |
(* make_equal thy t u tries to construct the theorem t == u under the |
449 |
signature thy. If it succeeds, SOME (t == u) is returned, otherwise |
|
15531 | 450 |
NONE is returned. *) |
14516 | 451 |
|
21078 | 452 |
fun make_equal thy t u = |
14516 | 453 |
let |
21588 | 454 |
val t_is_t' = norm_term thy t |
455 |
val u_is_u' = norm_term thy u |
|
36945 | 456 |
val th = Thm.transitive t_is_t' (Thm.symmetric u_is_u') |
21588 | 457 |
val _ = message ("make_equal: SOME " ^ (string_of_thm th)) |
14516 | 458 |
in |
21588 | 459 |
SOME th |
14516 | 460 |
end |
15531 | 461 |
handle e as THM _ => (message "make_equal: NONE";NONE) |
21588 | 462 |
|
14516 | 463 |
fun match_consts ignore t (* th *) = |
464 |
let |
|
21588 | 465 |
fun add_consts (Const (c, _), cs) = |
36692
54b64d4ad524
farewell to old-style mem infixes -- type inference in situations with mem_int and mem_string should provide enough information to resolve the type of (op =)
haftmann
parents:
36614
diff
changeset
|
466 |
if member (op =) ignore c |
21588 | 467 |
then cs |
468 |
else insert (op =) c cs |
|
469 |
| add_consts (t $ u, cs) = add_consts (t, add_consts (u, cs)) |
|
470 |
| add_consts (Abs (_, _, t), cs) = add_consts (t, cs) |
|
471 |
| add_consts (_, cs) = cs |
|
472 |
val t_consts = add_consts(t,[]) |
|
14516 | 473 |
in |
474 |
fn (name,th) => |
|
21588 | 475 |
let |
476 |
val th_consts = add_consts(prop_of th,[]) |
|
477 |
in |
|
33038 | 478 |
eq_set (op =) (t_consts, th_consts) |
21588 | 479 |
end |
14516 | 480 |
end |
21588 | 481 |
|
33040 | 482 |
val collect_ignored = fold_rev (fn thm => fn cs => |
483 |
let |
|
484 |
val (lhs, rhs) = Logic.dest_equals (prop_of thm); |
|
485 |
val consts_lhs = Term.add_const_names lhs []; |
|
486 |
val consts_rhs = Term.add_const_names rhs []; |
|
487 |
val ignore_lhs = subtract (op =) consts_rhs consts_lhs; |
|
488 |
val ignore_rhs = subtract (op =) consts_lhs consts_rhs; |
|
489 |
in |
|
490 |
fold_rev (insert (op =)) cs (ignore_lhs @ ignore_rhs) |
|
491 |
end) |
|
14516 | 492 |
|
493 |
(* set_prop t thms tries to make a theorem with the proposition t from |
|
494 |
one of the theorems thms, by shuffling the propositions around. If it |
|
15531 | 495 |
succeeds, SOME theorem is returned, otherwise NONE. *) |
14516 | 496 |
|
497 |
fun set_prop thy t = |
|
498 |
let |
|
44121 | 499 |
val vars = Misc_Legacy.add_term_frees (t, Misc_Legacy.add_term_vars (t,[])) |
27330 | 500 |
val closed_t = fold_rev Logic.all vars t |
21588 | 501 |
val rew_th = norm_term thy closed_t |
22902
ac833b4bb7ee
moved some Drule operations to Thm (see more_thm.ML);
wenzelm
parents:
22846
diff
changeset
|
502 |
val rhs = Thm.rhs_of rew_th |
14516 | 503 |
|
21588 | 504 |
fun process [] = NONE |
505 |
| process ((name,th)::thms) = |
|
506 |
let |
|
35845
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
wenzelm
parents:
35408
diff
changeset
|
507 |
val norm_th = Thm.varifyT_global (norm_thm thy (close_thm (Thm.transfer thy th))) |
36945 | 508 |
val triv_th = Thm.trivial rhs |
21588 | 509 |
val _ = message ("Shuffler.set_prop: Gluing together " ^ (string_of_thm norm_th) ^ " and " ^ (string_of_thm triv_th)) |
31945 | 510 |
val mod_th = case Seq.pull (Thm.bicompose false (*true*) (false,norm_th,0) 1 triv_th) of |
21588 | 511 |
SOME(th,_) => SOME th |
512 |
| NONE => NONE |
|
513 |
in |
|
514 |
case mod_th of |
|
515 |
SOME mod_th => |
|
516 |
let |
|
36945 | 517 |
val closed_th = Thm.equal_elim (Thm.symmetric rew_th) mod_th |
21588 | 518 |
in |
519 |
message ("Shuffler.set_prop succeeded by " ^ name); |
|
520 |
SOME (name,forall_elim_list (map (cterm_of thy) vars) closed_th) |
|
521 |
end |
|
522 |
| NONE => process thms |
|
523 |
end |
|
524 |
handle e as THM _ => process thms |
|
14516 | 525 |
in |
21588 | 526 |
fn thms => |
527 |
case process thms of |
|
528 |
res as SOME (name,th) => if (prop_of th) aconv t |
|
529 |
then res |
|
530 |
else error "Internal error in set_prop" |
|
531 |
| NONE => NONE |
|
14516 | 532 |
end |
533 |
||
534 |
fun find_potential thy t = |
|
535 |
let |
|
21588 | 536 |
val shuffles = ShuffleData.get thy |
537 |
val ignored = collect_ignored shuffles [] |
|
26662 | 538 |
val all_thms = |
39557
fe5722fce758
renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
wenzelm
parents:
39159
diff
changeset
|
539 |
map (`Thm.get_name_hint) (maps #2 (Facts.dest_static [] (Global_Theory.facts_of thy))) |
14516 | 540 |
in |
33317 | 541 |
filter (match_consts ignored t) all_thms |
14516 | 542 |
end |
543 |
||
42368
3b8498ac2314
proper subgoal addressing via SUBGOAL/CSUBGOAL -- assuming these tactics did not handle Subscript in any special way;
wenzelm
parents:
42364
diff
changeset
|
544 |
fun gen_shuffle_tac ctxt search thms = SUBGOAL (fn (t, i) => |
14516 | 545 |
let |
42361 | 546 |
val thy = Proof_Context.theory_of ctxt |
21588 | 547 |
val set = set_prop thy t |
548 |
fun process_tac thms st = |
|
549 |
case set thms of |
|
550 |
SOME (_,th) => Seq.of_list (compose (th,i,st)) |
|
551 |
| NONE => Seq.empty |
|
14516 | 552 |
in |
42368
3b8498ac2314
proper subgoal addressing via SUBGOAL/CSUBGOAL -- assuming these tactics did not handle Subscript in any special way;
wenzelm
parents:
42364
diff
changeset
|
553 |
process_tac thms APPEND |
3b8498ac2314
proper subgoal addressing via SUBGOAL/CSUBGOAL -- assuming these tactics did not handle Subscript in any special way;
wenzelm
parents:
42364
diff
changeset
|
554 |
(if search then process_tac (find_potential thy t) else no_tac) |
3b8498ac2314
proper subgoal addressing via SUBGOAL/CSUBGOAL -- assuming these tactics did not handle Subscript in any special way;
wenzelm
parents:
42364
diff
changeset
|
555 |
end) |
14516 | 556 |
|
31244
4ed31c673baf
fixed superficial ML lapses introduced in b3c7044d47b6;
wenzelm
parents:
31241
diff
changeset
|
557 |
fun shuffle_tac ctxt thms = |
4ed31c673baf
fixed superficial ML lapses introduced in b3c7044d47b6;
wenzelm
parents:
31241
diff
changeset
|
558 |
gen_shuffle_tac ctxt false (map (pair "") thms); |
4ed31c673baf
fixed superficial ML lapses introduced in b3c7044d47b6;
wenzelm
parents:
31241
diff
changeset
|
559 |
|
4ed31c673baf
fixed superficial ML lapses introduced in b3c7044d47b6;
wenzelm
parents:
31241
diff
changeset
|
560 |
fun search_tac ctxt = |
4ed31c673baf
fixed superficial ML lapses introduced in b3c7044d47b6;
wenzelm
parents:
31241
diff
changeset
|
561 |
gen_shuffle_tac ctxt true (map (pair "premise") (Assumption.all_prems_of ctxt)); |
14516 | 562 |
|
563 |
fun add_shuffle_rule thm thy = |
|
564 |
let |
|
21588 | 565 |
val shuffles = ShuffleData.get thy |
14516 | 566 |
in |
21588 | 567 |
if exists (curry Thm.eq_thm thm) shuffles |
568 |
then (warning ((string_of_thm thm) ^ " already known to the shuffler"); |
|
569 |
thy) |
|
570 |
else ShuffleData.put (thm::shuffles) thy |
|
14516 | 571 |
end |
572 |
||
20897 | 573 |
val shuffle_attr = Thm.declaration_attribute (fn th => Context.mapping (add_shuffle_rule th) I); |
14516 | 574 |
|
18708 | 575 |
val setup = |
31241 | 576 |
Method.setup @{binding shuffle_tac} |
31244
4ed31c673baf
fixed superficial ML lapses introduced in b3c7044d47b6;
wenzelm
parents:
31241
diff
changeset
|
577 |
(Attrib.thms >> (fn ths => fn ctxt => SIMPLE_METHOD' (shuffle_tac ctxt ths))) |
31241 | 578 |
"solve goal by shuffling terms around" #> |
579 |
Method.setup @{binding search_tac} |
|
580 |
(Scan.succeed (SIMPLE_METHOD' o search_tac)) "search for suitable theorems" #> |
|
18708 | 581 |
add_shuffle_rule weaken #> |
582 |
add_shuffle_rule equiv_comm #> |
|
583 |
add_shuffle_rule imp_comm #> |
|
584 |
add_shuffle_rule Drule.norm_hhf_eq #> |
|
585 |
add_shuffle_rule Drule.triv_forall_equality #> |
|
30528 | 586 |
Attrib.setup @{binding shuffle_rule} (Scan.succeed shuffle_attr) "declare rule for shuffler"; |
18708 | 587 |
|
14516 | 588 |
end |