aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/termops.mli
diff options
context:
space:
mode:
Diffstat (limited to 'pretyping/termops.mli')
-rw-r--r--pretyping/termops.mli12
1 files changed, 6 insertions, 6 deletions
diff --git a/pretyping/termops.mli b/pretyping/termops.mli
index 22a370aaf..bc483cfc3 100644
--- a/pretyping/termops.mli
+++ b/pretyping/termops.mli
@@ -131,16 +131,16 @@ val subst_term : constr -> constr -> constr
(* [replace_term d e c] replaces [d] by [e] in [c] *)
val replace_term : constr -> constr -> constr -> constr
-(* [subst_term_occ occl c d] replaces occurrences of [Rel 1] at
- positions [occl] by [c] in [d] *)
+(* [subst_term_occ_gen occl n c d] replaces occurrences of [c] at
+ positions [occl], counting from [n], by [Rel 1] in [d] *)
val subst_term_occ_gen : int list -> int -> constr -> types -> int * types
-(* [subst_term_occ occl c d] replaces occurrences of [Rel 1] at
- positions [occl] by [c] in [d] (see also Note OCC) *)
+(* [subst_term_occ occl c d] replaces occurrences of [c] at
+ positions [occl] by [Rel 1] in [d] (see also Note OCC) *)
val subst_term_occ : int list -> constr -> constr -> constr
-(* [subst_term_occ_decl occl c decl] replaces occurrences of [Rel 1] at
- positions [occl] by [c] in [decl] *)
+(* [subst_term_occ_decl occl c decl] replaces occurrences of [c] at
+ positions [occl] by [Rel 1] in [decl] *)
val subst_term_occ_decl :
int list -> constr -> named_declaration -> named_declaration