aboutsummaryrefslogtreecommitdiff
path: root/proofs
diff options
context:
space:
mode:
Diffstat (limited to 'proofs')
-rw-r--r--proofs/refiner.ml2
-rw-r--r--proofs/refiner.mli2
2 files changed, 0 insertions, 4 deletions
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index 3c6a5d1694..8e413c7a88 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -21,8 +21,6 @@ let project x = x.sigma
let pf_env gls = Global.env_of_context (Goal.V82.hyps (project gls) (sig_it gls))
let pf_hyps gls = EConstr.named_context_of_val (Goal.V82.hyps (project gls) (sig_it gls))
-let refiner = Logic.refiner
-
(* A special exception for levels for the Fail tactic *)
exception FailError of int * Pp.t Lazy.t
diff --git a/proofs/refiner.mli b/proofs/refiner.mli
index 0ea630fdbc..18ac5f4a76 100644
--- a/proofs/refiner.mli
+++ b/proofs/refiner.mli
@@ -22,8 +22,6 @@ val project : 'a sigma -> evar_map
val pf_env : Goal.goal sigma -> Environ.env
val pf_hyps : Goal.goal sigma -> named_context
-val refiner : check:bool -> Constr.t -> unit Proofview.tactic
-
(** A special exception for levels for the Fail tactic *)
exception FailError of int * Pp.t Lazy.t