author | huffman |
Tue, 17 Apr 2007 00:37:14 +0200 | |
changeset 22720 | 296813d7d306 |
parent 22662 | 3e492ba59355 |
child 23178 | 07ba6b58b3d2 |
permissions | -rw-r--r-- |
11522 | 1 |
(* Title: Pure/Proof/proof_rewrite_rules.ML |
2 |
ID: $Id$ |
|
11539 | 3 |
Author: Stefan Berghofer, TU Muenchen |
11522 | 4 |
|
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
5 |
Simplification functions for proof terms involving meta level rules. |
11522 | 6 |
*) |
7 |
||
8 |
signature PROOF_REWRITE_RULES = |
|
9 |
sig |
|
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
10 |
val rew : bool -> typ list -> Proofterm.proof -> Proofterm.proof option |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
11 |
val rprocs : bool -> (string * (typ list -> Proofterm.proof -> Proofterm.proof option)) list |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
12 |
val rewrite_terms : (term -> term) -> Proofterm.proof -> Proofterm.proof |
17203 | 13 |
val elim_defs : theory -> bool -> thm list -> Proofterm.proof -> Proofterm.proof |
13608 | 14 |
val elim_vars : (typ -> term) -> Proofterm.proof -> Proofterm.proof |
22280 | 15 |
val hhf_proof : term -> term -> Proofterm.proof -> Proofterm.proof |
16 |
val un_hhf_proof : term -> term -> Proofterm.proof -> Proofterm.proof |
|
11522 | 17 |
end; |
18 |
||
19 |
structure ProofRewriteRules : PROOF_REWRITE_RULES = |
|
20 |
struct |
|
21 |
||
22 |
open Proofterm; |
|
23 |
||
19309 | 24 |
fun rew b _ = |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
25 |
let |
17137 | 26 |
fun ?? x = if b then SOME x else NONE; |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
27 |
fun ax (prf as PAxm (s, prop, _)) Ts = |
15531 | 28 |
if b then PAxm (s, prop, SOME Ts) else prf; |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
29 |
fun ty T = if b then |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
30 |
let val Type (_, [Type (_, [U, _]), _]) = T |
15531 | 31 |
in SOME U end |
32 |
else NONE; |
|
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
33 |
val equal_intr_axm = ax equal_intr_axm []; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
34 |
val equal_elim_axm = ax equal_elim_axm []; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
35 |
val symmetric_axm = ax symmetric_axm [propT]; |
11522 | 36 |
|
21646
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
37 |
fun rew' (PThm ("ProtoPure.protectD", _, _, _) % _ %% |
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
38 |
(PThm ("ProtoPure.protectI", _, _, _) % _ %% prf)) = SOME prf |
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
39 |
| rew' (PThm ("ProtoPure.conjunctionD1", _, _, _) % _ % _ %% |
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
40 |
(PThm ("ProtoPure.conjunctionI", _, _, _) % _ % _ %% prf %% _)) = SOME prf |
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
41 |
| rew' (PThm ("ProtoPure.conjunctionD2", _, _, _) % _ % _ %% |
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
42 |
(PThm ("ProtoPure.conjunctionI", _, _, _) % _ % _ %% _ %% prf)) = SOME prf |
19309 | 43 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % _ % _ %% |
15531 | 44 |
(PAxm ("ProtoPure.equal_intr", _, _) % _ % _ %% prf %% _)) = SOME prf |
19309 | 45 |
| rew' (PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
46 |
(PAxm ("ProtoPure.equal_intr", _, _) % A % B %% prf1 %% prf2)) = |
15531 | 47 |
SOME (equal_intr_axm % B % A %% prf2 %% prf1) |
12002 | 48 |
|
19309 | 49 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % SOME (_ $ A) % SOME (_ $ B) %% |
18024 | 50 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("prop", _)) % |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
51 |
_ % _ % _ %% (PAxm ("ProtoPure.reflexive", _, _) % _) %% prf1) %% |
21646
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
52 |
((tg as PThm ("ProtoPure.protectI", _, _, _)) % _ %% prf2)) = |
15531 | 53 |
SOME (tg %> B %% (equal_elim_axm %> A %> B %% prf1 %% prf2)) |
12002 | 54 |
|
19309 | 55 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % SOME (_ $ A) % SOME (_ $ B) %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
56 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
18024 | 57 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("prop", _)) % |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
58 |
_ % _ % _ %% (PAxm ("ProtoPure.reflexive", _, _) % _) %% prf1)) %% |
21646
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
59 |
((tg as PThm ("ProtoPure.protectI", _, _, _)) % _ %% prf2)) = |
15531 | 60 |
SOME (tg %> B %% (equal_elim_axm %> A %> B %% |
17137 | 61 |
(symmetric_axm % ?? B % ?? A %% prf1) %% prf2)) |
11522 | 62 |
|
19309 | 63 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % SOME X % SOME Y %% |
11612 | 64 |
(PAxm ("ProtoPure.combination", _, _) % _ % _ % _ % _ %% |
15531 | 65 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("==>", _)) % _ % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
66 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% prf1) %% prf2)) = |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
67 |
let |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
68 |
val _ $ A $ C = Envir.beta_norm X; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
69 |
val _ $ B $ D = Envir.beta_norm Y |
17137 | 70 |
in SOME (AbsP ("H1", ?? X, AbsP ("H2", ?? B, |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
71 |
equal_elim_axm %> C %> D %% incr_pboundvars 2 0 prf2 %% |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
72 |
(PBound 1 %% (equal_elim_axm %> B %> A %% |
17137 | 73 |
(symmetric_axm % ?? A % ?? B %% incr_pboundvars 2 0 prf1) %% PBound 0))))) |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
74 |
end |
11522 | 75 |
|
19309 | 76 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % SOME X % SOME Y %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
77 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
78 |
(PAxm ("ProtoPure.combination", _, _) % _ % _ % _ % _ %% |
15531 | 79 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("==>", _)) % _ % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
80 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% prf1) %% prf2))) = |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
81 |
let |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
82 |
val _ $ A $ C = Envir.beta_norm Y; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
83 |
val _ $ B $ D = Envir.beta_norm X |
17137 | 84 |
in SOME (AbsP ("H1", ?? X, AbsP ("H2", ?? A, |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
85 |
equal_elim_axm %> D %> C %% |
17137 | 86 |
(symmetric_axm % ?? C % ?? D %% incr_pboundvars 2 0 prf2) |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
87 |
%% (PBound 1 %% (equal_elim_axm %> A %> B %% incr_pboundvars 2 0 prf1 %% PBound 0))))) |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
88 |
end |
11522 | 89 |
|
19309 | 90 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % SOME X % SOME Y %% |
15531 | 91 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("all", _)) % _ % _ % _ %% |
11612 | 92 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
93 |
(PAxm ("ProtoPure.abstract_rule", _, _) % _ % _ %% prf))) = |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
94 |
let |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
95 |
val Const (_, T) $ P = Envir.beta_norm X; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
96 |
val _ $ Q = Envir.beta_norm Y; |
17137 | 97 |
in SOME (AbsP ("H", ?? X, Abst ("x", ty T, |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
98 |
equal_elim_axm %> incr_boundvars 1 P $ Bound 0 %> incr_boundvars 1 Q $ Bound 0 %% |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
99 |
(incr_pboundvars 1 1 prf %> Bound 0) %% (PBound 0 %> Bound 0)))) |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
100 |
end |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
101 |
|
19309 | 102 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % SOME X % SOME Y %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
103 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
15531 | 104 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("all", _)) % _ % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
105 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
106 |
(PAxm ("ProtoPure.abstract_rule", _, _) % _ % _ %% prf)))) = |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
107 |
let |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
108 |
val Const (_, T) $ P = Envir.beta_norm X; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
109 |
val _ $ Q = Envir.beta_norm Y; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
110 |
val t = incr_boundvars 1 P $ Bound 0; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
111 |
val u = incr_boundvars 1 Q $ Bound 0 |
17137 | 112 |
in SOME (AbsP ("H", ?? X, Abst ("x", ty T, |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
113 |
equal_elim_axm %> t %> u %% |
17137 | 114 |
(symmetric_axm % ?? u % ?? t %% (incr_pboundvars 1 1 prf %> Bound 0)) |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
115 |
%% (PBound 0 %> Bound 0)))) |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
116 |
end |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
117 |
|
19309 | 118 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % SOME A % SOME C %% |
15531 | 119 |
(PAxm ("ProtoPure.transitive", _, _) % _ % SOME B % _ %% prf1 %% prf2) %% prf3) = |
120 |
SOME (equal_elim_axm %> B %> C %% prf2 %% |
|
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
121 |
(equal_elim_axm %> A %> B %% prf1 %% prf3)) |
19309 | 122 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % SOME A % SOME C %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
123 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
15531 | 124 |
(PAxm ("ProtoPure.transitive", _, _) % _ % SOME B % _ %% prf1 %% prf2)) %% prf3) = |
17137 | 125 |
SOME (equal_elim_axm %> B %> C %% (symmetric_axm % ?? C % ?? B %% prf1) %% |
126 |
(equal_elim_axm %> A %> B %% (symmetric_axm % ?? B % ?? A %% prf2) %% prf3)) |
|
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
127 |
|
19309 | 128 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % _ % _ %% |
15531 | 129 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% prf) = SOME prf |
19309 | 130 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
131 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
15531 | 132 |
(PAxm ("ProtoPure.reflexive", _, _) % _)) %% prf) = SOME prf |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
133 |
|
19309 | 134 |
| rew' (PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
15531 | 135 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% prf)) = SOME prf |
11522 | 136 |
|
19309 | 137 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % _ % _ %% |
15531 | 138 |
(PAxm ("ProtoPure.equal_elim", _, _) % SOME (_ $ A $ C) % SOME (_ $ B $ D) %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
139 |
(PAxm ("ProtoPure.combination", _, _) % _ % _ % _ % _ %% |
15531 | 140 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("==", _)) % _ % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
141 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% prf1) %% prf2) %% prf3) %% prf4) = |
15531 | 142 |
SOME (equal_elim_axm %> C %> D %% prf2 %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
143 |
(equal_elim_axm %> A %> C %% prf3 %% |
17137 | 144 |
(equal_elim_axm %> B %> A %% (symmetric_axm % ?? A % ?? B %% prf1) %% prf4))) |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
145 |
|
19309 | 146 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
147 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
15531 | 148 |
(PAxm ("ProtoPure.equal_elim", _, _) % SOME (_ $ A $ C) % SOME (_ $ B $ D) %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
149 |
(PAxm ("ProtoPure.combination", _, _) % _ % _ % _ % _ %% |
15531 | 150 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("==", _)) % _ % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
151 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% prf1) %% prf2) %% prf3)) %% prf4) = |
15531 | 152 |
SOME (equal_elim_axm %> A %> B %% prf1 %% |
17137 | 153 |
(equal_elim_axm %> C %> A %% (symmetric_axm % ?? A % ?? C %% prf3) %% |
154 |
(equal_elim_axm %> D %> C %% (symmetric_axm % ?? C % ?? D %% prf2) %% prf4))) |
|
11522 | 155 |
|
19309 | 156 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % _ % _ %% |
15531 | 157 |
(PAxm ("ProtoPure.equal_elim", _, _) % SOME (_ $ B $ D) % SOME (_ $ A $ C) %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
158 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
159 |
(PAxm ("ProtoPure.combination", _, _) % _ % _ % _ % _ %% |
15531 | 160 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("==", _)) % _ % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
161 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% prf1) %% prf2)) %% prf3) %% prf4) = |
17137 | 162 |
SOME (equal_elim_axm %> D %> C %% (symmetric_axm % ?? C % ?? D %% prf2) %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
163 |
(equal_elim_axm %> B %> D %% prf3 %% |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
164 |
(equal_elim_axm %> A %> B %% prf1 %% prf4))) |
11522 | 165 |
|
19309 | 166 |
| rew' (PAxm ("ProtoPure.equal_elim", _, _) % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
167 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
15531 | 168 |
(PAxm ("ProtoPure.equal_elim", _, _) % SOME (_ $ B $ D) % SOME (_ $ A $ C) %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
169 |
(PAxm ("ProtoPure.symmetric", _, _) % _ % _ %% |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
170 |
(PAxm ("ProtoPure.combination", _, _) % _ % _ % _ % _ %% |
15531 | 171 |
(PAxm ("ProtoPure.combination", _, _) % SOME (Const ("==", _)) % _ % _ % _ %% |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
172 |
(PAxm ("ProtoPure.reflexive", _, _) % _) %% prf1) %% prf2)) %% prf3)) %% prf4) = |
17137 | 173 |
SOME (equal_elim_axm %> B %> A %% (symmetric_axm % ?? A % ?? B %% prf1) %% |
174 |
(equal_elim_axm %> D %> B %% (symmetric_axm % ?? B % ?? D %% prf3) %% |
|
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
175 |
(equal_elim_axm %> C %> D %% prf2 %% prf4))) |
11522 | 176 |
|
19309 | 177 |
| rew' ((prf as PAxm ("ProtoPure.combination", _, _) % |
15531 | 178 |
SOME ((eq as Const ("==", T)) $ t) % _ % _ % _) %% |
13257 | 179 |
(PAxm ("ProtoPure.reflexive", _, _) % _)) = |
180 |
let val (U, V) = (case T of |
|
181 |
Type (_, [U, V]) => (U, V) | _ => (dummyT, dummyT)) |
|
17137 | 182 |
in SOME (prf %% (ax combination_axm [V, U] %> eq % ?? eq % ?? t % ?? t %% |
183 |
(ax reflexive_axm [T] % ?? eq) %% (ax reflexive_axm [U] % ?? t))) |
|
13257 | 184 |
end |
185 |
||
19309 | 186 |
| rew' _ = NONE; |
12866
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
187 |
in rew' end; |
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
188 |
|
c00df7765656
Rewrite procedure now works for both compact and full proof objects.
berghofe
parents:
12237
diff
changeset
|
189 |
fun rprocs b = [("Pure/meta_equality", rew b)]; |
22662 | 190 |
val _ = Context.add_setup (fold Proofterm.add_prf_rproc (rprocs false)); |
11522 | 191 |
|
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
192 |
|
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
193 |
(**** apply rewriting function to all terms in proof ****) |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
194 |
|
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
195 |
fun rewrite_terms r = |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
196 |
let |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
197 |
fun rew_term Ts t = |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
198 |
let |
20076 | 199 |
val frees = map Free (Name.invent_list (add_term_names (t, [])) "xa" (length Ts) ~~ Ts); |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
200 |
val t' = r (subst_bounds (frees, t)); |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
201 |
fun strip [] t = t |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
202 |
| strip (_ :: xs) (Abs (_, _, t)) = strip xs t; |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
203 |
in |
19473 | 204 |
strip Ts (fold lambda frees t') |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
205 |
end; |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
206 |
|
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
207 |
fun rew Ts (prf1 %% prf2) = rew Ts prf1 %% rew Ts prf2 |
15531 | 208 |
| rew Ts (prf % SOME t) = rew Ts prf % SOME (rew_term Ts t) |
209 |
| rew Ts (Abst (s, SOME T, prf)) = Abst (s, SOME T, rew (T :: Ts) prf) |
|
210 |
| rew Ts (AbsP (s, SOME t, prf)) = AbsP (s, SOME (rew_term Ts t), rew Ts prf) |
|
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
211 |
| rew _ prf = prf |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
212 |
|
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
213 |
in rew [] end; |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
214 |
|
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
215 |
|
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
216 |
(**** eliminate definitions in proof ****) |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
217 |
|
16861 | 218 |
fun vars_of t = rev (fold_aterms (fn v as Var _ => insert (op =) v | _ => I) t []); |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
219 |
|
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
220 |
fun insert_refl defs Ts (prf1 %% prf2) = |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
221 |
insert_refl defs Ts prf1 %% insert_refl defs Ts prf2 |
15531 | 222 |
| insert_refl defs Ts (Abst (s, SOME T, prf)) = |
223 |
Abst (s, SOME T, insert_refl defs (T :: Ts) prf) |
|
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
224 |
| insert_refl defs Ts (AbsP (s, t, prf)) = |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
225 |
AbsP (s, t, insert_refl defs Ts prf) |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
226 |
| insert_refl defs Ts prf = (case strip_combt prf of |
21646
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
227 |
(PThm (s, _, prop, SOME Ts), ts) => |
20664 | 228 |
if member (op =) defs s then |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
229 |
let |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
230 |
val vs = vars_of prop; |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
231 |
val tvars = term_tvars prop; |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
232 |
val (_, rhs) = Logic.dest_equals prop; |
18185 | 233 |
val rhs' = Term.betapplys (subst_TVars (map fst tvars ~~ Ts) |
15574
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
234 |
(foldr (fn p => Abs ("", dummyT, abstract_over p)) rhs vs), |
19466 | 235 |
map the ts); |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
236 |
in |
15531 | 237 |
change_type (SOME [fastype_of1 (Ts, rhs')]) reflexive_axm %> rhs' |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
238 |
end |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
239 |
else prf |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
240 |
| (_, []) => prf |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
241 |
| (prf', ts) => proof_combt' (insert_refl defs Ts prf', ts)); |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
242 |
|
17203 | 243 |
fun elim_defs thy r defs prf = |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
244 |
let |
13341 | 245 |
val defs' = map (Logic.dest_equals o prop_of o Drule.abs_def) defs |
21646
c07b5b0e8492
thm/prf: separate official name vs. additional tags;
wenzelm
parents:
20664
diff
changeset
|
246 |
val defnames = map Thm.get_name defs; |
13341 | 247 |
val f = if not r then I else |
248 |
let |
|
249 |
val cnames = map (fst o dest_Const o fst) defs'; |
|
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19473
diff
changeset
|
250 |
val thms = maps (fn (s, ps) => |
20664 | 251 |
if member (op =) defnames s then [] |
15531 | 252 |
else map (pair s o SOME o fst) (filter_out (fn (p, _) => |
13646 | 253 |
null (term_consts p inter cnames)) ps)) |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19473
diff
changeset
|
254 |
(Symtab.dest (thms_of_proof prf Symtab.empty)) |
17203 | 255 |
in Reconstruct.expand_proof thy thms end |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
256 |
in |
17203 | 257 |
rewrite_terms (Pattern.rewrite_term thy defs' []) |
13341 | 258 |
(insert_refl defnames [] (f prf)) |
12906
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
259 |
end; |
165f4e1937f4
New function for eliminating definitions in proof term.
berghofe
parents:
12866
diff
changeset
|
260 |
|
13608 | 261 |
|
262 |
(**** eliminate all variables that don't occur in the proposition ****) |
|
263 |
||
264 |
fun elim_vars mk_default prf = |
|
265 |
let |
|
266 |
val prop = Reconstruct.prop_of prf; |
|
19309 | 267 |
val tv = Term.add_vars prop []; |
268 |
val tf = Term.add_frees prop []; |
|
269 |
||
270 |
fun hidden_variable (Var v) = not (member (op =) tv v) |
|
271 |
| hidden_variable (Free f) = not (member (op =) tf f) |
|
272 |
| hidden_variable _ = false; |
|
13917 | 273 |
|
274 |
fun mk_default' T = list_abs |
|
275 |
(apfst (map (pair "x")) (apsnd mk_default (strip_type T))); |
|
276 |
||
277 |
fun elim_varst (t $ u) = elim_varst t $ elim_varst u |
|
278 |
| elim_varst (Abs (s, T, t)) = Abs (s, T, elim_varst t) |
|
19309 | 279 |
| elim_varst (t as Free (x, T)) = if member (op =) tf (x, T) then t else mk_default' T |
280 |
| elim_varst (t as Var (xi, T)) = if member (op =) tv (xi, T) then t else mk_default' T |
|
281 |
| elim_varst t = t; |
|
13608 | 282 |
in |
19309 | 283 |
map_proof_terms (fn t => |
284 |
if Term.exists_subterm hidden_variable t then Envir.beta_norm (elim_varst t) else t) I prf |
|
13608 | 285 |
end; |
286 |
||
22280 | 287 |
|
288 |
(**** convert between hhf and non-hhf form ****) |
|
289 |
||
290 |
fun hhf_proof P Q prf = |
|
291 |
let |
|
292 |
val params = Logic.strip_params Q; |
|
293 |
val Hs = Logic.strip_assums_hyp P; |
|
294 |
val Hs' = Logic.strip_assums_hyp Q; |
|
295 |
val k = length Hs; |
|
296 |
val l = length params; |
|
297 |
fun mk_prf i j Hs Hs' (Const ("all", _) $ Abs (_, _, P)) prf = |
|
298 |
mk_prf i (j - 1) Hs Hs' P (prf %> Bound j) |
|
299 |
| mk_prf i j (H :: Hs) (H' :: Hs') (Const ("==>", _) $ _ $ P) prf = |
|
300 |
mk_prf (i - 1) j Hs Hs' P (prf %% un_hhf_proof H' H (PBound i)) |
|
301 |
| mk_prf _ _ _ _ _ prf = prf |
|
302 |
in |
|
303 |
prf |> Proofterm.incr_pboundvars k l |> mk_prf (k - 1) (l - 1) Hs Hs' P |> |
|
304 |
fold_rev (fn P => fn prf => AbsP ("H", SOME P, prf)) Hs' |> |
|
305 |
fold_rev (fn (s, T) => fn prf => Abst (s, SOME T, prf)) params |
|
306 |
end |
|
307 |
and un_hhf_proof P Q prf = |
|
308 |
let |
|
309 |
val params = Logic.strip_params Q; |
|
310 |
val Hs = Logic.strip_assums_hyp P; |
|
311 |
val Hs' = Logic.strip_assums_hyp Q; |
|
312 |
val k = length Hs; |
|
313 |
val l = length params; |
|
314 |
fun mk_prf (Const ("all", _) $ Abs (s, T, P)) prf = |
|
315 |
Abst (s, SOME T, mk_prf P prf) |
|
316 |
| mk_prf (Const ("==>", _) $ P $ Q) prf = |
|
317 |
AbsP ("H", SOME P, mk_prf Q prf) |
|
318 |
| mk_prf _ prf = prf |
|
319 |
in |
|
320 |
prf |> Proofterm.incr_pboundvars k l |> |
|
321 |
fold (fn i => fn prf => prf %> Bound i) (l - 1 downto 0) |> |
|
322 |
fold (fn ((H, H'), i) => fn prf => prf %% hhf_proof H' H (PBound i)) |
|
323 |
(Hs ~~ Hs' ~~ (k - 1 downto 0)) |> |
|
324 |
mk_prf Q |
|
325 |
end; |
|
326 |
||
11522 | 327 |
end; |