aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/funind/recdef.ml
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-11-08 21:09:53 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-11-08 21:09:53 +0000
commit6cf364b18897c61b3200ed9c5795c7b48cf23b59 (patch)
treeb6408927b2b16817fb12fee15b664a11db245958 /plugins/funind/recdef.ml
parent0077eb84e8eda65e5ac327aecba7e3fbf77ee016 (diff)
Porting Tactics.assumption to the new engine.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@17073 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/funind/recdef.ml')
-rw-r--r--plugins/funind/recdef.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/plugins/funind/recdef.ml b/plugins/funind/recdef.ml
index 881d930fc..64bf71ec6 100644
--- a/plugins/funind/recdef.ml
+++ b/plugins/funind/recdef.ml
@@ -517,7 +517,7 @@ let rec prove_lt hyple g =
(
tclTHENLIST[
apply (delayed_force lt_S_n);
- (observe_tac (str "assumption: " ++ Printer.pr_goal g) (h_assumption))
+ (observe_tac (str "assumption: " ++ Printer.pr_goal g) (Proofview.V82.of_tactic h_assumption))
])
)
end
@@ -757,7 +757,7 @@ let terminate_app_rec (f,args) expr_info continuation_tac _ =
tclTHENS (* proof of args < formal args *)
(apply (Lazy.force expr_info.acc_inv))
[
- observe_tac (str "h_assumption") h_assumption;
+ observe_tac (str "h_assumption") (Proofview.V82.of_tactic h_assumption);
tclTHENLIST
[
tclTRY(list_rewrite true
@@ -802,7 +802,7 @@ let rec prove_le g =
(List.hd args,List.hd (List.tl args))
in
tclFIRST[
- h_assumption;
+ Proofview.V82.of_tactic h_assumption;
apply (delayed_force le_n);
begin
try