added trace flag, official tracing operation;
added named CRITICAL';
schedule: tuned signature, actually observe dependencies on running tasks;
(* Title: Pure/ML-Systems/multithreading_polyml.ML
ID: $Id$
Author: Makarius
Multithreading in Poly/ML (version 5.1).
*)
open Thread;
structure Multithreading: MULTITHREADING =
struct
val trace = ref false;
fun tracing msg =
if ! trace
then (TextIO.output (TextIO.stdErr, (">>> " ^ msg () ^ "\n")); TextIO.flushOut TextIO.stdErr)
else ();
val available = true;
val max_threads = ref 1;
(* critical section -- may be nested within the same thread *)
local
val critical_lock = Mutex.mutex ();
val critical_thread = ref (NONE: Thread.thread option);
in
fun self_critical () =
(case ! critical_thread of
NONE => false
| SOME id => Thread.equal (id, Thread.self ()));
fun CRITICAL' name e =
if self_critical () then e ()
else
let
val _ =
if Mutex.trylock critical_lock then ()
else
(tracing (fn () => "CRITICAL " ^ name ^ ": waiting for lock");
Mutex.lock critical_lock;
tracing (fn () => "CRITICAL " ^ name ^ ": obtained lock"));
val _ = critical_thread := SOME (Thread.self ());
val result = Exn.capture e ();
val _ = critical_thread := NONE;
val _ = Mutex.unlock critical_lock;
in Exn.release result end;
fun CRITICAL e = CRITICAL' "" e;
end;
(* scheduling -- non-interruptible threads working on a queue of tasks *)
fun schedule n next_task tasks =
let
(*protected execution*)
val lock = Mutex.mutex ();
fun PROTECTED k e =
let
val _ =
if Mutex.trylock lock then ()
else
(tracing (fn () => "PROTECTED " ^ Int.toString k ^ ": waiting for lock");
Mutex.lock lock;
tracing (fn () => "PROTECTED " ^ Int.toString k ^ ": obtained lock"));
val res = Exn.capture e ();
val _ = Mutex.unlock lock;
in Exn.release res end;
(*the queue of tasks*)
val queue = ref tasks;
fun dequeue k = PROTECTED k (fn () =>
let
val (next, tasks') = next_task (! queue);
val _ = queue := tasks';
in next end);
(*worker threads*)
val running = ref 0;
val status = ref ([]: exn list);
val finished = ConditionVar.conditionVar ();
fun wait () = ConditionVar.waitUntil (finished, lock, Time.fromMilliseconds 500);
fun continue cont k =
(PROTECTED k (fn () => queue := cont (! queue)); ConditionVar.signal finished; work k ())
and work k () =
(case dequeue k of
(Task.Task f, cont) =>
(tracing (fn () => "TASK " ^ Int.toString k);
case Exn.capture f () of
Exn.Result () => continue cont k
| Exn.Exn exn =>
(PROTECTED k (fn () => status := exn :: ! status); continue cont k))
| (Task.Running, _) =>
(tracing (fn () => "WAITING " ^ Int.toString k);
PROTECTED k wait; work k ())
| (Task.Finished, _) =>
(tracing (fn () => "TERMINATING " ^ Int.toString k);
PROTECTED k (fn () => running := ! running - 1);
ConditionVar.signal finished));
(*main control: fork and wait*)
fun fork 0 = ()
| fork k =
(running := ! running + 1;
Thread.fork (work k, [Thread.InterruptState Thread.InterruptDefer]);
fork (k - 1));
val _ = PROTECTED 0 (fn () =>
(fork (Int.max (n, 1)); while ! running <> 0 do (tracing (fn () => "MAIN WAIT"); wait ())));
in ! status end;
end;
val CRITICAL' = Multithreading.CRITICAL';
val CRITICAL = Multithreading.CRITICAL;