aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/extratactics.ml4
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-04-27 19:37:33 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-04-27 19:37:33 +0000
commit61d11c649b4cd68e92861e2fea86f6c6a6b5bb6a (patch)
treeff162856b856b8fa11ac367ecf9bfa4a9de29034 /tactics/extratactics.ml4
parent2ec958c3c8d2942242837787a3941abb14702b5c (diff)
Standardisation nom option_app en option_map
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8752 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/extratactics.ml4')
-rw-r--r--tactics/extratactics.ml42
1 files changed, 1 insertions, 1 deletions
diff --git a/tactics/extratactics.ml4 b/tactics/extratactics.ml4
index 97aeedc6b..1c0e04276 100644
--- a/tactics/extratactics.ml4
+++ b/tactics/extratactics.ml4
@@ -80,7 +80,7 @@ END
TACTIC EXTEND replace
| ["replace" constr(c1) "with" constr(c2) in_arg_hyp(in_hyp) by_arg_tac(tac) ] ->
- [ new_replace c1 c2 in_hyp (Util.option_app Tacinterp.eval_tactic tac) ]
+ [ new_replace c1 c2 in_hyp (Util.option_map Tacinterp.eval_tactic tac) ]
END
(* Julien: