author | paulson |
Thu, 06 Jul 2000 13:28:36 +0200 | |
changeset 9264 | 051592f4236a |
parent 9158 | 084abf3d0eff |
child 9472 | b63b21f370ca |
permissions | -rw-r--r-- |
2469 | 1 |
(* Title: FOL/cladata.ML |
2 |
ID: $Id$ |
|
3 |
Author: Tobias Nipkow |
|
4 |
Copyright 1996 University of Cambridge |
|
5 |
||
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
7156
diff
changeset
|
6 |
Setting up the classical reasoner. |
2469 | 7 |
*) |
8 |
||
9 |
section "Classical Reasoner"; |
|
10 |
||
9158 | 11 |
(*** Applying Make_Elim_Fun to create a classical "make_elim" rule ***) |
12 |
structure Make_Elim_Data = |
|
13 |
struct |
|
14 |
val classical = classical |
|
15 |
end; |
|
16 |
||
17 |
structure Make_Elim = Make_Elim_Fun (Make_Elim_Data); |
|
18 |
||
19 |
(*we don't redeclare the original make_elim (Tactic.make_elim) for |
|
20 |
compatibliity with strange things done in many existing proofs *) |
|
21 |
val cla_make_elim = Make_Elim.make_elim; |
|
2844 | 22 |
|
2469 | 23 |
(*** Applying ClassicalFun to create a classical prover ***) |
24 |
structure Classical_Data = |
|
25 |
struct |
|
9158 | 26 |
val make_elim = cla_make_elim |
2469 | 27 |
val mp = mp |
28 |
val not_elim = notE |
|
29 |
val classical = classical |
|
9158 | 30 |
val sizef = size_of_thm |
2469 | 31 |
val hyp_subst_tacs=[hyp_subst_tac] |
32 |
end; |
|
33 |
||
34 |
structure Cla = ClassicalFun(Classical_Data); |
|
8099 | 35 |
structure BasicClassical: BASIC_CLASSICAL = Cla; open BasicClassical; |
36 |
structure Obtain = ObtainFun(val that_atts = [Simplifier.simp_add_local, Cla.haz_intro_local]); |
|
2469 | 37 |
|
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
7156
diff
changeset
|
38 |
|
2844 | 39 |
(*Better for fast_tac: needs no quantifier duplication!*) |
40 |
qed_goal "alt_ex1E" IFOL.thy |
|
3835 | 41 |
"[| EX! x. P(x); \ |
2844 | 42 |
\ !!x. [| P(x); ALL y y'. P(y) & P(y') --> y=y' |] ==> R \ |
43 |
\ |] ==> R" |
|
44 |
(fn major::prems => |
|
45 |
[ (rtac (major RS ex1E) 1), |
|
46 |
(REPEAT (ares_tac (allI::prems) 1)), |
|
47 |
(etac (dup_elim allE) 1), |
|
48 |
(IntPr.fast_tac 1)]); |
|
49 |
||
50 |
||
4305
03d7de40ee4f
The change from iffE to iffCE means fewer case splits in most cases. Very few
paulson
parents:
4095
diff
changeset
|
51 |
(*Propositional rules*) |
2469 | 52 |
val prop_cs = empty_cs addSIs [refl,TrueI,conjI,disjCI,impI,notI,iffI] |
4305
03d7de40ee4f
The change from iffE to iffCE means fewer case splits in most cases. Very few
paulson
parents:
4095
diff
changeset
|
53 |
addSEs [conjE,disjE,impCE,FalseE,iffCE]; |
2469 | 54 |
|
55 |
(*Quantifier rules*) |
|
2844 | 56 |
val FOL_cs = prop_cs addSIs [allI,ex_ex1I] addIs [exI] |
57 |
addSEs [exE,alt_ex1E] addEs [allE]; |
|
2469 | 58 |
|
7355
4c43090659ca
proper bootstrap of IFOL/FOL theories and packages;
wenzelm
parents:
7156
diff
changeset
|
59 |
val clasetup = [fn thy => (claset_ref_of thy := FOL_cs; thy)]; |