aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/quote
diff options
context:
space:
mode:
authorGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-11-02 15:34:15 +0000
committerGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-11-02 15:34:15 +0000
commit6e42eb07daf38213853bf4a9b9008c0e9e67f224 (patch)
tree7fafc79f2e3773aa9d247c56f4c1f2915556337a /plugins/quote
parent84357f0d15a1137a4b1cc5cacb86d3af5c1ca93e (diff)
Clean-up: removed redundant notations (>>-) and (>>--) from Proofview.Notations.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16971 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/quote')
-rw-r--r--plugins/quote/quote.ml18
1 files changed, 9 insertions, 9 deletions
diff --git a/plugins/quote/quote.ml b/plugins/quote/quote.ml
index 80053ea4d..bf061095c 100644
--- a/plugins/quote/quote.ml
+++ b/plugins/quote/quote.ml
@@ -453,11 +453,11 @@ let quote_terms ivs lc =
yet. *)
let quote f lid =
- Tacmach.New.pf_global f >>- fun f ->
- Proofview.Goal.lift (Goal.sensitive_list_map Tacmach.New.pf_global_sensitive lid) >>- fun cl ->
- Proofview.Goal.lift (compute_ivs f cl) >>- fun ivs ->
- Proofview.Goal.concl >>- fun concl ->
- Proofview.Goal.lift (quote_terms ivs [concl]) >>- fun quoted_terms ->
+ Tacmach.New.pf_global f >>= fun f ->
+ Proofview.Goal.lift (Goal.sensitive_list_map Tacmach.New.pf_global_sensitive lid) >>= fun cl ->
+ Proofview.Goal.lift (compute_ivs f cl) >>= fun ivs ->
+ Proofview.Goal.concl >>= fun concl ->
+ Proofview.Goal.lift (quote_terms ivs [concl]) >>= fun quoted_terms ->
let (p, vm) = match quoted_terms with
| [p], vm -> (p,vm)
| _ -> assert false
@@ -467,10 +467,10 @@ let quote f lid =
| Some _ -> Proofview.V82.tactic (Tactics.convert_concl (mkApp (f, [| vm; p |])) DEFAULTcast)
let gen_quote cont c f lid =
- Tacmach.New.pf_global f >>- fun f ->
- Proofview.Goal.lift (Goal.sensitive_list_map Tacmach.New.pf_global_sensitive lid) >>- fun cl ->
- Proofview.Goal.lift (compute_ivs f cl) >>- fun ivs ->
- Proofview.Goal.lift (quote_terms ivs [c]) >>- fun quoted_terms ->
+ Tacmach.New.pf_global f >>= fun f ->
+ Proofview.Goal.lift (Goal.sensitive_list_map Tacmach.New.pf_global_sensitive lid) >>= fun cl ->
+ Proofview.Goal.lift (compute_ivs f cl) >>= fun ivs ->
+ Proofview.Goal.lift (quote_terms ivs [c]) >>= fun quoted_terms ->
let (p, vm) = match quoted_terms with
| [p], vm -> (p,vm)
| _ -> assert false