aboutsummaryrefslogtreecommitdiffhomepage
path: root/ltac/g_class.ml4
diff options
context:
space:
mode:
Diffstat (limited to 'ltac/g_class.ml4')
-rw-r--r--ltac/g_class.ml46
1 files changed, 3 insertions, 3 deletions
diff --git a/ltac/g_class.ml4 b/ltac/g_class.ml4
index b7f0881f1..f47c03dfc 100644
--- a/ltac/g_class.ml4
+++ b/ltac/g_class.ml4
@@ -74,7 +74,7 @@ TACTIC EXTEND is_ground
END
TACTIC EXTEND autoapply
- [ "autoapply" constr(c) "using" preident(i) ] -> [ Proofview.V82.tactic (autoapply c i) ]
+ [ "autoapply" constr(c) "using" preident(i) ] -> [ autoapply c i ]
END
(** TODO: DEPRECATE *)
@@ -90,10 +90,10 @@ let rec eq_constr_mod_evars sigma x y =
| _, _ -> compare_constr sigma (fun x y -> eq_constr_mod_evars sigma x y) x y
let progress_evars t =
- Proofview.Goal.nf_enter { enter = begin fun gl ->
+ Proofview.Goal.enter { enter = begin fun gl ->
let concl = Proofview.Goal.concl gl in
let check =
- Proofview.Goal.nf_enter { enter = begin fun gl' ->
+ Proofview.Goal.enter { enter = begin fun gl' ->
let sigma = Tacmach.New.project gl' in
let newconcl = Proofview.Goal.concl gl' in
if eq_constr_mod_evars sigma concl newconcl