aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/auto.ml
diff options
context:
space:
mode:
Diffstat (limited to 'tactics/auto.ml')
-rw-r--r--tactics/auto.ml10
1 files changed, 5 insertions, 5 deletions
diff --git a/tactics/auto.ml b/tactics/auto.ml
index 0dc0a9f4c..66454059e 100644
--- a/tactics/auto.ml
+++ b/tactics/auto.ml
@@ -44,10 +44,10 @@ open Tacexpr
(****************************************************************************)
type auto_tactic =
- | Res_pf of constr * wc clausenv (* Hint Apply *)
- | ERes_pf of constr * wc clausenv (* Hint EApply *)
+ | Res_pf of constr * clausenv (* Hint Apply *)
+ | ERes_pf of constr * clausenv (* Hint EApply *)
| Give_exact of constr
- | Res_pf_THEN_trivial_fail of constr * wc clausenv (* Hint Immediate *)
+ | Res_pf_THEN_trivial_fail of constr * clausenv (* Hint Immediate *)
| Unfold_nth of global_reference (* Hint Unfold *)
| Extern of glob_tactic_expr (* Hint Extern *)
@@ -195,7 +195,7 @@ let make_apply_entry env sigma (eapply,verbose) name (c,cty) =
match kind_of_term cty with
| Prod _ ->
let ce = mk_clenv_from dummy_goal (c,cty) in
- let c' = (clenv_template_type ce).rebus in
+ let c' = clenv_type ce in
let pat = Pattern.pattern_of_constr c' in
let hd = (try head_pattern_bound pat
with BoundPattern -> failwith "make_apply_entry") in
@@ -263,7 +263,7 @@ let make_trivial env sigma (name,c) =
let ce = mk_clenv_from dummy_goal (c,t) in
(hd, { hname = name;
pri=1;
- pat = Some (Pattern.pattern_of_constr (clenv_template_type ce).rebus);
+ pat = Some (Pattern.pattern_of_constr (clenv_type ce));
code=Res_pf_THEN_trivial_fail(c,ce) })
open Vernacexpr