aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/dn.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-03-03 02:22:56 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-03-03 02:34:17 +0100
commit37f624d80e82d655021f2beb7d72794a120ff8b5 (patch)
tree35954a2abc642ebc3f8a2cec54082bf43dcde7f7 /tactics/dn.mli
parentb076e7f88124db576c4f3c06e2ac93673236be7a (diff)
Extruding code not depending of the functor argument in Termdn.
Diffstat (limited to 'tactics/dn.mli')
-rw-r--r--tactics/dn.mli30
1 files changed, 12 insertions, 18 deletions
diff --git a/tactics/dn.mli b/tactics/dn.mli
index 662ac19af..bab925a20 100644
--- a/tactics/dn.mli
+++ b/tactics/dn.mli
@@ -1,48 +1,42 @@
+type 'res lookup_res = Label of 'res | Nothing | Everything
-
-
-
-
-
-module Make :
+module Make :
functor (X : Set.OrderedType) ->
functor (Y : Map.OrderedType) ->
functor (Z : Map.OrderedType) ->
sig
type decompose_fun = X.t -> (Y.t * X.t list) option
-
+
type t
val create : unit -> t
-
+
(** [add t f (tree,inf)] adds a structured object [tree] together with
the associated information [inf] to the table [t]; the function
[f] is used to translated [tree] into its prefix decomposition: [f]
must decompose any tree into a label characterizing its root node and
the list of its subtree *)
-
+
val add : t -> decompose_fun -> X.t * Z.t -> t
-
+
val rmv : t -> decompose_fun -> X.t * Z.t -> t
-
- type 'res lookup_res = Label of 'res | Nothing | Everything
-
+
type 'tree lookup_fun = 'tree -> (Y.t * 'tree list) lookup_res
-
+
(** [lookup t f tree] looks for trees (and their associated
information) in table [t] such that the structured object [tree]
matches against them; [f] is used to translated [tree] into its
prefix decomposition: [f] must decompose any tree into a label
characterizing its root node and the list of its subtree *)
-
+
val lookup : t -> 'term lookup_fun -> 'term
-> (X.t * Z.t) list
-
+
val app : ((X.t * Z.t) -> unit) -> t -> unit
-
+
val skip_arg : int -> t -> (t * bool) list
-
+
end