aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eauto.ml4
diff options
context:
space:
mode:
Diffstat (limited to 'tactics/eauto.ml4')
-rw-r--r--tactics/eauto.ml48
1 files changed, 0 insertions, 8 deletions
diff --git a/tactics/eauto.ml4 b/tactics/eauto.ml4
index 6c3c55efd..0ab426cd2 100644
--- a/tactics/eauto.ml4
+++ b/tactics/eauto.ml4
@@ -58,8 +58,6 @@ let registered_e_assumption gl =
(*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 =
@@ -201,10 +199,6 @@ module SearchProblem = struct
let pr_ev evs ev = Printer.pr_constr_env (Evd.evar_env ev) (Evarutil.nf_evar evs ev.Evd.evar_concl)
- let pr_goals gls =
- let evars = Evarutil.nf_evar_map (Refiner.project gls) in
- prlist (pr_ev evars) (sig_it gls)
-
let filter_tactics glls l =
(* let _ = Proof_trees.db_pr_goal (List.hd (sig_it glls)) in *)
(* let evars = Evarutil.nf_evars (Refiner.project glls) in *)
@@ -489,8 +483,6 @@ let autounfold_tac db cls gl =
in
autounfold dbs cls gl
-open Extraargs
-
TACTIC EXTEND autounfold
| [ "autounfold" hintbases(db) clause(cl) ] -> [ Proofview.V82.tactic (autounfold_tac db cl) ]
END