aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-04-06 19:08:11 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-04-06 19:18:11 +0200
commitaba9691ef2d8d6ffd184e3d97de47d9c48f1a1b3 (patch)
tree1dfc529b52c8a46d80bf82305b4b20c908a64c6b /tactics
parentb3b302837a5a9ff4e50a7f69ecb3fb333c94bf01 (diff)
Removing unused functions in Refiner.
Diffstat (limited to 'tactics')
-rw-r--r--tactics/eauto.ml421
1 files changed, 21 insertions, 0 deletions
diff --git a/tactics/eauto.ml4 b/tactics/eauto.ml4
index 21c5a88c7..65f030742 100644
--- a/tactics/eauto.ml4
+++ b/tactics/eauto.ml4
@@ -56,6 +56,27 @@ let registered_e_assumption gl =
(* PROLOG tactic *)
(************************************************************************)
+(*s Tactics handling a list of goals. *)
+
+type tactic_list = (goal list sigma) -> (goal list sigma)
+
+(* first_goal : goal list sigma -> goal sigma *)
+
+let first_goal gls =
+ let gl = gls.Evd.it and sig_0 = gls.Evd.sigma in
+ if List.is_empty gl then error "first_goal";
+ { Evd.it = List.hd gl; Evd.sigma = sig_0; }
+
+(* tactic -> tactic_list : Apply a tactic to the first goal in the list *)
+
+let apply_tac_list tac glls =
+ let (sigr,lg) = unpackage glls in
+ match lg with
+ | (g1::rest) ->
+ let gl = apply_sig_tac sigr tac g1 in
+ repackage sigr (gl@rest)
+ | _ -> error "apply_tac_list"
+
let one_step l gl =
[Proofview.V82.of_tactic Tactics.intro]
@ (List.map Tactics.Simple.eapply (List.map mkVar (pf_ids_of_hyps gl)))