aboutsummaryrefslogtreecommitdiffhomepage
path: root/lib/dag.ml
blob: 5a695ce1bc5b1dabe46480da0d87457ce25586ff (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
90
91
92
93
94
95
96
97
98
99
100
101
(************************************************************************)
(*  v      *   The Coq Proof Assistant  /  The Coq Development Team     *)
(* <O___,, *   INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2013     *)
(*   \VV/  **************************************************************)
(*    //   *      This file is distributed under the terms of the       *)
(*         *       GNU Lesser General Public License Version 2.1        *)
(************************************************************************)

module type S = sig

  module Cluster :
  sig
    type t
    val equal : t -> t -> bool
    val compare : t -> t -> int
    val to_string : t -> string
  end

  type node
  type ('edge,'info) t
  
  val empty : ('e,'i) t

  val add_edge : ('e,'i) t -> node -> 'e -> node -> ('e,'i) t
  val from_node : ('e,'i) t -> node -> (node * 'e) list
  val mem : ('e,'i) t -> node -> bool

  val iter : ('e,'i) t -> 
    (node -> Cluster.t option -> 'i option ->
      (node * 'e) list -> unit) -> unit

  val create_cluster : ('e,'i) t -> node list -> ('e,'i) t
  val cluster_of : ('e,'i) t -> node -> Cluster.t option

  val get_info : ('e,'i) t -> node -> 'i option
  val set_info : ('e,'i) t -> node -> 'i -> ('e,'i) t
  val clear_info : ('e,'i) t -> node -> ('e,'i) t

end

module Make(OT : Map.OrderedType) = struct

module Cluster =
struct
  type t = int
  let equal = Int.equal
  let compare = Int.compare
  let to_string = string_of_int
end

type node = OT.t

module NodeMap = Map.Make(OT)
module NodeSet = Set.Make(OT)

type ('edge,'info) t = {
  graph : (node * 'edge) list NodeMap.t;
  clusters : Cluster.t NodeMap.t;
  infos : 'info NodeMap.t;
}

let empty = {
  graph = NodeMap.empty;
  clusters = NodeMap.empty;
  infos = NodeMap.empty;
}

let mem { graph } id = NodeMap.mem id graph

let add_edge dag from trans dest = { dag with
  graph =
    let extra = [dest, trans] in
    try NodeMap.add from (extra @ NodeMap.find from dag.graph) dag.graph
    with Not_found -> NodeMap.add from extra dag.graph }

let from_node { graph } id = NodeMap.find id graph 

let clid = ref 1
let create_cluster dag l=
  incr clid;
  { dag with clusters =
     List.fold_right (fun x clusters ->
       NodeMap.add x !clid clusters) l dag.clusters }

let cluster_of dag id =
  try Some (NodeMap.find id dag.clusters)
  with Not_found -> None

let get_info dag id =
  try Some (NodeMap.find id dag.infos)
  with Not_found -> None

let set_info dag id info = { dag with infos = NodeMap.add id info dag.infos }

let clear_info dag id = { dag with infos = NodeMap.remove id dag.infos }

let iter dag f =
  NodeMap.iter (fun k v -> f k (cluster_of dag k) (get_info dag k) v) dag.graph

end