src/Tools/Metis/src/Lazy.sig
author haftmann
Sat, 06 Mar 2010 09:58:30 +0100
changeset 35607 896f01fe825b
parent 23510 4521fead5609
child 39353 7f11d833d65b
permissions -rw-r--r--
added dom_option_map, map_of_map_keys

(* ========================================================================= *)
(* SUPPORT FOR LAZY EVALUATION                                               *)
(* Copyright (c) 2007 Joe Hurd, distributed under the BSD License      *)
(* ========================================================================= *)

signature Lazy =
sig

type 'a lazy

val delay : (unit -> 'a) -> 'a lazy

val force : 'a lazy -> 'a

val memoize : (unit -> 'a) -> unit -> 'a

end