aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.ml
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-11-02 14:41:17 -0500
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-11-02 16:23:15 -0500
commitc920b420a27bd561967e316dcaca41d5e019a7b8 (patch)
tree0db30f3892d9ef24499917315c62d0d2e371a9b2 /tactics/tactics.ml
parent739d8e50b3681491bd82b516dbbba892ac5b424b (diff)
Fix bug #4151: discrepancy between exact and eexact/eassumption.
Diffstat (limited to 'tactics/tactics.ml')
-rw-r--r--tactics/tactics.ml5
1 files changed, 3 insertions, 2 deletions
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 0b920066f..56896bbc4 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -223,8 +223,9 @@ let convert_hyp_no_check = convert_hyp ~check:false
let convert_gen pb x y =
Proofview.Goal.enter begin fun gl ->
try
- let sigma = Tacmach.New.pf_apply Evd.conversion gl pb x y in
- Proofview.Unsafe.tclEVARS sigma
+ let sigma, b = Tacmach.New.pf_apply (Reductionops.infer_conv ~pb) gl x y in
+ if b then Proofview.Unsafe.tclEVARS sigma
+ else Tacticals.New.tclFAIL 0 (str "Not convertible")
with (* Reduction.NotConvertible *) _ ->
(** FIXME: Sometimes an anomaly is raised from conversion *)
Tacticals.New.tclFAIL 0 (str "Not convertible")