aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-23 17:48:13 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-24 13:52:34 +0200
commit89dc208ff140ba6ecd7b2c931401f9c58fb2985e (patch)
treedbc00054387bce1ab4c7452ea13d0900afe7201a /proofs
parentefa3add0c03b70ecda3890cc6c69e66850605e7d (diff)
Clenvtac.res_pf is in the new tactic monad.
Diffstat (limited to 'proofs')
-rw-r--r--proofs/clenvtac.ml6
-rw-r--r--proofs/clenvtac.mli2
2 files changed, 5 insertions, 3 deletions
diff --git a/proofs/clenvtac.ml b/proofs/clenvtac.ml
index 941d789dd..e8af6ffbd 100644
--- a/proofs/clenvtac.ml
+++ b/proofs/clenvtac.ml
@@ -78,8 +78,10 @@ open Unification
let dft = default_unify_flags
-let res_pf clenv ?(with_evars=false) ?(flags=dft ()) gls =
- clenv_refine with_evars (clenv_unique_resolver ~flags clenv gls) gls
+let res_pf clenv ?(with_evars=false) ?(flags=dft ()) =
+ Proofview.V82.tactic begin fun gl ->
+ clenv_refine with_evars (clenv_unique_resolver ~flags clenv gl) gl
+ end
(* [unifyTerms] et [unify] ne semble pas gérer les Meta, en
particulier ne semblent pas vérifier que des instances différentes
diff --git a/proofs/clenvtac.mli b/proofs/clenvtac.mli
index 3cfe1f315..eea32019e 100644
--- a/proofs/clenvtac.mli
+++ b/proofs/clenvtac.mli
@@ -15,7 +15,7 @@ open Unification
(** Tactics *)
val unify : ?flags:unify_flags -> constr -> unit Proofview.tactic
val clenv_refine : evars_flag -> ?with_classes:bool -> clausenv -> tactic
-val res_pf : clausenv -> ?with_evars:evars_flag -> ?flags:unify_flags -> tactic
+val res_pf : clausenv -> ?with_evars:evars_flag -> ?flags:unify_flags -> unit Proofview.tactic
val clenv_pose_dependent_evars : evars_flag -> clausenv -> clausenv
val clenv_value_cast_meta : clausenv -> constr