aboutsummaryrefslogtreecommitdiffhomepage
path: root/engine/eConstr.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-05-19 21:24:55 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-05-19 21:25:59 +0200
commit8bd3e4eba54ace61f49a53b8ce74517de71006ec (patch)
tree4ca4c75f1628e7500aae6d7d129eb9df72191f9d /engine/eConstr.mli
parent234dc568769602cb91655929a344027a15f52845 (diff)
Exporting some functions of vars.ml as functions operating on EConstr.
Diffstat (limited to 'engine/eConstr.mli')
-rw-r--r--engine/eConstr.mli13
1 files changed, 11 insertions, 2 deletions
diff --git a/engine/eConstr.mli b/engine/eConstr.mli
index 693b592fd..9d705b4d5 100644
--- a/engine/eConstr.mli
+++ b/engine/eConstr.mli
@@ -205,12 +205,21 @@ val fold : Evd.evar_map -> ('a -> t -> 'a) -> 'a -> t -> 'a
module Vars :
sig
+
+(** See vars.mli for the documentation of the functions below *)
+
+type substl = t list
+
val lift : int -> t -> t
val liftn : int -> int -> t -> t
-val substnl : t list -> int -> t -> t
-val substl : t list -> t -> t
+val substnl : substl -> int -> t -> t
+val substl : substl -> t -> t
val subst1 : t -> t -> t
+val substnl_decl : substl -> int -> rel_declaration -> rel_declaration
+val substl_decl : substl -> rel_declaration -> rel_declaration
+val subst1_decl : t -> rel_declaration -> rel_declaration
+
val replace_vars : (Id.t * t) list -> t -> t
val substn_vars : int -> Id.t list -> t -> t
val subst_vars : Id.t list -> t -> t