src/Pure/Concurrent/par_exn.ML
author wenzelm
Wed, 17 Aug 2011 23:37:23 +0200
changeset 44249 64620f1d6f87
parent 44248 6a3541412b23
child 44264 c21ecbb028b6
permissions -rw-r--r--
identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
44247
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     1
(*  Title:      Pure/Concurrent/par_exn.ML
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     2
    Author:     Makarius
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     3
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     4
Parallel exceptions as flattened results from acyclic graph of
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     5
evaluations.  Interrupt counts as neutral element.
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     6
*)
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     7
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     8
signature PAR_EXN =
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
     9
sig
44249
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    10
  val serial: exn -> serial * exn
44247
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    11
  val make: exn list -> exn
44249
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    12
  val dest: exn -> exn list option
44247
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    13
  val release_all: 'a Exn.result list -> 'a list
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    14
  val release_first: 'a Exn.result list -> 'a list
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    15
end;
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    16
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    17
structure Par_Exn =
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    18
struct
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    19
44249
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    20
(* identification via serial numbers *)
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    21
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    22
fun serial exn =
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    23
  (case get_exn_serial exn of
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    24
    SOME i => (i, exn)
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    25
  | NONE => let val i = Library.serial () in (i, set_exn_serial i exn) end);
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    26
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    27
val exn_ord = rev_order o int_ord o pairself (the o get_exn_serial);
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    28
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    29
44247
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    30
(* parallel exceptions *)
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    31
44249
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    32
exception Par_Exn of exn Ord_List.T;
44247
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    33
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    34
fun par_exns (Par_Exn exns) = SOME exns
44249
64620f1d6f87 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm
parents: 44248
diff changeset
    35
  | par_exns exn = if Exn.is_interrupt exn then NONE else SOME [#2 (serial exn)];
44247
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    36
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    37
fun make exns =
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    38
  (case map_filter par_exns exns of
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    39
    [] => Exn.Interrupt
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    40
  | e :: es => Par_Exn (Library.foldl (Ord_List.merge exn_ord) (e, es)));
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    41
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    42
fun dest (Par_Exn exns) = SOME (rev exns)
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    43
  | dest _ = NONE;
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    44
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    45
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    46
(* parallel results *)
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    47
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    48
fun all_res results = forall (fn Exn.Res _ => true | _ => false) results;
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    49
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    50
fun release_all results =
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    51
  if all_res results then map Exn.release results
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    52
  else raise make (map_filter Exn.get_exn results);
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    53
44248
6a3541412b23 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm
parents: 44247
diff changeset
    54
fun release_first results =
6a3541412b23 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm
parents: 44247
diff changeset
    55
  if all_res results then map Exn.release results
6a3541412b23 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm
parents: 44247
diff changeset
    56
  else
6a3541412b23 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm
parents: 44247
diff changeset
    57
    (case get_first
6a3541412b23 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm
parents: 44247
diff changeset
    58
        (fn res => if Exn.is_interrupt_exn res then NONE else Exn.get_exn res) results of
6a3541412b23 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm
parents: 44247
diff changeset
    59
      NONE => Exn.interrupt ()
6a3541412b23 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm
parents: 44247
diff changeset
    60
    | SOME exn => reraise exn);
44247
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    61
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    62
end;
270366301bd7 more systematic handling of parallel exceptions;
wenzelm
parents:
diff changeset
    63