author | wenzelm |
Tue, 29 Dec 2015 16:23:34 +0100 | |
changeset 61959 | 364007370bb7 |
parent 61841 | 4d3527b94f2a |
child 62916 | 621afc4607ec |
permissions | -rw-r--r-- |
32169 | 1 |
(* Title: Pure/tactical.ML |
2244
dacee519738a
Converted I/O operatios for Basis Library compatibility
paulson
parents:
2158
diff
changeset
|
2 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
0 | 3 |
|
16179 | 4 |
Tacticals. |
0 | 5 |
*) |
6 |
||
4602 | 7 |
infix 1 THEN THEN' THEN_ALL_NEW; |
46463 | 8 |
infix 0 ORELSE APPEND ORELSE' APPEND'; |
671 | 9 |
infix 0 THEN_ELSE; |
10 |
||
0 | 11 |
signature TACTICAL = |
11916 | 12 |
sig |
23538 | 13 |
type tactic = thm -> thm Seq.seq |
14 |
val THEN: tactic * tactic -> tactic |
|
15 |
val ORELSE: tactic * tactic -> tactic |
|
16 |
val APPEND: tactic * tactic -> tactic |
|
17 |
val THEN_ELSE: tactic * (tactic*tactic) -> tactic |
|
18 |
val THEN': ('a -> tactic) * ('a -> tactic) -> 'a -> tactic |
|
19 |
val ORELSE': ('a -> tactic) * ('a -> tactic) -> 'a -> tactic |
|
20 |
val APPEND': ('a -> tactic) * ('a -> tactic) -> 'a -> tactic |
|
21 |
val all_tac: tactic |
|
22 |
val no_tac: tactic |
|
23 |
val DETERM: tactic -> tactic |
|
24 |
val COND: (thm -> bool) -> tactic -> tactic -> tactic |
|
25 |
val TRY: tactic -> tactic |
|
26 |
val EVERY: tactic list -> tactic |
|
27 |
val EVERY': ('a -> tactic) list -> 'a -> tactic |
|
28 |
val EVERY1: (int -> tactic) list -> tactic |
|
29 |
val FIRST: tactic list -> tactic |
|
30 |
val FIRST': ('a -> tactic) list -> 'a -> tactic |
|
31 |
val FIRST1: (int -> tactic) list -> tactic |
|
32 |
val RANGE: (int -> tactic) list -> int -> tactic |
|
56491 | 33 |
val print_tac: Proof.context -> string -> tactic |
23538 | 34 |
val pause_tac: tactic |
32738 | 35 |
val trace_REPEAT: bool Unsynchronized.ref |
36 |
val suppress_tracing: bool Unsynchronized.ref |
|
37 |
val tracify: bool Unsynchronized.ref -> tactic -> tactic |
|
23538 | 38 |
val traced_tac: (thm -> (thm * thm Seq.seq) option) -> tactic |
39 |
val REPEAT_DETERM_N: int -> tactic -> tactic |
|
40 |
val REPEAT_DETERM: tactic -> tactic |
|
41 |
val REPEAT: tactic -> tactic |
|
42 |
val REPEAT_DETERM1: tactic -> tactic |
|
43 |
val REPEAT1: tactic -> tactic |
|
44 |
val FILTER: (thm -> bool) -> tactic -> tactic |
|
45 |
val CHANGED: tactic -> tactic |
|
46 |
val CHANGED_PROP: tactic -> tactic |
|
47 |
val ALLGOALS: (int -> tactic) -> tactic |
|
48 |
val SOMEGOAL: (int -> tactic) -> tactic |
|
49 |
val FIRSTGOAL: (int -> tactic) -> tactic |
|
61841
4d3527b94f2a
more general types Proof.method / context_tactic;
wenzelm
parents:
60941
diff
changeset
|
50 |
val HEADGOAL: (int -> tactic) -> tactic |
23538 | 51 |
val REPEAT_SOME: (int -> tactic) -> tactic |
52 |
val REPEAT_DETERM_SOME: (int -> tactic) -> tactic |
|
53 |
val REPEAT_FIRST: (int -> tactic) -> tactic |
|
703
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
lcp
parents:
671
diff
changeset
|
54 |
val REPEAT_DETERM_FIRST: (int -> tactic) -> tactic |
23538 | 55 |
val TRYALL: (int -> tactic) -> tactic |
56 |
val CSUBGOAL: ((cterm * int) -> tactic) -> int -> tactic |
|
57 |
val SUBGOAL: ((term * int) -> tactic) -> int -> tactic |
|
49865 | 58 |
val ASSERT_SUBGOAL: (int -> tactic) -> int -> tactic |
23538 | 59 |
val CHANGED_GOAL: (int -> tactic) -> int -> tactic |
34885
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
60 |
val SOLVED': (int -> tactic) -> int -> tactic |
23538 | 61 |
val THEN_ALL_NEW: (int -> tactic) * (int -> tactic) -> int -> tactic |
62 |
val REPEAT_ALL_NEW: (int -> tactic) -> int -> tactic |
|
63 |
val PRIMSEQ: (thm -> thm Seq.seq) -> tactic |
|
64 |
val PRIMITIVE: (thm -> thm) -> tactic |
|
65 |
val SINGLE: tactic -> thm -> thm option |
|
66 |
val CONVERSION: conv -> int -> tactic |
|
11916 | 67 |
end; |
0 | 68 |
|
13108 | 69 |
structure Tactical : TACTICAL = |
0 | 70 |
struct |
71 |
||
72 |
(**** Tactics ****) |
|
73 |
||
74 |
(*A tactic maps a proof tree to a sequence of proof trees: |
|
75 |
if length of sequence = 0 then the tactic does not apply; |
|
76 |
if length > 1 then backtracking on the alternatives can occur.*) |
|
77 |
||
4270 | 78 |
type tactic = thm -> thm Seq.seq; |
0 | 79 |
|
80 |
||
81 |
(*** LCF-style tacticals ***) |
|
82 |
||
83 |
(*the tactical THEN performs one tactic followed by another*) |
|
17344 | 84 |
fun (tac1 THEN tac2) st = Seq.maps tac2 (tac1 st); |
0 | 85 |
|
86 |
||
87 |
(*The tactical ORELSE uses the first tactic that returns a nonempty sequence. |
|
88 |
Like in LCF, ORELSE commits to either tac1 or tac2 immediately. |
|
89 |
Does not backtrack to tac2 if tac1 was initially chosen. *) |
|
1502 | 90 |
fun (tac1 ORELSE tac2) st = |
60941 | 91 |
(case Seq.pull (tac1 st) of |
92 |
NONE => tac2 st |
|
93 |
| some => Seq.make (fn () => some)); |
|
0 | 94 |
|
95 |
||
96 |
(*The tactical APPEND combines the results of two tactics. |
|
97 |
Like ORELSE, but allows backtracking on both tac1 and tac2. |
|
98 |
The tactic tac2 is not applied until needed.*) |
|
13108 | 99 |
fun (tac1 APPEND tac2) st = |
19861 | 100 |
Seq.append (tac1 st) (Seq.make(fn()=> Seq.pull (tac2 st))); |
0 | 101 |
|
671 | 102 |
(*Conditional tactic. |
2244
dacee519738a
Converted I/O operatios for Basis Library compatibility
paulson
parents:
2158
diff
changeset
|
103 |
tac1 ORELSE tac2 = tac1 THEN_ELSE (all_tac, tac2) |
dacee519738a
Converted I/O operatios for Basis Library compatibility
paulson
parents:
2158
diff
changeset
|
104 |
tac1 THEN tac2 = tac1 THEN_ELSE (tac2, no_tac) |
671 | 105 |
*) |
13108 | 106 |
fun (tac THEN_ELSE (tac1, tac2)) st = |
60941 | 107 |
(case Seq.pull (tac st) of |
108 |
NONE => tac2 st (*failed; try tactic 2*) |
|
109 |
| some => Seq.maps tac1 (Seq.make (fn () => some))); (*succeeded; use tactic 1*) |
|
671 | 110 |
|
111 |
||
0 | 112 |
(*Versions for combining tactic-valued functions, as in |
113 |
SOMEGOAL (resolve_tac rls THEN' assume_tac) *) |
|
1502 | 114 |
fun (tac1 THEN' tac2) x = tac1 x THEN tac2 x; |
115 |
fun (tac1 ORELSE' tac2) x = tac1 x ORELSE tac2 x; |
|
116 |
fun (tac1 APPEND' tac2) x = tac1 x APPEND tac2 x; |
|
0 | 117 |
|
118 |
(*passes all proofs through unchanged; identity of THEN*) |
|
4270 | 119 |
fun all_tac st = Seq.single st; |
0 | 120 |
|
121 |
(*passes no proofs through; identity of ORELSE and APPEND*) |
|
4270 | 122 |
fun no_tac st = Seq.empty; |
0 | 123 |
|
124 |
||
125 |
(*Make a tactic deterministic by chopping the tail of the proof sequence*) |
|
12851 | 126 |
fun DETERM tac = Seq.DETERM tac; |
0 | 127 |
|
128 |
(*Conditional tactical: testfun controls which tactic to use next. |
|
129 |
Beware: due to eager evaluation, both thentac and elsetac are evaluated.*) |
|
60941 | 130 |
fun COND testfun thenf elsef = |
131 |
(fn st => if testfun st then thenf st else elsef st); |
|
0 | 132 |
|
133 |
(*Do the tactic or else do nothing*) |
|
134 |
fun TRY tac = tac ORELSE all_tac; |
|
135 |
||
60941 | 136 |
|
2672
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
paulson
parents:
2627
diff
changeset
|
137 |
(*** List-oriented tactics ***) |
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
paulson
parents:
2627
diff
changeset
|
138 |
|
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
paulson
parents:
2627
diff
changeset
|
139 |
local |
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
paulson
parents:
2627
diff
changeset
|
140 |
(*This version of EVERY avoids backtracking over repeated states*) |
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
paulson
parents:
2627
diff
changeset
|
141 |
|
13108 | 142 |
fun EVY (trail, []) st = |
60941 | 143 |
Seq.make (fn () => SOME (st, Seq.make (fn () => Seq.pull (evyBack trail)))) |
144 |
| EVY (trail, tac :: tacs) st = |
|
145 |
(case Seq.pull (tac st) of |
|
146 |
NONE => evyBack trail (*failed: backtrack*) |
|
147 |
| SOME (st', q) => EVY ((st', q, tacs) :: trail, tacs) st') |
|
4270 | 148 |
and evyBack [] = Seq.empty (*no alternatives*) |
60941 | 149 |
| evyBack ((st', q, tacs) :: trail) = |
150 |
(case Seq.pull q of |
|
151 |
NONE => evyBack trail |
|
152 |
| SOME (st, q') => |
|
153 |
if Thm.eq_thm (st', st) |
|
154 |
then evyBack ((st', q', tacs) :: trail) |
|
155 |
else EVY ((st, q', tacs) :: trail, tacs) st); |
|
2672
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
paulson
parents:
2627
diff
changeset
|
156 |
in |
60941 | 157 |
(* EVERY [tac1,...,tacn] equals tac1 THEN ... THEN tacn *) |
158 |
fun EVERY tacs = EVY ([], tacs); |
|
2672
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
paulson
parents:
2627
diff
changeset
|
159 |
end; |
2627 | 160 |
|
0 | 161 |
|
1502 | 162 |
(* EVERY' [tac1,...,tacn] i equals tac1 i THEN ... THEN tacn i *) |
2672
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
paulson
parents:
2627
diff
changeset
|
163 |
fun EVERY' tacs i = EVERY (map (fn f => f i) tacs); |
0 | 164 |
|
165 |
(*Apply every tactic to 1*) |
|
1502 | 166 |
fun EVERY1 tacs = EVERY' tacs 1; |
0 | 167 |
|
168 |
(* FIRST [tac1,...,tacn] equals tac1 ORELSE ... ORELSE tacn *) |
|
23178 | 169 |
fun FIRST tacs = fold_rev (curry op ORELSE) tacs no_tac; |
0 | 170 |
|
1502 | 171 |
(* FIRST' [tac1,...,tacn] i equals tac1 i ORELSE ... ORELSE tacn i *) |
23178 | 172 |
fun FIRST' tacs = fold_rev (curry op ORELSE') tacs (K no_tac); |
0 | 173 |
|
174 |
(*Apply first tactic to 1*) |
|
1502 | 175 |
fun FIRST1 tacs = FIRST' tacs 1; |
0 | 176 |
|
11916 | 177 |
(*Apply tactics on consecutive subgoals*) |
178 |
fun RANGE [] _ = all_tac |
|
179 |
| RANGE (tac :: tacs) i = RANGE tacs (i + 1) THEN tac i; |
|
180 |
||
0 | 181 |
|
182 |
(*** Tracing tactics ***) |
|
183 |
||
184 |
(*Print the current proof state and pass it on.*) |
|
56491 | 185 |
fun print_tac ctxt msg st = |
186 |
(tracing (msg ^ "\n" ^ Pretty.string_of (Pretty.chunks (Goal_Display.pretty_goals ctxt st))); |
|
32145
220c9e439d39
clarified pretty_goals, pretty_thm_aux: plain context;
wenzelm
parents:
32089
diff
changeset
|
187 |
Seq.single st); |
0 | 188 |
|
189 |
(*Pause until a line is typed -- if non-empty then fail. *) |
|
13108 | 190 |
fun pause_tac st = |
60941 | 191 |
(tracing "** Press RETURN to continue:"; |
192 |
if TextIO.inputLine TextIO.stdIn = SOME "\n" then Seq.single st |
|
193 |
else (tracing "Goodbye"; Seq.empty)); |
|
0 | 194 |
|
195 |
exception TRACE_EXIT of thm |
|
196 |
and TRACE_QUIT; |
|
197 |
||
631
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
lcp
parents:
230
diff
changeset
|
198 |
(*Tracing flags*) |
32738 | 199 |
val trace_REPEAT= Unsynchronized.ref false |
200 |
and suppress_tracing = Unsynchronized.ref false; |
|
631
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
lcp
parents:
230
diff
changeset
|
201 |
|
0 | 202 |
(*Handle all tracing commands for current state and tactic *) |
13108 | 203 |
fun exec_trace_command flag (tac, st) = |
60941 | 204 |
(case TextIO.inputLine TextIO.stdIn of |
205 |
SOME "\n" => tac st |
|
206 |
| SOME "f\n" => Seq.empty |
|
207 |
| SOME "o\n" => (flag := false; tac st) |
|
208 |
| SOME "s\n" => (suppress_tracing := true; tac st) |
|
209 |
| SOME "x\n" => (tracing "Exiting now"; raise (TRACE_EXIT st)) |
|
210 |
| SOME "quit\n" => raise TRACE_QUIT |
|
211 |
| _ => |
|
212 |
(tracing |
|
213 |
"Type RETURN to continue or...\n\ |
|
214 |
\ f - to fail here\n\ |
|
215 |
\ o - to switch tracing off\n\ |
|
216 |
\ s - to suppress tracing until next entry to a tactical\n\ |
|
217 |
\ x - to exit at this point\n\ |
|
218 |
\ quit - to abort this tracing run\n\ |
|
219 |
\** Well? "; exec_trace_command flag (tac, st))); |
|
0 | 220 |
|
221 |
||
222 |
(*Extract from a tactic, a thm->thm seq function that handles tracing*) |
|
1502 | 223 |
fun tracify flag tac st = |
32145
220c9e439d39
clarified pretty_goals, pretty_thm_aux: plain context;
wenzelm
parents:
32089
diff
changeset
|
224 |
if !flag andalso not (!suppress_tracing) then |
32168
116461b8fc01
eliminated print_goals_without_context -- proper pretty printing;
wenzelm
parents:
32145
diff
changeset
|
225 |
(tracing (Pretty.string_of (Pretty.chunks |
56493
1f660d858a75
prefer regular Goal_Display.pretty_goals, without censorship of options;
wenzelm
parents:
56491
diff
changeset
|
226 |
(Goal_Display.pretty_goals (Syntax.init_pretty_global (Thm.theory_of_thm st)) st @ |
32168
116461b8fc01
eliminated print_goals_without_context -- proper pretty printing;
wenzelm
parents:
32145
diff
changeset
|
227 |
[Pretty.str "** Press RETURN to continue:"]))); |
116461b8fc01
eliminated print_goals_without_context -- proper pretty printing;
wenzelm
parents:
32145
diff
changeset
|
228 |
exec_trace_command flag (tac, st)) |
1502 | 229 |
else tac st; |
0 | 230 |
|
231 |
(*Create a tactic whose outcome is given by seqf, handling TRACE_EXIT*) |
|
13108 | 232 |
fun traced_tac seqf st = |
60941 | 233 |
(suppress_tracing := false; |
234 |
Seq.make (fn () => seqf st handle TRACE_EXIT st' => SOME (st', Seq.empty))); |
|
0 | 235 |
|
236 |
||
13108 | 237 |
(*Deterministic REPEAT: only retains the first outcome; |
703
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
lcp
parents:
671
diff
changeset
|
238 |
uses less space than REPEAT; tail recursive. |
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
lcp
parents:
671
diff
changeset
|
239 |
If non-negative, n bounds the number of repetitions.*) |
13108 | 240 |
fun REPEAT_DETERM_N n tac = |
60941 | 241 |
let |
242 |
val tac = tracify trace_REPEAT tac; |
|
243 |
fun drep 0 st = SOME (st, Seq.empty) |
|
244 |
| drep n st = |
|
245 |
(case Seq.pull (tac st) of |
|
246 |
NONE => SOME(st, Seq.empty) |
|
247 |
| SOME (st', _) => drep (n - 1) st'); |
|
248 |
in traced_tac (drep n) end; |
|
703
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
lcp
parents:
671
diff
changeset
|
249 |
|
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
lcp
parents:
671
diff
changeset
|
250 |
(*Allows any number of repetitions*) |
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
lcp
parents:
671
diff
changeset
|
251 |
val REPEAT_DETERM = REPEAT_DETERM_N ~1; |
0 | 252 |
|
253 |
(*General REPEAT: maintains a stack of alternatives; tail recursive*) |
|
13108 | 254 |
fun REPEAT tac = |
60941 | 255 |
let |
256 |
val tac = tracify trace_REPEAT tac; |
|
257 |
fun rep qs st = |
|
258 |
(case Seq.pull (tac st) of |
|
259 |
NONE => SOME (st, Seq.make (fn () => repq qs)) |
|
260 |
| SOME (st', q) => rep (q :: qs) st') |
|
261 |
and repq [] = NONE |
|
262 |
| repq (q :: qs) = |
|
263 |
(case Seq.pull q of |
|
264 |
NONE => repq qs |
|
265 |
| SOME (st, q) => rep (q :: qs) st); |
|
266 |
in traced_tac (rep []) end; |
|
0 | 267 |
|
268 |
(*Repeat 1 or more times*) |
|
703
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
lcp
parents:
671
diff
changeset
|
269 |
fun REPEAT_DETERM1 tac = DETERM tac THEN REPEAT_DETERM tac; |
0 | 270 |
fun REPEAT1 tac = tac THEN REPEAT tac; |
271 |
||
272 |
||
273 |
(** Filtering tacticals **) |
|
274 |
||
4270 | 275 |
fun FILTER pred tac st = Seq.filter pred (tac st); |
0 | 276 |
|
13650
31bd2a8cdbe2
fixing the cut_tac method to work when there are no instantiations and the
paulson
parents:
13108
diff
changeset
|
277 |
(*Accept only next states that change the theorem somehow*) |
13108 | 278 |
fun CHANGED tac st = |
279 |
let fun diff st' = not (Thm.eq_thm (st, st')); |
|
280 |
in Seq.filter diff (tac st) end; |
|
0 | 281 |
|
13650
31bd2a8cdbe2
fixing the cut_tac method to work when there are no instantiations and the
paulson
parents:
13108
diff
changeset
|
282 |
(*Accept only next states that change the theorem's prop field |
31bd2a8cdbe2
fixing the cut_tac method to work when there are no instantiations and the
paulson
parents:
13108
diff
changeset
|
283 |
(changes to signature, hyps, etc. don't count)*) |
13108 | 284 |
fun CHANGED_PROP tac st = |
22360
26ead7ed4f4b
moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
wenzelm
parents:
20664
diff
changeset
|
285 |
let fun diff st' = not (Thm.eq_thm_prop (st, st')); |
13108 | 286 |
in Seq.filter diff (tac st) end; |
10821 | 287 |
|
0 | 288 |
|
289 |
(*** Tacticals based on subgoal numbering ***) |
|
290 |
||
13108 | 291 |
(*For n subgoals, performs tac(n) THEN ... THEN tac(1) |
1502 | 292 |
Essential to work backwards since tac(i) may add/delete subgoals at i. *) |
13108 | 293 |
fun ALLGOALS tac st = |
60941 | 294 |
let |
295 |
fun doall 0 = all_tac |
|
296 |
| doall n = tac n THEN doall (n - 1); |
|
297 |
in doall (Thm.nprems_of st) st end; |
|
0 | 298 |
|
1502 | 299 |
(*For n subgoals, performs tac(n) ORELSE ... ORELSE tac(1) *) |
13108 | 300 |
fun SOMEGOAL tac st = |
60941 | 301 |
let |
302 |
fun find 0 = no_tac |
|
303 |
| find n = tac n ORELSE find (n - 1); |
|
304 |
in find (Thm.nprems_of st) st end; |
|
0 | 305 |
|
1502 | 306 |
(*For n subgoals, performs tac(1) ORELSE ... ORELSE tac(n). |
0 | 307 |
More appropriate than SOMEGOAL in some cases.*) |
13108 | 308 |
fun FIRSTGOAL tac st = |
60941 | 309 |
let fun find (i, n) = if i > n then no_tac else tac i ORELSE find (i + 1, n) |
310 |
in find (1, Thm.nprems_of st) st end; |
|
0 | 311 |
|
46466
61c7214b4885
tuned signature, according to actual usage of these operations;
wenzelm
parents:
46463
diff
changeset
|
312 |
(*First subgoal only.*) |
61c7214b4885
tuned signature, according to actual usage of these operations;
wenzelm
parents:
46463
diff
changeset
|
313 |
fun HEADGOAL tac = tac 1; |
61c7214b4885
tuned signature, according to actual usage of these operations;
wenzelm
parents:
46463
diff
changeset
|
314 |
|
1502 | 315 |
(*Repeatedly solve some using tac. *) |
316 |
fun REPEAT_SOME tac = REPEAT1 (SOMEGOAL (REPEAT1 o tac)); |
|
317 |
fun REPEAT_DETERM_SOME tac = REPEAT_DETERM1 (SOMEGOAL (REPEAT_DETERM1 o tac)); |
|
0 | 318 |
|
1502 | 319 |
(*Repeatedly solve the first possible subgoal using tac. *) |
320 |
fun REPEAT_FIRST tac = REPEAT1 (FIRSTGOAL (REPEAT1 o tac)); |
|
321 |
fun REPEAT_DETERM_FIRST tac = REPEAT_DETERM1 (FIRSTGOAL (REPEAT_DETERM1 o tac)); |
|
0 | 322 |
|
1502 | 323 |
(*For n subgoals, tries to apply tac to n,...1 *) |
324 |
fun TRYALL tac = ALLGOALS (TRY o tac); |
|
0 | 325 |
|
326 |
||
327 |
(*Make a tactic for subgoal i, if there is one. *) |
|
23224 | 328 |
fun CSUBGOAL goalfun i st = |
329 |
(case SOME (Thm.cprem_of st i) handle THM _ => NONE of |
|
16510
606d919ad3c3
tuned SUBGOAL: Logic.nth_prem instead of List.nth o prems_of;
wenzelm
parents:
16179
diff
changeset
|
330 |
SOME goal => goalfun (goal, i) st |
606d919ad3c3
tuned SUBGOAL: Logic.nth_prem instead of List.nth o prems_of;
wenzelm
parents:
16179
diff
changeset
|
331 |
| NONE => Seq.empty); |
0 | 332 |
|
23224 | 333 |
fun SUBGOAL goalfun = |
334 |
CSUBGOAL (fn (goal, i) => goalfun (Thm.term_of goal, i)); |
|
335 |
||
60941 | 336 |
fun ASSERT_SUBGOAL (tac: int -> tactic) i st = |
337 |
(Logic.get_goal (Thm.prop_of st) i; tac i st); |
|
49865 | 338 |
|
5141 | 339 |
(*Returns all states that have changed in subgoal i, counted from the LAST |
340 |
subgoal. For stac, for example.*) |
|
13108 | 341 |
fun CHANGED_GOAL tac i st = |
56231
b98813774a63
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
wenzelm
parents:
52131
diff
changeset
|
342 |
SUBGOAL (fn (t, _) => |
b98813774a63
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
wenzelm
parents:
52131
diff
changeset
|
343 |
let |
b98813774a63
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
wenzelm
parents:
52131
diff
changeset
|
344 |
val np = Thm.nprems_of st; |
b98813774a63
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
wenzelm
parents:
52131
diff
changeset
|
345 |
val d = np - i; (*distance from END*) |
b98813774a63
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
wenzelm
parents:
52131
diff
changeset
|
346 |
fun diff st' = |
b98813774a63
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
wenzelm
parents:
52131
diff
changeset
|
347 |
Thm.nprems_of st' - d <= 0 orelse (*the subgoal no longer exists*) |
b98813774a63
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
wenzelm
parents:
52131
diff
changeset
|
348 |
not (Envir.aeconv (t, Thm.term_of (Thm.cprem_of st' (Thm.nprems_of st' - d)))); |
b98813774a63
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
wenzelm
parents:
52131
diff
changeset
|
349 |
in Seq.filter diff o tac i end) i st; |
5141 | 350 |
|
34885
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
351 |
(*Returns all states where some subgoals have been solved. For |
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
352 |
subgoal-based tactics this means subgoal i has been solved |
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
353 |
altogether -- no new subgoals have emerged.*) |
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
354 |
fun SOLVED' tac i st = |
59582 | 355 |
tac i st |> Seq.filter (fn st' => Thm.nprems_of st' < Thm.nprems_of st); |
34885
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
356 |
|
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
357 |
(*Apply second tactic to all subgoals emerging from the first -- |
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
358 |
following usual convention for subgoal-based tactics.*) |
4602 | 359 |
fun (tac1 THEN_ALL_NEW tac2) i st = |
59660
49e498cedd02
support structural composition (THEN_ALL_NEW) for proof methods;
wenzelm
parents:
59582
diff
changeset
|
360 |
st |> (tac1 i THEN (fn st' => |
61841
4d3527b94f2a
more general types Proof.method / context_tactic;
wenzelm
parents:
60941
diff
changeset
|
361 |
st' |> Seq.INTERVAL tac2 i (i + Thm.nprems_of st' - Thm.nprems_of st))); |
4602 | 362 |
|
34885
6587c24ef6d8
added SOLVED' -- a more direct version of THEN_ALL_NEW (K no_tac) -- strictly speaking it does not even depend on subgoal addressing, but it would be too confusing without it;
wenzelm
parents:
32738
diff
changeset
|
363 |
(*Repeatedly dig into any emerging subgoals.*) |
8341 | 364 |
fun REPEAT_ALL_NEW tac = |
365 |
tac THEN_ALL_NEW (TRY o (fn i => REPEAT_ALL_NEW tac i)); |
|
366 |
||
15006
107e4dfd3b96
Merging the meta-simplifier with the Provers-simplifier. Next step:
skalberg
parents:
13664
diff
changeset
|
367 |
(*Makes a tactic whose effect on a state is given by thmfun: thm->thm seq.*) |
107e4dfd3b96
Merging the meta-simplifier with the Provers-simplifier. Next step:
skalberg
parents:
13664
diff
changeset
|
368 |
fun PRIMSEQ thmfun st = thmfun st handle THM _ => Seq.empty; |
107e4dfd3b96
Merging the meta-simplifier with the Provers-simplifier. Next step:
skalberg
parents:
13664
diff
changeset
|
369 |
|
107e4dfd3b96
Merging the meta-simplifier with the Provers-simplifier. Next step:
skalberg
parents:
13664
diff
changeset
|
370 |
(*Makes a tactic whose effect on a state is given by thmfun: thm->thm.*) |
107e4dfd3b96
Merging the meta-simplifier with the Provers-simplifier. Next step:
skalberg
parents:
13664
diff
changeset
|
371 |
fun PRIMITIVE thmfun = PRIMSEQ (Seq.single o thmfun); |
107e4dfd3b96
Merging the meta-simplifier with the Provers-simplifier. Next step:
skalberg
parents:
13664
diff
changeset
|
372 |
|
23538 | 373 |
(*Inverse (more or less) of PRIMITIVE*) |
15570 | 374 |
fun SINGLE tacf = Option.map fst o Seq.pull o tacf |
19455 | 375 |
|
23538 | 376 |
(*Conversions as tactics*) |
23584 | 377 |
fun CONVERSION cv i st = Seq.single (Conv.gconv_rule cv i st) |
23561 | 378 |
handle THM _ => Seq.empty |
379 |
| CTERM _ => Seq.empty |
|
380 |
| TERM _ => Seq.empty |
|
381 |
| TYPE _ => Seq.empty; |
|
23538 | 382 |
|
0 | 383 |
end; |
1502 | 384 |
|
385 |
open Tactical; |