aboutsummaryrefslogtreecommitdiff
path: root/plugins/micromega/persistent_cache.mli
diff options
context:
space:
mode:
Diffstat (limited to 'plugins/micromega/persistent_cache.mli')
-rw-r--r--plugins/micromega/persistent_cache.mli33
1 files changed, 15 insertions, 18 deletions
diff --git a/plugins/micromega/persistent_cache.mli b/plugins/micromega/persistent_cache.mli
index cb14d73972..7d459a66e7 100644
--- a/plugins/micromega/persistent_cache.mli
+++ b/plugins/micromega/persistent_cache.mli
@@ -10,32 +10,29 @@
open Hashtbl
-module type PHashtable =
- sig
- type 'a t
- type key
+module type PHashtable = sig
+ type 'a t
+ type key
- val open_in : string -> 'a t
- (** [open_in f] rebuilds a table from the records stored in file [f].
+ val open_in : string -> 'a t
+ (** [open_in f] rebuilds a table from the records stored in file [f].
As marshaling is not type-safe, it might segfault.
*)
- val find : 'a t -> key -> 'a
- (** find has the specification of Hashtable.find *)
+ val find : 'a t -> key -> 'a
+ (** find has the specification of Hashtable.find *)
- val add : 'a t -> key -> 'a -> unit
- (** [add tbl key elem] adds the binding [key] [elem] to the table [tbl].
+ val add : 'a t -> key -> 'a -> unit
+ (** [add tbl key elem] adds the binding [key] [elem] to the table [tbl].
(and writes the binding to the file associated with [tbl].)
If [key] is already bound, raises KeyAlreadyBound *)
- val memo : string -> (key -> 'a) -> (key -> 'a)
- (** [memo cache f] returns a memo function for [f] using file [cache] as persistent table.
+ val memo : string -> (key -> 'a) -> key -> 'a
+ (** [memo cache f] returns a memo function for [f] using file [cache] as persistent table.
Note that the cache will only be loaded when the function is used for the first time *)
- val memo_cond : string -> (key -> bool) -> (key -> 'a) -> (key -> 'a)
- (** [memo cache cond f] only use the cache if [cond k] holds for the key [k]. *)
+ val memo_cond : string -> (key -> bool) -> (key -> 'a) -> key -> 'a
+ (** [memo cache cond f] only use the cache if [cond k] holds for the key [k]. *)
+end
-
- end
-
-module PHashtable(Key:HashedType) : PHashtable with type key = Key.t
+module PHashtable (Key : HashedType) : PHashtable with type key = Key.t