author | oheimb |
Tue, 30 Jan 2001 18:47:00 +0100 | |
changeset 11000 | 498d0db8cd8a |
parent 10431 | bb67f704d631 |
child 11232 | 558a4feebb04 |
permissions | -rw-r--r-- |
9889 | 1 |
(* Title: FOL/simpdata.ML |
0 | 2 |
ID: $Id$ |
1459 | 3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
282 | 4 |
Copyright 1994 University of Cambridge |
0 | 5 |
|
9889 | 6 |
Simplification data for FOL. |
0 | 7 |
*) |
8 |
||
9300 | 9 |
|
5496 | 10 |
(* Elimination of True from asumptions: *) |
11 |
||
12 |
val True_implies_equals = prove_goal IFOL.thy |
|
13 |
"(True ==> PROP P) == PROP P" |
|
14 |
(K [rtac equal_intr_rule 1, atac 2, |
|
15 |
METAHYPS (fn prems => resolve_tac prems 1) 1, |
|
16 |
rtac TrueI 1]); |
|
17 |
||
18 |
||
0 | 19 |
(*** Rewrite rules ***) |
20 |
||
10431 | 21 |
fun int_prove_fun s = |
22 |
(writeln s; |
|
282 | 23 |
prove_goal IFOL.thy s |
10431 | 24 |
(fn prems => [ (cut_facts_tac prems 1), |
2601
b301958c465d
Renamed structure Int (intuitionistic prover) to IntPr to prevent clash
paulson
parents:
2469
diff
changeset
|
25 |
(IntPr.fast_tac 1) ])); |
0 | 26 |
|
1953 | 27 |
val conj_simps = map int_prove_fun |
1459 | 28 |
["P & True <-> P", "True & P <-> P", |
0 | 29 |
"P & False <-> False", "False & P <-> False", |
2801 | 30 |
"P & P <-> P", "P & P & Q <-> P & Q", |
1459 | 31 |
"P & ~P <-> False", "~P & P <-> False", |
0 | 32 |
"(P & Q) & R <-> P & (Q & R)"]; |
33 |
||
1953 | 34 |
val disj_simps = map int_prove_fun |
1459 | 35 |
["P | True <-> True", "True | P <-> True", |
36 |
"P | False <-> P", "False | P <-> P", |
|
2801 | 37 |
"P | P <-> P", "P | P | Q <-> P | Q", |
0 | 38 |
"(P | Q) | R <-> P | (Q | R)"]; |
39 |
||
1953 | 40 |
val not_simps = map int_prove_fun |
282 | 41 |
["~(P|Q) <-> ~P & ~Q", |
1459 | 42 |
"~ False <-> True", "~ True <-> False"]; |
0 | 43 |
|
1953 | 44 |
val imp_simps = map int_prove_fun |
1459 | 45 |
["(P --> False) <-> ~P", "(P --> True) <-> True", |
10431 | 46 |
"(False --> P) <-> True", "(True --> P) <-> P", |
1459 | 47 |
"(P --> P) <-> True", "(P --> ~P) <-> ~P"]; |
0 | 48 |
|
1953 | 49 |
val iff_simps = map int_prove_fun |
1459 | 50 |
["(True <-> P) <-> P", "(P <-> True) <-> P", |
0 | 51 |
"(P <-> P) <-> True", |
1459 | 52 |
"(False <-> P) <-> ~P", "(P <-> False) <-> ~P"]; |
0 | 53 |
|
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
54 |
(*The x=t versions are needed for the simplification procedures*) |
1953 | 55 |
val quant_simps = map int_prove_fun |
10431 | 56 |
["(ALL x. P) <-> P", |
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
57 |
"(ALL x. x=t --> P(x)) <-> P(t)", |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
58 |
"(ALL x. t=x --> P(x)) <-> P(t)", |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
59 |
"(EX x. P) <-> P", |
10431 | 60 |
"(EX x. x=t & P(x)) <-> P(t)", |
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
61 |
"(EX x. t=x & P(x)) <-> P(t)"]; |
0 | 62 |
|
63 |
(*These are NOT supplied by default!*) |
|
1953 | 64 |
val distrib_simps = map int_prove_fun |
10431 | 65 |
["P & (Q | R) <-> P&Q | P&R", |
282 | 66 |
"(Q | R) & P <-> Q&P | R&P", |
0 | 67 |
"(P | Q --> R) <-> (P --> R) & (Q --> R)"]; |
68 |
||
282 | 69 |
(** Conversion into rewrite rules **) |
0 | 70 |
|
53 | 71 |
fun gen_all th = forall_elim_vars (#maxidx(rep_thm th)+1) th; |
72 |
||
282 | 73 |
val P_iff_F = int_prove_fun "~P ==> (P <-> False)"; |
74 |
val iff_reflection_F = P_iff_F RS iff_reflection; |
|
75 |
||
76 |
val P_iff_T = int_prove_fun "P ==> (P <-> True)"; |
|
77 |
val iff_reflection_T = P_iff_T RS iff_reflection; |
|
78 |
||
79 |
(*Make meta-equalities. The operator below is Trueprop*) |
|
5555 | 80 |
|
282 | 81 |
fun mk_meta_eq th = case concl_of th of |
5555 | 82 |
_ $ (Const("op =",_)$_$_) => th RS eq_reflection |
83 |
| _ $ (Const("op <->",_)$_$_) => th RS iff_reflection |
|
10431 | 84 |
| _ => |
5555 | 85 |
error("conclusion must be a =-equality or <->");; |
86 |
||
87 |
fun mk_eq th = case concl_of th of |
|
394
432bb9995893
Modified mk_meta_eq to leave meta-equlities on unchanged.
nipkow
parents:
371
diff
changeset
|
88 |
Const("==",_)$_$_ => th |
5555 | 89 |
| _ $ (Const("op =",_)$_$_) => mk_meta_eq th |
90 |
| _ $ (Const("op <->",_)$_$_) => mk_meta_eq th |
|
282 | 91 |
| _ $ (Const("Not",_)$_) => th RS iff_reflection_F |
92 |
| _ => th RS iff_reflection_T; |
|
0 | 93 |
|
6114
45958e54d72e
congruence rules finally use == instead of = and <->
paulson
parents:
5555
diff
changeset
|
94 |
(*Replace premises x=y, X<->Y by X==Y*) |
10431 | 95 |
val mk_meta_prems = |
96 |
rule_by_tactic |
|
6114
45958e54d72e
congruence rules finally use == instead of = and <->
paulson
parents:
5555
diff
changeset
|
97 |
(REPEAT_FIRST (resolve_tac [meta_eq_to_obj_eq, def_imp_iff])); |
45958e54d72e
congruence rules finally use == instead of = and <->
paulson
parents:
5555
diff
changeset
|
98 |
|
9713 | 99 |
(*Congruence rules for = or <-> (instead of ==)*) |
6114
45958e54d72e
congruence rules finally use == instead of = and <->
paulson
parents:
5555
diff
changeset
|
100 |
fun mk_meta_cong rl = |
45958e54d72e
congruence rules finally use == instead of = and <->
paulson
parents:
5555
diff
changeset
|
101 |
standard(mk_meta_eq (mk_meta_prems rl)) |
45958e54d72e
congruence rules finally use == instead of = and <->
paulson
parents:
5555
diff
changeset
|
102 |
handle THM _ => |
45958e54d72e
congruence rules finally use == instead of = and <->
paulson
parents:
5555
diff
changeset
|
103 |
error("Premises and conclusion of congruence rules must use =-equality or <->"); |
5555 | 104 |
|
5304 | 105 |
val mksimps_pairs = |
106 |
[("op -->", [mp]), ("op &", [conjunct1,conjunct2]), |
|
107 |
("All", [spec]), ("True", []), ("False", [])]; |
|
108 |
||
5555 | 109 |
(* ###FIXME: move to Provers/simplifier.ML |
5304 | 110 |
val mk_atomize: (string * thm list) list -> thm -> thm list |
111 |
*) |
|
5555 | 112 |
(* ###FIXME: move to Provers/simplifier.ML *) |
5304 | 113 |
fun mk_atomize pairs = |
114 |
let fun atoms th = |
|
115 |
(case concl_of th of |
|
116 |
Const("Trueprop",_) $ p => |
|
117 |
(case head_of p of |
|
118 |
Const(a,_) => |
|
119 |
(case assoc(pairs,a) of |
|
120 |
Some(rls) => flat (map atoms ([th] RL rls)) |
|
121 |
| None => [th]) |
|
122 |
| _ => [th]) |
|
123 |
| _ => [th]) |
|
124 |
in atoms end; |
|
125 |
||
5555 | 126 |
fun mksimps pairs = (map mk_eq o mk_atomize pairs o gen_all); |
981 | 127 |
|
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
128 |
(*** Classical laws ***) |
282 | 129 |
|
10431 | 130 |
fun prove_fun s = |
131 |
(writeln s; |
|
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
6391
diff
changeset
|
132 |
prove_goal (the_context ()) s |
10431 | 133 |
(fn prems => [ (cut_facts_tac prems 1), |
1459 | 134 |
(Cla.fast_tac FOL_cs 1) ])); |
745 | 135 |
|
10431 | 136 |
(*Avoids duplication of subgoals after expand_if, when the true and false |
137 |
cases boil down to the same thing.*) |
|
1953 | 138 |
val cases_simp = prove_fun "(P --> Q) & (~P --> Q) <-> Q"; |
139 |
||
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
140 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
141 |
(*** Miniscoping: pushing quantifiers in |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
142 |
We do NOT distribute of ALL over &, or dually that of EX over | |
10431 | 143 |
Baaz and Leitsch, On Skolemization and Proof Complexity (1994) |
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
144 |
show that this step can increase proof length! |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
145 |
***) |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
146 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
147 |
(*existential miniscoping*) |
10431 | 148 |
val int_ex_simps = map int_prove_fun |
9713 | 149 |
["(EX x. P(x) & Q) <-> (EX x. P(x)) & Q", |
150 |
"(EX x. P & Q(x)) <-> P & (EX x. Q(x))", |
|
151 |
"(EX x. P(x) | Q) <-> (EX x. P(x)) | Q", |
|
152 |
"(EX x. P | Q(x)) <-> P | (EX x. Q(x))"]; |
|
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
153 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
154 |
(*classical rules*) |
10431 | 155 |
val cla_ex_simps = map prove_fun |
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
156 |
["(EX x. P(x) --> Q) <-> (ALL x. P(x)) --> Q", |
9713 | 157 |
"(EX x. P --> Q(x)) <-> P --> (EX x. Q(x))"]; |
0 | 158 |
|
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
159 |
val ex_simps = int_ex_simps @ cla_ex_simps; |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
160 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
161 |
(*universal miniscoping*) |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
162 |
val int_all_simps = map int_prove_fun |
9713 | 163 |
["(ALL x. P(x) & Q) <-> (ALL x. P(x)) & Q", |
164 |
"(ALL x. P & Q(x)) <-> P & (ALL x. Q(x))", |
|
165 |
"(ALL x. P(x) --> Q) <-> (EX x. P(x)) --> Q", |
|
166 |
"(ALL x. P --> Q(x)) <-> P --> (ALL x. Q(x))"]; |
|
1953 | 167 |
|
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
168 |
(*classical rules*) |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
169 |
val cla_all_simps = map prove_fun |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
170 |
["(ALL x. P(x) | Q) <-> (ALL x. P(x)) | Q", |
9713 | 171 |
"(ALL x. P | Q(x)) <-> P | (ALL x. Q(x))"]; |
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
172 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
173 |
val all_simps = int_all_simps @ cla_all_simps; |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
174 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
175 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
176 |
(*** Named rewrite rules proved for IFOL ***) |
1953 | 177 |
|
1914 | 178 |
fun int_prove nm thm = qed_goal nm IFOL.thy thm |
10431 | 179 |
(fn prems => [ (cut_facts_tac prems 1), |
2601
b301958c465d
Renamed structure Int (intuitionistic prover) to IntPr to prevent clash
paulson
parents:
2469
diff
changeset
|
180 |
(IntPr.fast_tac 1) ]); |
1914 | 181 |
|
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
6391
diff
changeset
|
182 |
fun prove nm thm = qed_goal nm (the_context ()) thm (fn _ => [Blast_tac 1]); |
1914 | 183 |
|
184 |
int_prove "conj_commute" "P&Q <-> Q&P"; |
|
185 |
int_prove "conj_left_commute" "P&(Q&R) <-> Q&(P&R)"; |
|
186 |
val conj_comms = [conj_commute, conj_left_commute]; |
|
187 |
||
188 |
int_prove "disj_commute" "P|Q <-> Q|P"; |
|
189 |
int_prove "disj_left_commute" "P|(Q|R) <-> Q|(P|R)"; |
|
190 |
val disj_comms = [disj_commute, disj_left_commute]; |
|
191 |
||
192 |
int_prove "conj_disj_distribL" "P&(Q|R) <-> (P&Q | P&R)"; |
|
193 |
int_prove "conj_disj_distribR" "(P|Q)&R <-> (P&R | Q&R)"; |
|
194 |
||
195 |
int_prove "disj_conj_distribL" "P|(Q&R) <-> (P|Q) & (P|R)"; |
|
196 |
int_prove "disj_conj_distribR" "(P&Q)|R <-> (P|R) & (Q|R)"; |
|
197 |
||
198 |
int_prove "imp_conj_distrib" "(P --> (Q&R)) <-> (P-->Q) & (P-->R)"; |
|
199 |
int_prove "imp_conj" "((P&Q)-->R) <-> (P --> (Q --> R))"; |
|
200 |
int_prove "imp_disj" "(P|Q --> R) <-> (P-->R) & (Q-->R)"; |
|
201 |
||
3910 | 202 |
prove "imp_disj1" "(P-->Q) | R <-> (P-->Q | R)"; |
203 |
prove "imp_disj2" "Q | (P-->R) <-> (P-->Q | R)"; |
|
204 |
||
1914 | 205 |
int_prove "de_Morgan_disj" "(~(P | Q)) <-> (~P & ~Q)"; |
206 |
prove "de_Morgan_conj" "(~(P & Q)) <-> (~P | ~Q)"; |
|
207 |
||
208 |
prove "not_iff" "~(P <-> Q) <-> (P <-> ~Q)"; |
|
209 |
||
3835 | 210 |
prove "not_all" "(~ (ALL x. P(x))) <-> (EX x.~P(x))"; |
211 |
prove "imp_all" "((ALL x. P(x)) --> Q) <-> (EX x. P(x) --> Q)"; |
|
212 |
int_prove "not_ex" "(~ (EX x. P(x))) <-> (ALL x.~P(x))"; |
|
1914 | 213 |
int_prove "imp_ex" "((EX x. P(x)) --> Q) <-> (ALL x. P(x) --> Q)"; |
214 |
||
215 |
int_prove "ex_disj_distrib" |
|
216 |
"(EX x. P(x) | Q(x)) <-> ((EX x. P(x)) | (EX x. Q(x)))"; |
|
217 |
int_prove "all_conj_distrib" |
|
218 |
"(ALL x. P(x) & Q(x)) <-> ((ALL x. P(x)) & (ALL x. Q(x)))"; |
|
219 |
||
220 |
||
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
221 |
(** make simplification procedures for quantifier elimination **) |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
222 |
structure Quantifier1 = Quantifier1Fun( |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
223 |
struct |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
224 |
(*abstract syntax*) |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
225 |
fun dest_eq((c as Const("op =",_)) $ s $ t) = Some(c,s,t) |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
226 |
| dest_eq _ = None; |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
227 |
fun dest_conj((c as Const("op &",_)) $ s $ t) = Some(c,s,t) |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
228 |
| dest_conj _ = None; |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
229 |
val conj = FOLogic.conj |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
230 |
val imp = FOLogic.imp |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
231 |
(*rules*) |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
232 |
val iff_reflection = iff_reflection |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
233 |
val iffI = iffI |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
234 |
val sym = sym |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
235 |
val conjI= conjI |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
236 |
val conjE= conjE |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
237 |
val impI = impI |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
238 |
val impE = impE |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
239 |
val mp = mp |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
240 |
val exI = exI |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
241 |
val exE = exE |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
242 |
val allI = allI |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
243 |
val allE = allE |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
244 |
end); |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
245 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
246 |
local |
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
6391
diff
changeset
|
247 |
|
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
248 |
val ex_pattern = |
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
6391
diff
changeset
|
249 |
read_cterm (Theory.sign_of (the_context ())) ("EX x. P(x) & Q(x)", FOLogic.oT) |
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
250 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
251 |
val all_pattern = |
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
6391
diff
changeset
|
252 |
read_cterm (Theory.sign_of (the_context ())) ("ALL x. P(x) & P'(x) --> Q(x)", FOLogic.oT) |
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
253 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
254 |
in |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
255 |
val defEX_regroup = |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
256 |
mk_simproc "defined EX" [ex_pattern] Quantifier1.rearrange_ex; |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
257 |
val defALL_regroup = |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
258 |
mk_simproc "defined ALL" [all_pattern] Quantifier1.rearrange_all; |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
259 |
end; |
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
260 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
261 |
|
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
262 |
(*** Case splitting ***) |
0 | 263 |
|
5304 | 264 |
val meta_eq_to_iff = prove_goal IFOL.thy "x==y ==> x<->y" |
265 |
(fn [prem] => [rewtac prem, rtac iffI 1, atac 1, atac 1]); |
|
1722 | 266 |
|
5304 | 267 |
structure SplitterData = |
268 |
struct |
|
269 |
structure Simplifier = Simplifier |
|
5555 | 270 |
val mk_eq = mk_eq |
5304 | 271 |
val meta_eq_to_iff = meta_eq_to_iff |
272 |
val iffD = iffD2 |
|
273 |
val disjE = disjE |
|
274 |
val conjE = conjE |
|
275 |
val exE = exE |
|
276 |
val contrapos = contrapos |
|
277 |
val contrapos2 = contrapos2 |
|
278 |
val notnotD = notnotD |
|
279 |
end; |
|
1722 | 280 |
|
5304 | 281 |
structure Splitter = SplitterFun(SplitterData); |
1722 | 282 |
|
5304 | 283 |
val split_tac = Splitter.split_tac; |
284 |
val split_inside_tac = Splitter.split_inside_tac; |
|
285 |
val split_asm_tac = Splitter.split_asm_tac; |
|
5307 | 286 |
val op addsplits = Splitter.addsplits; |
287 |
val op delsplits = Splitter.delsplits; |
|
5304 | 288 |
val Addsplits = Splitter.Addsplits; |
289 |
val Delsplits = Splitter.Delsplits; |
|
4325 | 290 |
|
291 |
||
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
292 |
(*** Standard simpsets ***) |
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
293 |
|
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
294 |
structure Induction = InductionFun(struct val spec=IFOL.spec end); |
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
295 |
|
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
296 |
open Induction; |
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
297 |
|
5555 | 298 |
|
5496 | 299 |
val meta_simps = |
300 |
[triv_forall_equality, (* prunes params *) |
|
301 |
True_implies_equals]; (* prune asms `True' *) |
|
302 |
||
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
303 |
val IFOL_simps = |
10431 | 304 |
[refl RS P_iff_T] @ conj_simps @ disj_simps @ not_simps @ |
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
305 |
imp_simps @ iff_simps @ quant_simps; |
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
306 |
|
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
307 |
val notFalseI = int_prove_fun "~False"; |
6114
45958e54d72e
congruence rules finally use == instead of = and <->
paulson
parents:
5555
diff
changeset
|
308 |
val triv_rls = [TrueI,refl,reflexive_thm,iff_refl,notFalseI]; |
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
309 |
|
2633
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
310 |
fun unsafe_solver prems = FIRST'[resolve_tac (triv_rls@prems), |
9713 | 311 |
atac, etac FalseE]; |
2633
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
312 |
(*No premature instantiation of variables during simplification*) |
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
313 |
fun safe_solver prems = FIRST'[match_tac (triv_rls@prems), |
9713 | 314 |
eq_assume_tac, ematch_tac [FalseE]]; |
2633
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
315 |
|
3910 | 316 |
(*No simprules, but basic infastructure for simplification*) |
10431 | 317 |
val FOL_basic_ss = empty_ss |
318 |
setsubgoaler asm_simp_tac |
|
319 |
setSSolver (mk_solver "FOL safe" safe_solver) |
|
320 |
setSolver (mk_solver "FOL unsafe" unsafe_solver) |
|
321 |
setmksimps (mksimps mksimps_pairs) |
|
322 |
setmkcong mk_meta_cong; |
|
5304 | 323 |
|
2633
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
324 |
|
3910 | 325 |
(*intuitionistic simprules only*) |
10431 | 326 |
val IFOL_ss = FOL_basic_ss |
327 |
addsimps (meta_simps @ IFOL_simps @ int_ex_simps @ int_all_simps) |
|
328 |
addsimprocs [defALL_regroup, defEX_regroup] |
|
329 |
addcongs [imp_cong]; |
|
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
330 |
|
9713 | 331 |
val cla_simps = |
3910 | 332 |
[de_Morgan_conj, de_Morgan_disj, imp_disj1, imp_disj2, |
333 |
not_all, not_ex, cases_simp] @ |
|
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
334 |
map prove_fun |
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
335 |
["~(P&Q) <-> ~P | ~Q", |
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
336 |
"P | ~P", "~P | P", |
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
337 |
"~ ~ P <-> P", "(~P --> P) <-> P", |
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
338 |
"(~P <-> ~Q) <-> (P<->Q)"]; |
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
339 |
|
3910 | 340 |
(*classical simprules too*) |
4349
50403e5a44c0
Instantiated the one-point-rule quantifier simpprocs for FOL
paulson
parents:
4325
diff
changeset
|
341 |
val FOL_ss = IFOL_ss addsimps (cla_simps @ cla_ex_simps @ cla_all_simps); |
2074
30a65172e003
Added the de Morgan laws (incl quantifier versions) to basic simpset
paulson
parents:
2065
diff
changeset
|
342 |
|
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
6391
diff
changeset
|
343 |
val simpsetup = [fn thy => (simpset_ref_of thy := FOL_ss; thy)]; |
2633
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
344 |
|
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
345 |
|
5219 | 346 |
(*** integration of simplifier with classical reasoner ***) |
2633
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
347 |
|
5219 | 348 |
structure Clasimp = ClasimpFun |
8472 | 349 |
(structure Simplifier = Simplifier and Splitter = Splitter |
9851 | 350 |
and Classical = Cla and Blast = Blast |
351 |
val dest_Trueprop = FOLogic.dest_Trueprop |
|
352 |
val iff_const = FOLogic.iff val not_const = FOLogic.not |
|
353 |
val notE = notE val iffD1 = iffD1 val iffD2 = iffD2 |
|
354 |
val cla_make_elim = cla_make_elim); |
|
4652
d24cca140eeb
factored out common code of HOL/simpdata.ML and FOL/simpdata.ML concerning
oheimb
parents:
4649
diff
changeset
|
355 |
open Clasimp; |
2633
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
356 |
|
37c0b5a7ee5d
added delcongs, Delcongs, unsafe_solver, safe_solver, FOL_basic_ss,
oheimb
parents:
2601
diff
changeset
|
357 |
val FOL_css = (FOL_cs, FOL_ss); |
9889 | 358 |
|
359 |
||
360 |
(* rulify setup *) |
|
361 |
||
362 |
local |
|
363 |
val ss = FOL_basic_ss addsimps (Drule.norm_hhf_eq :: map Thm.symmetric (thms "atomize")); |
|
364 |
in |
|
365 |
||
366 |
structure Rulify = RulifyFun |
|
367 |
(val make_meta = Simplifier.simplify ss |
|
368 |
val full_make_meta = Simplifier.full_simplify ss); |
|
369 |
||
370 |
structure BasicRulify: BASIC_RULIFY = Rulify; |
|
371 |
open BasicRulify; |
|
372 |
||
373 |
end; |