author | wenzelm |
Fri, 05 Jul 2013 17:09:28 +0200 | |
changeset 52533 | a95440dcd59c |
parent 52532 | c81d76f7f63d |
child 52534 | 341ae9cd4743 |
permissions | -rw-r--r-- |
47336 | 1 |
(* Title: Pure/PIDE/command.ML |
2 |
Author: Makarius |
|
3 |
||
4 |
Prover command execution. |
|
5 |
*) |
|
6 |
||
7 |
signature COMMAND = |
|
8 |
sig |
|
52509 | 9 |
type span = Token.T list |
10 |
val range: span -> Position.range |
|
11 |
val proper_range: span -> Position.range |
|
47341
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
12 |
type 'a memo |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
13 |
val memo: (unit -> 'a) -> 'a memo |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
14 |
val memo_value: 'a -> 'a memo |
47342
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
15 |
val memo_eval: 'a memo -> 'a |
52526 | 16 |
val memo_fork: Future.params -> 'a memo -> unit |
47342
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
17 |
val memo_result: 'a memo -> 'a |
52526 | 18 |
val memo_stable: 'a memo -> bool |
52510 | 19 |
val read: span -> Toplevel.transition |
52526 | 20 |
type eval_state = |
21 |
{failed: bool, malformed: bool, command: Toplevel.transition, state: Toplevel.state} |
|
52533 | 22 |
type eval = {exec_id: Document_ID.exec, eval: eval_state memo} |
52526 | 23 |
val no_eval: eval |
52533 | 24 |
val eval_result: eval -> eval_state |
52526 | 25 |
val eval: span -> Toplevel.transition -> eval_state -> eval_state |
26 |
type print_fn = Toplevel.transition -> Toplevel.state -> unit |
|
52530
99dd8b4ef3fe
explicit module Document_ID as source of globally unique identifiers across ML/Scala;
wenzelm
parents:
52527
diff
changeset
|
27 |
type print = {name: string, pri: int, exec_id: Document_ID.exec, print: unit memo} |
99dd8b4ef3fe
explicit module Document_ID as source of globally unique identifiers across ML/Scala;
wenzelm
parents:
52527
diff
changeset
|
28 |
val print: string -> eval -> print list |
52526 | 29 |
val print_function: {name: string, pri: int} -> (string -> print_fn option) -> unit |
52533 | 30 |
type exec = eval * print list |
52532 | 31 |
val no_exec: exec |
32 |
val exec_ids: exec -> Document_ID.exec list |
|
33 |
val exec_result: exec -> eval_state |
|
34 |
val exec_run: exec -> unit |
|
52533 | 35 |
val stable_eval: eval -> bool |
52532 | 36 |
val stable_print: print -> bool |
47336 | 37 |
end; |
38 |
||
39 |
structure Command: COMMAND = |
|
40 |
struct |
|
41 |
||
52509 | 42 |
(* source *) |
43 |
||
44 |
type span = Token.T list; |
|
48771
2ea997196d04
clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents:
47395
diff
changeset
|
45 |
|
49866 | 46 |
val range = Token.position_range_of; |
51266
3007d0bc9cb1
unified Command.is_proper in ML with Scala (see also 123be08eed88);
wenzelm
parents:
50914
diff
changeset
|
47 |
val proper_range = Token.position_range_of o #1 o take_suffix Token.is_improper; |
48771
2ea997196d04
clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents:
47395
diff
changeset
|
48 |
|
2ea997196d04
clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents:
47395
diff
changeset
|
49 |
|
47341
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
50 |
(* memo results *) |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
51 |
|
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
52 |
datatype 'a expr = |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
53 |
Expr of unit -> 'a | |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
54 |
Result of 'a Exn.result; |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
55 |
|
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
56 |
abstype 'a memo = Memo of 'a expr Synchronized.var |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
57 |
with |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
58 |
|
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
59 |
fun memo e = Memo (Synchronized.var "Command.memo" (Expr e)); |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
60 |
fun memo_value a = Memo (Synchronized.var "Command.memo" (Result (Exn.Res a))); |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
61 |
|
47342
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
62 |
fun memo_eval (Memo v) = |
47341
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
63 |
(case Synchronized.value v of |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
64 |
Result res => res |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
65 |
| _ => |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
66 |
Synchronized.guarded_access v |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
67 |
(fn Result res => SOME (res, Result res) |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
68 |
| Expr e => |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
69 |
let val res = Exn.capture e (); (*memoing of physical interrupts!*) |
47342
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
70 |
in SOME (res, Result res) end)) |
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
71 |
|> Exn.release; |
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
72 |
|
52526 | 73 |
fun memo_fork params (Memo v) = |
74 |
(case Synchronized.value v of |
|
75 |
Result _ => () |
|
76 |
| _ => ignore ((singleton o Future.forks) params (fn () => memo_eval (Memo v)))); |
|
77 |
||
47342
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
78 |
fun memo_result (Memo v) = |
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
79 |
(case Synchronized.value v of |
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
80 |
Result res => Exn.release res |
7828c7b3c143
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents:
47341
diff
changeset
|
81 |
| _ => raise Fail "Unfinished memo result"); |
47341
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
82 |
|
52526 | 83 |
fun memo_stable (Memo v) = |
84 |
(case Synchronized.value v of |
|
85 |
Expr _ => true |
|
86 |
| Result res => not (Exn.is_interrupt_exn res)); |
|
87 |
||
47341
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
88 |
end; |
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
89 |
|
00f6279bb67a
Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents:
47336
diff
changeset
|
90 |
|
52532 | 91 |
(** main phases: read -- eval -- print **) |
92 |
||
52510 | 93 |
(* read *) |
52509 | 94 |
|
52510 | 95 |
fun read span = |
96 |
let |
|
97 |
val outer_syntax = #2 (Outer_Syntax.get_syntax ()); |
|
98 |
val command_reports = Outer_Syntax.command_reports outer_syntax; |
|
52509 | 99 |
|
52510 | 100 |
val proper_range = Position.set_range (proper_range span); |
101 |
val pos = |
|
102 |
(case find_first Token.is_command span of |
|
103 |
SOME tok => Token.position_of tok |
|
104 |
| NONE => proper_range); |
|
52509 | 105 |
|
52510 | 106 |
val (is_malformed, token_reports) = Thy_Syntax.reports_of_tokens span; |
107 |
val _ = Position.reports_text (token_reports @ maps command_reports span); |
|
108 |
in |
|
109 |
if is_malformed then Toplevel.malformed pos "Malformed command syntax" |
|
110 |
else |
|
111 |
(case Outer_Syntax.read_spans outer_syntax span of |
|
112 |
[tr] => |
|
113 |
if Keyword.is_control (Toplevel.name_of tr) then |
|
114 |
Toplevel.malformed pos "Illegal control command" |
|
115 |
else tr |
|
116 |
| [] => Toplevel.ignored (Position.set_range (range span)) |
|
117 |
| _ => Toplevel.malformed proper_range "Exactly one command expected") |
|
118 |
handle ERROR msg => Toplevel.malformed proper_range msg |
|
119 |
end; |
|
52509 | 120 |
|
121 |
||
122 |
(* eval *) |
|
47336 | 123 |
|
52526 | 124 |
type eval_state = |
125 |
{failed: bool, malformed: bool, command: Toplevel.transition, state: Toplevel.state}; |
|
126 |
val no_eval_state: eval_state = |
|
127 |
{failed = false, malformed = false, command = Toplevel.empty, state = Toplevel.toplevel}; |
|
128 |
||
52533 | 129 |
type eval = {exec_id: Document_ID.exec, eval: eval_state memo}; |
130 |
||
131 |
val no_eval: eval = {exec_id = Document_ID.none, eval = memo_value no_eval_state}; |
|
132 |
fun eval_result ({eval, ...}: eval) = memo_result eval; |
|
52526 | 133 |
|
47336 | 134 |
local |
135 |
||
136 |
fun run int tr st = |
|
51284
59a03019f3bf
fork diagnostic commands (theory loader and PIDE interaction);
wenzelm
parents:
51266
diff
changeset
|
137 |
if Goal.future_enabled () andalso Keyword.is_diag (Toplevel.name_of tr) then |
51605
eca8acb42e4a
more explicit Goal.fork_params -- avoid implicit arguments via thread data;
wenzelm
parents:
51603
diff
changeset
|
138 |
(Goal.fork_params {name = "Toplevel.diag", pos = Toplevel.pos_of tr, pri = ~1} |
eca8acb42e4a
more explicit Goal.fork_params -- avoid implicit arguments via thread data;
wenzelm
parents:
51603
diff
changeset
|
139 |
(fn () => Toplevel.command_exception int tr st); ([], SOME st)) |
51284
59a03019f3bf
fork diagnostic commands (theory loader and PIDE interaction);
wenzelm
parents:
51266
diff
changeset
|
140 |
else Toplevel.command_errors int tr st; |
47336 | 141 |
|
52510 | 142 |
fun check_cmts span tr st' = |
143 |
Toplevel.setmp_thread_position tr |
|
144 |
(fn () => |
|
145 |
Outer_Syntax.side_comments span |> maps (fn cmt => |
|
146 |
(Thy_Output.check_text (Token.source_position_of cmt) st'; []) |
|
147 |
handle exn => ML_Compiler.exn_messages_ids exn)) (); |
|
148 |
||
47336 | 149 |
fun proof_status tr st = |
150 |
(case try Toplevel.proof_of st of |
|
151 |
SOME prf => Toplevel.status tr (Proof.status_markup prf) |
|
152 |
| NONE => ()); |
|
153 |
||
154 |
in |
|
155 |
||
52526 | 156 |
fun eval span tr ({malformed, state = st, ...}: eval_state) = |
52509 | 157 |
if malformed then |
52526 | 158 |
{failed = true, malformed = malformed, command = tr, state = Toplevel.toplevel} |
48772 | 159 |
else |
160 |
let |
|
161 |
val malformed' = Toplevel.is_malformed tr; |
|
162 |
val is_init = Toplevel.is_init tr; |
|
163 |
val is_proof = Keyword.is_proof (Toplevel.name_of tr); |
|
47336 | 164 |
|
48772 | 165 |
val _ = Multithreading.interrupted (); |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49866
diff
changeset
|
166 |
val _ = Toplevel.status tr Markup.running; |
48918
6e5fd4585512
check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents:
48772
diff
changeset
|
167 |
val (errs1, result) = run (is_init orelse is_proof) (Toplevel.set_print false tr) st; |
52509 | 168 |
val errs2 = (case result of NONE => [] | SOME st' => check_cmts span tr st'); |
48918
6e5fd4585512
check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents:
48772
diff
changeset
|
169 |
val errs = errs1 @ errs2; |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49866
diff
changeset
|
170 |
val _ = Toplevel.status tr Markup.finished; |
50914
fe4714886d92
identify future results more carefully, to avoid odd duplication of error messages, notably from forked goals;
wenzelm
parents:
50911
diff
changeset
|
171 |
val _ = List.app (Future.error_msg (Toplevel.pos_of tr)) errs; |
48772 | 172 |
in |
173 |
(case result of |
|
174 |
NONE => |
|
175 |
let |
|
176 |
val _ = if null errs then Exn.interrupt () else (); |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49866
diff
changeset
|
177 |
val _ = Toplevel.status tr Markup.failed; |
52526 | 178 |
in {failed = true, malformed = malformed', command = tr, state = st} end |
48772 | 179 |
| SOME st' => |
180 |
let |
|
181 |
val _ = proof_status tr st'; |
|
52526 | 182 |
in {failed = false, malformed = malformed', command = tr, state = st'} end) |
48772 | 183 |
end; |
47336 | 184 |
|
185 |
end; |
|
186 |
||
52509 | 187 |
|
188 |
(* print *) |
|
189 |
||
52530
99dd8b4ef3fe
explicit module Document_ID as source of globally unique identifiers across ML/Scala;
wenzelm
parents:
52527
diff
changeset
|
190 |
type print = {name: string, pri: int, exec_id: Document_ID.exec, print: unit memo}; |
52526 | 191 |
type print_fn = Toplevel.transition -> Toplevel.state -> unit; |
52515 | 192 |
|
52511 | 193 |
local |
194 |
||
52526 | 195 |
type print_function = string * (int * (string -> print_fn option)); |
196 |
val print_functions = Synchronized.var "Command.print_functions" ([]: print_function list); |
|
52511 | 197 |
|
52516
b5b3c888df9f
more exception handling -- make print functions total;
wenzelm
parents:
52515
diff
changeset
|
198 |
fun output_error tr exn = |
b5b3c888df9f
more exception handling -- make print functions total;
wenzelm
parents:
52515
diff
changeset
|
199 |
List.app (Future.error_msg (Toplevel.pos_of tr)) (ML_Compiler.exn_messages_ids exn); |
b5b3c888df9f
more exception handling -- make print functions total;
wenzelm
parents:
52515
diff
changeset
|
200 |
|
b5b3c888df9f
more exception handling -- make print functions total;
wenzelm
parents:
52515
diff
changeset
|
201 |
fun print_error tr f x = |
b5b3c888df9f
more exception handling -- make print functions total;
wenzelm
parents:
52515
diff
changeset
|
202 |
(Toplevel.setmp_thread_position tr o Runtime.controlled_execution) f x |
b5b3c888df9f
more exception handling -- make print functions total;
wenzelm
parents:
52515
diff
changeset
|
203 |
handle exn => output_error tr exn; |
b5b3c888df9f
more exception handling -- make print functions total;
wenzelm
parents:
52515
diff
changeset
|
204 |
|
52511 | 205 |
in |
52509 | 206 |
|
52530
99dd8b4ef3fe
explicit module Document_ID as source of globally unique identifiers across ML/Scala;
wenzelm
parents:
52527
diff
changeset
|
207 |
fun print command_name eval = |
52526 | 208 |
rev (Synchronized.value print_functions) |> map_filter (fn (name, (pri, get_print_fn)) => |
209 |
(case Exn.capture (Runtime.controlled_execution get_print_fn) command_name of |
|
52516
b5b3c888df9f
more exception handling -- make print functions total;
wenzelm
parents:
52515
diff
changeset
|
210 |
Exn.Res NONE => NONE |
52526 | 211 |
| Exn.Res (SOME print_fn) => |
52527
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
212 |
let |
52530
99dd8b4ef3fe
explicit module Document_ID as source of globally unique identifiers across ML/Scala;
wenzelm
parents:
52527
diff
changeset
|
213 |
val exec_id = Document_ID.make (); |
52527
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
214 |
fun body () = |
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
215 |
let |
52533 | 216 |
val {failed, command, state = st', ...} = eval_result eval; |
52527
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
217 |
val tr = Toplevel.put_id exec_id command; |
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
218 |
in if failed then () else print_error tr (fn () => print_fn tr st') () end; |
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
219 |
in SOME {name = name, pri = pri, exec_id = exec_id, print = memo body} end |
52526 | 220 |
| Exn.Exn exn => |
52527
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
221 |
let |
52530
99dd8b4ef3fe
explicit module Document_ID as source of globally unique identifiers across ML/Scala;
wenzelm
parents:
52527
diff
changeset
|
222 |
val exec_id = Document_ID.make (); |
52527
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
223 |
fun body () = |
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
224 |
let |
52533 | 225 |
val {command, ...} = eval_result eval; |
52527
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
226 |
val tr = Toplevel.put_id exec_id command; |
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
227 |
in output_error tr exn end; |
dbac84eab3bc
separate exec_id assignment for Command.print states, without affecting result of eval;
wenzelm
parents:
52526
diff
changeset
|
228 |
in SOME {name = name, pri = pri, exec_id = exec_id, print = memo body} end)); |
52511 | 229 |
|
52526 | 230 |
fun print_function {name, pri} f = |
52511 | 231 |
Synchronized.change print_functions (fn funs => |
232 |
(if not (AList.defined (op =) funs name) then () |
|
233 |
else warning ("Redefining command print function: " ^ quote name); |
|
52515 | 234 |
AList.update (op =) (name, (pri, f)) funs)); |
52511 | 235 |
|
236 |
end; |
|
237 |
||
52526 | 238 |
val _ = |
239 |
print_function {name = "print_state", pri = 0} (fn command_name => SOME (fn tr => fn st' => |
|
240 |
let |
|
241 |
val is_init = Keyword.is_theory_begin command_name; |
|
242 |
val is_proof = Keyword.is_proof command_name; |
|
243 |
val do_print = |
|
244 |
not is_init andalso |
|
245 |
(Toplevel.print_of tr orelse (is_proof andalso Toplevel.is_proof st')); |
|
246 |
in if do_print then Toplevel.print_state false st' else () end)); |
|
52509 | 247 |
|
52532 | 248 |
|
249 |
||
52533 | 250 |
(** managed evaluation **) |
52532 | 251 |
|
252 |
(* execution *) |
|
253 |
||
52533 | 254 |
type exec = eval * print list; |
255 |
val no_exec: exec = (no_eval, []); |
|
52532 | 256 |
|
52533 | 257 |
fun exec_ids (({exec_id, ...}, prints): exec) = exec_id :: map #exec_id prints; |
52532 | 258 |
|
52533 | 259 |
fun exec_result (({eval, ...}, _): exec) = memo_result eval; |
52532 | 260 |
|
52533 | 261 |
fun exec_run (({eval, ...}, prints): exec) = |
52532 | 262 |
(memo_eval eval; |
263 |
prints |> List.app (fn {name, pri, print, ...} => |
|
264 |
memo_fork {name = name, group = NONE, deps = [], pri = pri, interrupts = true} print)); |
|
265 |
||
266 |
||
52533 | 267 |
(* stable situations after cancellation *) |
52532 | 268 |
|
269 |
fun stable_goals exec_id = |
|
270 |
not (Par_Exn.is_interrupted (Future.join_results (Goal.peek_futures exec_id))); |
|
271 |
||
52533 | 272 |
fun stable_eval ({exec_id, eval}: eval) = |
52532 | 273 |
stable_goals exec_id andalso memo_stable eval; |
274 |
||
275 |
fun stable_print ({exec_id, print, ...}: print) = |
|
276 |
stable_goals exec_id andalso memo_stable print; |
|
277 |
||
47336 | 278 |
end; |
279 |