aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/auto.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-17 14:26:02 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-17 15:44:38 +0200
commit90d64647d3fd5dbf5c337944dc0038f0b19b8a51 (patch)
treeb33528c72730ec541a75e3d0baaead6789f4dcb9 /tactics/auto.ml
parentd412844753ef25f4431c209f47b97b9fa498297d (diff)
Removing dead code.
Diffstat (limited to 'tactics/auto.ml')
-rw-r--r--tactics/auto.ml15
1 files changed, 0 insertions, 15 deletions
diff --git a/tactics/auto.ml b/tactics/auto.ml
index aa70d55cc..4f5f53ef0 100644
--- a/tactics/auto.ml
+++ b/tactics/auto.ml
@@ -141,12 +141,6 @@ type search_entry = stored_data list * stored_data list * Bounded_net.t
let empty_se = ([],[],Bounded_net.create ())
-let eq_constr_or_reference x y =
- match x, y with
- | IsConstr (x,_), IsConstr (y,_) -> eq_constr x y
- | IsGlobRef x, IsGlobRef y -> eq_gr x y
- | _, _ -> false
-
let eq_pri_auto_tactic (_, x) (_, y) =
if Int.equal x.pri y.pri && Option.equal constr_pattern_eq x.pat y.pat then
match x.code,y.code with
@@ -189,11 +183,6 @@ let is_transparent_gr (ids, csts) = function
let dummy_goal = Goal.V82.dummy_goal
-let instantiate_constr_or_ref env sigma c =
- let c, ctx = Universes.fresh_global_or_constr_instance env c in
- let cty = Retyping.get_type_of env sigma c in
- (c, cty), ctx
-
let strip_params env c =
match kind_of_term c with
| App (f, args) ->
@@ -875,10 +864,6 @@ let (forward_intern_tac, extern_intern_tac) = Hook.make ()
type hnf = bool
-let pr_hint_term = function
- | IsConstr (c,_) -> pr_constr c
- | IsGlobRef gr -> pr_global gr
-
type hints_entry =
| HintsResolveEntry of (int option * polymorphic * hnf * hints_path_atom * hint_term) list
| HintsImmediateEntry of (hints_path_atom * polymorphic * hint_term) list