aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-08-23 00:58:17 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-08-23 00:58:17 +0200
commit47fbb3a74b9bd52b19e63e695fb1902ed345488e (patch)
tree1fa04bcc4d12d45b5682cb87447b289ced3b6a6a /tactics/tactics.ml
parenta67cc6941434124465f20b14a1256f2ede31a60e (diff)
Tactics.unify in the new monad.
Diffstat (limited to 'tactics/tactics.ml')
-rw-r--r--tactics/tactics.ml10
1 files changed, 6 insertions, 4 deletions
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 7a8bb36b9..5c76ce776 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -4004,7 +4004,8 @@ let admit_as_an_axiom =
(* gl *)
(* >>>>>>> .merge_file_iUuzZK *)
-let unify ?(state=full_transparent_state) x y gl =
+let unify ?(state=full_transparent_state) x y =
+ Proofview.Goal.enter begin fun gl ->
try
let flags =
{(default_unify_flags ()) with
@@ -4013,9 +4014,10 @@ let unify ?(state=full_transparent_state) x y gl =
modulo_delta_in_merge = Some state;
modulo_conv_on_closed_terms = Some state}
in
- let evd = w_unify (pf_env gl) (project gl) Reduction.CONV ~flags x y
- in tclEVARS evd gl
- with e when Errors.noncritical e -> tclFAIL 0 (str"Not unifiable") gl
+ let evd = w_unify (Tacmach.New.pf_env gl) (Proofview.Goal.sigma gl) Reduction.CONV ~flags x y
+ in Proofview.V82.tclEVARS evd
+ with e when Errors.noncritical e -> Tacticals.New.tclFAIL 0 (str"Not unifiable")
+ end
module Simple = struct
(** Simplified version of some of the above tactics *)