aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tacticals.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-04-06 00:04:26 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-04-22 11:23:36 +0200
commitf76c0b3b89ce433de5cad7d35c437ce26f1e7477 (patch)
treeb16c30fd84ed5d1fc4354a048c07b374df5720ec /tactics/tacticals.ml
parent4c6a5f56ef5ab248d9e816b4d7bee3001cab9a2e (diff)
Using the new monad tactic in Inv.
Diffstat (limited to 'tactics/tacticals.ml')
-rw-r--r--tactics/tacticals.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/tactics/tacticals.ml b/tactics/tacticals.ml
index 967b6d544..f1b52ebc7 100644
--- a/tactics/tacticals.ml
+++ b/tactics/tacticals.ml
@@ -542,8 +542,9 @@ module New = struct
(* Find the right elimination suffix corresponding to the sort of the goal *)
(* c should be of type A1->.. An->B with B an inductive definition *)
let general_elim_then_using mk_elim
- isrec allnames tac predicate ind indclause =
+ isrec allnames tac predicate ind (c, t) =
Proofview.Goal.enter begin fun gl ->
+ let indclause = Tacmach.New.of_old (fun gl -> mk_clenv_from gl (c, t)) gl in
let elim = Tacmach.New.of_old (mk_elim ind) gl in
(* applying elimination_scheme just a little modified *)
let elimclause = Tacmach.New.of_old (fun gls -> mk_clenv_from gls (elim,Tacmach.New.pf_type_of gl elim)) gl in
@@ -599,13 +600,12 @@ module New = struct
let elimination_then tac c =
Proofview.Goal.enter begin fun gl ->
let (ind,t) = pf_reduce_to_quantified_ind gl (pf_type_of gl c) in
- let indclause = Tacmach.New.of_old (fun gl -> mk_clenv_from gl (c,t)) gl in
let isrec,mkelim =
if (Global.lookup_mind (fst ind)).mind_record
then false,gl_make_case_dep
else true,gl_make_elim
in
- general_elim_then_using mkelim isrec None tac None ind indclause
+ general_elim_then_using mkelim isrec None tac None ind (c, t)
end
let case_then_using =