aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/matching.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-01-21 17:18:23 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-01-21 17:18:23 +0000
commitd7b2414b631d71e89e677d650b84bd4fadd44895 (patch)
tree47b653e7e0ae9b83dbc8a96b2c5be4717b2eefbd /pretyping/matching.mli
parentea6bd4e5496f0fd7e059cd9b924f29ca80a38ae2 (diff)
Compatibilité ocamlweb pour cible doc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@6616 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping/matching.mli')
-rw-r--r--pretyping/matching.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/pretyping/matching.mli b/pretyping/matching.mli
index 2b0b8f240..b4f6c3245 100644
--- a/pretyping/matching.mli
+++ b/pretyping/matching.mli
@@ -40,7 +40,7 @@ val is_matching : constr_pattern -> constr -> bool
val matches_conv :env -> Evd.evar_map -> constr_pattern -> constr -> patvar_map
(* [match_subterm n pat c] returns the substitution and the context
- corresponding to the [n+1]th _closed_ subterm of [c] matching [pat];
+ corresponding to the [n+1]th **closed** subterm of [c] matching [pat];
It raises PatternMatchingFailure if no such matching exists *)
val match_subterm : int -> constr_pattern -> constr -> patvar_map * constr