author | wenzelm |
Wed, 16 Nov 2005 17:45:26 +0100 | |
changeset 18180 | db712213504d |
parent 18145 | 6757627acf59 |
child 18207 | 9edbeda7e39a |
permissions | -rw-r--r-- |
17980 | 1 |
(* Title: Pure/goal.ML |
2 |
ID: $Id$ |
|
3 |
Author: Makarius and Lawrence C Paulson |
|
4 |
||
18139 | 5 |
Goals in tactical theorem proving. |
17980 | 6 |
*) |
7 |
||
8 |
signature BASIC_GOAL = |
|
9 |
sig |
|
10 |
val SELECT_GOAL: tactic -> int -> tactic |
|
11 |
end; |
|
12 |
||
13 |
signature GOAL = |
|
14 |
sig |
|
15 |
include BASIC_GOAL |
|
16 |
val init: cterm -> thm |
|
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
17 |
val protect: thm -> thm |
17980 | 18 |
val conclude: thm -> thm |
19 |
val finish: thm -> thm |
|
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
20 |
val norm_hhf: thm -> thm |
18180 | 21 |
val norm_hhf': thm -> thm |
18119 | 22 |
val compose_hhf: thm -> int -> thm -> thm Seq.seq |
23 |
val compose_hhf_tac: thm -> int -> tactic |
|
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
24 |
val comp_hhf: thm -> thm -> thm |
17980 | 25 |
val prove_multi: theory -> string list -> term list -> term list -> |
26 |
(thm list -> tactic) -> thm list |
|
18139 | 27 |
val prove: theory -> string list -> term list -> term -> (thm list -> tactic) -> thm |
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
28 |
val prove_raw: cterm list -> cterm -> (thm list -> tactic) -> thm |
17980 | 29 |
end; |
30 |
||
31 |
structure Goal: GOAL = |
|
32 |
struct |
|
33 |
||
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
34 |
(** goals **) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
35 |
|
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
36 |
(* |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
37 |
-------- (init) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
38 |
C ==> #C |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
39 |
*) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
40 |
fun init ct = Drule.instantiate' [] [SOME ct] Drule.protectI; |
17980 | 41 |
|
42 |
(* |
|
18119 | 43 |
C |
44 |
--- (protect) |
|
45 |
#C |
|
17980 | 46 |
*) |
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
47 |
fun protect th = th COMP Drule.incr_indexes th Drule.protectI; |
17980 | 48 |
|
49 |
(* |
|
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
50 |
A ==> ... ==> #C |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
51 |
---------------- (conclude) |
17980 | 52 |
A ==> ... ==> C |
53 |
*) |
|
54 |
fun conclude th = |
|
55 |
(case SINGLE (Thm.bicompose false (false, th, Thm.nprems_of th) 1) |
|
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
56 |
(Drule.incr_indexes th Drule.protectD) of |
17980 | 57 |
SOME th' => th' |
58 |
| NONE => raise THM ("Failed to conclude goal", 0, [th])); |
|
59 |
||
60 |
(* |
|
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
61 |
#C |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
62 |
--- (finish) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
63 |
C |
17983 | 64 |
*) |
17980 | 65 |
fun finish th = |
66 |
(case Thm.nprems_of th of |
|
67 |
0 => conclude th |
|
68 |
| n => raise THM ("Proof failed.\n" ^ |
|
69 |
Pretty.string_of (Pretty.chunks (Display.pretty_goals n th)) ^ |
|
70 |
("\n" ^ string_of_int n ^ " unsolved goal(s)!"), 0, [th])); |
|
71 |
||
72 |
||
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
73 |
|
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
74 |
(** results **) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
75 |
|
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
76 |
(* HHF normal form *) |
17980 | 77 |
|
18180 | 78 |
val norm_hhf_ss = |
79 |
MetaSimplifier.theory_context ProtoPure.thy MetaSimplifier.empty_ss |
|
80 |
addsimps [Drule.norm_hhf_eq]; |
|
81 |
||
82 |
val norm_hhf_ss' = norm_hhf_ss addeqcongs [Drule.protect_cong]; |
|
83 |
||
84 |
fun gen_norm_hhf protected = |
|
17980 | 85 |
(not o Drule.is_norm_hhf o Thm.prop_of) ? |
18180 | 86 |
Drule.fconv_rule (MetaSimplifier.rewrite_cterm (true, false, false) (K (K NONE)) |
87 |
(if protected then norm_hhf_ss else norm_hhf_ss')) |
|
17980 | 88 |
#> Thm.adjust_maxidx_thm |
89 |
#> Drule.gen_all; |
|
90 |
||
18180 | 91 |
val norm_hhf = gen_norm_hhf true; |
92 |
val norm_hhf' = gen_norm_hhf false; |
|
93 |
||
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
94 |
|
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
95 |
(* composition of normal results *) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
96 |
|
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
97 |
fun compose_hhf tha i thb = |
18145 | 98 |
Thm.bicompose false (false, Drule.lift_all (Thm.cprem_of thb i) tha, 0) i thb; |
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
99 |
|
18119 | 100 |
fun compose_hhf_tac th i = PRIMSEQ (compose_hhf th i); |
101 |
||
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
102 |
fun comp_hhf tha thb = |
18119 | 103 |
(case Seq.chop (2, compose_hhf tha 1 thb) of |
104 |
([th], _) => th |
|
105 |
| ([], _) => raise THM ("comp_hhf: no unifiers", 1, [tha, thb]) |
|
106 |
| _ => raise THM ("comp_hhf: multiple unifiers", 1, [tha, thb])); |
|
17986 | 107 |
|
108 |
||
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
109 |
|
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
110 |
(** tactical theorem proving **) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
111 |
|
18119 | 112 |
(* prove_multi *) |
17986 | 113 |
|
18119 | 114 |
fun prove_multi thy xs asms props tac = |
17980 | 115 |
let |
116 |
val prop = Logic.mk_conjunction_list props; |
|
117 |
val statement = Logic.list_implies (asms, prop); |
|
18139 | 118 |
val frees = Term.add_frees statement []; |
17980 | 119 |
val fixed_frees = filter_out (member (op =) xs o #1) frees; |
18139 | 120 |
val fixed_tfrees = fold (Term.add_tfreesT o #2) fixed_frees []; |
17980 | 121 |
val params = List.mapPartial (fn x => Option.map (pair x) (AList.lookup (op =) frees x)) xs; |
122 |
||
123 |
fun err msg = raise ERROR_MESSAGE |
|
124 |
(msg ^ "\nThe error(s) above occurred for the goal statement:\n" ^ |
|
125 |
Sign.string_of_term thy (Term.list_all_free (params, statement))); |
|
126 |
||
127 |
fun cert_safe t = Thm.cterm_of thy (Envir.beta_norm t) |
|
128 |
handle TERM (msg, _) => err msg | TYPE (msg, _, _) => err msg; |
|
129 |
||
130 |
val _ = cert_safe statement; |
|
131 |
val _ = Term.no_dummy_patterns statement handle TERM (msg, _) => err msg; |
|
132 |
||
133 |
val cparams = map (cert_safe o Free) params; |
|
134 |
val casms = map cert_safe asms; |
|
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
135 |
val prems = map (norm_hhf o Thm.assume) casms; |
17980 | 136 |
|
137 |
val goal = init (cert_safe prop); |
|
18119 | 138 |
val goal' = case SINGLE (tac prems) goal of SOME goal' => goal' | _ => err "Tactic failed."; |
17980 | 139 |
val raw_result = finish goal' handle THM (msg, _, _) => err msg; |
140 |
||
141 |
val prop' = Thm.prop_of raw_result; |
|
17986 | 142 |
val _ = conditional (not (Pattern.matches thy (Envir.beta_norm prop, prop'))) (fn () => |
17980 | 143 |
err ("Proved a different theorem: " ^ Sign.string_of_term thy prop')); |
144 |
in |
|
145 |
Drule.conj_elim_precise (length props) raw_result |
|
146 |
|> map |
|
147 |
(Drule.implies_intr_list casms |
|
148 |
#> Drule.forall_intr_list cparams |
|
18119 | 149 |
#> norm_hhf |
18139 | 150 |
#> Thm.varifyT' fixed_tfrees |
151 |
#-> K Drule.zero_var_indexes) |
|
17980 | 152 |
end; |
153 |
||
154 |
||
18119 | 155 |
(* prove *) |
17980 | 156 |
|
157 |
fun prove thy xs asms prop tac = hd (prove_multi thy xs asms [prop] tac); |
|
158 |
||
159 |
||
18027
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
160 |
(* prove_raw -- no checks, no normalization of result! *) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
161 |
|
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
162 |
fun prove_raw casms cprop tac = |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
163 |
(case SINGLE (tac (map (norm_hhf o Thm.assume) casms)) (init cprop) of |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
164 |
SOME th => Drule.implies_intr_list casms (finish th) |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
165 |
| NONE => raise ERROR_MESSAGE "Tactic failed."); |
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
166 |
|
09ab79d4e8e1
renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents:
17986
diff
changeset
|
167 |
|
17980 | 168 |
(* SELECT_GOAL *) |
169 |
||
170 |
(*Tactical for restricting the effect of a tactic to subgoal i. Works |
|
171 |
by making a new state from subgoal i, applying tac to it, and |
|
172 |
composing the resulting thm with the original state.*) |
|
173 |
||
174 |
fun SELECT tac i st = |
|
18145 | 175 |
init (Thm.adjust_maxidx (Thm.cprem_of st i)) |
17980 | 176 |
|> tac |
177 |
|> Seq.maps (fn st' => Thm.bicompose false (false, conclude st', Thm.nprems_of st') i st); |
|
178 |
||
179 |
fun SELECT_GOAL tac i st = |
|
180 |
let val n = Thm.nprems_of st in |
|
181 |
if 1 <= i andalso i <= n then |
|
182 |
if n = 1 then tac st else SELECT tac i st |
|
183 |
else Seq.empty |
|
184 |
end; |
|
185 |
||
186 |
end; |
|
187 |
||
188 |
structure BasicGoal: BASIC_GOAL = Goal; |
|
189 |
open BasicGoal; |