aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-08 16:13:37 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-08 16:13:37 +0000
commit47e5f716f7ded0eec43b00d49955d56c370c3596 (patch)
treee7fbe16925eacc72bdd9ebeb65c2a20b8bb0eef0 /pretyping
parent70f8c345685278a567fbb075f222c79f0533e90e (diff)
- Extension de "generalize" en "generalize c as id at occs".
- Ajout clause "in" à "remember" (et passage du code en ML). - Ajout clause "in" à "induction"/"destruct" qui, en ce cas, ajoute aussi une égalité pour se souvenir du terme sur lequel l'induction ou l'analyse de cas s'applique. - Ajout "pose t as id" en standard (Matthieu: j'ai enlevé celui de Programs qui avait la sémantique de "pose proof" tandis que le nouveau a la même sémantique que "pose (id:=t)"). - Un peu de réorganisation, uniformisation de noms dans Arith, et ajout EqNat dans Arith. - Documentation tactiques et notations de tactiques. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11072 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping')
-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