aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-05-08 18:59:55 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-05-08 19:59:03 +0200
commitf461e7657cab9917c5b405427ddba3d56f197efb (patch)
tree467ac699f78d0360b05174238aeb1177da892503 /tactics
parent9fe0471ef0127e9301d0450aacaeb1690abb82ad (diff)
Removing dead code and unused opens.
Diffstat (limited to 'tactics')
-rw-r--r--tactics/autorewrite.ml2
-rw-r--r--tactics/contradiction.ml2
-rw-r--r--tactics/eauto.ml13
-rw-r--r--tactics/eqdecide.ml2
-rw-r--r--tactics/tactics.ml1
5 files changed, 0 insertions, 20 deletions
diff --git a/tactics/autorewrite.ml b/tactics/autorewrite.ml
index 950eeef52..6d6e51536 100644
--- a/tactics/autorewrite.ml
+++ b/tactics/autorewrite.ml
@@ -15,10 +15,8 @@ open Term
open Termops
open Errors
open Util
-open Tacexpr
open Mod_subst
open Locus
-open Sigma.Notations
open Proofview.Notations
(* Rewriting rules *)
diff --git a/tactics/contradiction.ml b/tactics/contradiction.ml
index ab6fb37fd..26166bd83 100644
--- a/tactics/contradiction.ml
+++ b/tactics/contradiction.ml
@@ -6,14 +6,12 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-open Errors
open Term
open Hipattern
open Tactics
open Coqlib
open Reductionops
open Misctypes
-open Sigma.Notations
open Proofview.Notations
open Context.Named.Declaration
diff --git a/tactics/eauto.ml b/tactics/eauto.ml
index 9cfb805d4..6bbd9b2e8 100644
--- a/tactics/eauto.ml
+++ b/tactics/eauto.ml
@@ -17,12 +17,10 @@ open Proof_type
open Tacticals
open Tacmach
open Tactics
-open Patternops
open Clenv
open Auto
open Genredexpr
open Tacexpr
-open Misctypes
open Locus
open Locusops
open Hints
@@ -52,16 +50,6 @@ let registered_e_assumption =
(Tacmach.New.pf_ids_of_hyps gl))
end }
-let eval_uconstrs ist cs =
- let flags = {
- Pretyping.use_typeclasses = false;
- use_unif_heuristics = true;
- use_hook = Some Pfedit.solve_by_implicit_tactic;
- fail_evar = false;
- expand_evars = true
- } in
- List.map (fun c -> Pretyping.type_uconstr ~flags ist c) cs
-
(************************************************************************)
(* PROLOG tactic *)
(************************************************************************)
@@ -114,7 +102,6 @@ let prolog_tac l n =
end
open Auto
-open Unification
(***************************************************************************)
(* A tactic similar to Auto, but using EApply, Assumption and e_give_exact *)
diff --git a/tactics/eqdecide.ml b/tactics/eqdecide.ml
index 011296a8d..ef361d326 100644
--- a/tactics/eqdecide.ml
+++ b/tactics/eqdecide.ml
@@ -12,7 +12,6 @@
(* by Eduardo Gimenez *)
(************************************************************************)
-open Errors
open Util
open Names
open Namegen
@@ -27,7 +26,6 @@ open Hipattern
open Pretyping
open Tacmach.New
open Coqlib
-open Proofview.Notations
(* This file containts the implementation of the tactics ``Decide
Equality'' and ``Compare''. They can be used to decide the
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 0bb842601..2fe4d620e 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -4652,7 +4652,6 @@ let rec shrink ctx sign c t accu =
| _ -> assert false
let shrink_entry sign const =
- let open Context.Named.Declaration in
let open Entries in
let typ = match const.const_entry_type with
| None -> assert false