aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--contrib/ring/quote.ml7
-rw-r--r--tactics/equality.mli16
2 files changed, 5 insertions, 18 deletions
diff --git a/contrib/ring/quote.ml b/contrib/ring/quote.ml
index ed93a13dc..44cbd7868 100644
--- a/contrib/ring/quote.ml
+++ b/contrib/ring/quote.ml
@@ -113,8 +113,11 @@ open Proof_type
the constants are loaded in the environment *)
let constant dir s =
- Declare.global_absolute_reference
- (make_path ("Coq"::"ring"::dir) (id_of_string s) CCI)
+ let dir = "Coq"::"ring"::dir in
+ try
+ Declare.global_reference_in_absolute_module dir (id_of_string s)
+ with Not_found ->
+ anomaly ("Quote: cannot find "^(string_of_qualid (make_qualid dir s)))
let coq_Empty_vm = lazy (constant ["Quote"] "Empty_vm")
let coq_Node_vm = lazy (constant ["Quote"] "Node_vm")
diff --git a/tactics/equality.mli b/tactics/equality.mli
index 69777da3e..d1543e47e 100644
--- a/tactics/equality.mli
+++ b/tactics/equality.mli
@@ -16,22 +16,6 @@ open Tacticals
open Tactics
(*i*)
-type leibniz_eq = {
- eq : marked_term;
- ind : marked_term;
- rrec : marked_term option;
- rect : marked_term option;
- congr: marked_term;
- sym : marked_term }
-
-val eq : leibniz_eq
-val eqT : leibniz_eq
-val idT : leibniz_eq
-
-val eq_pattern : unit -> constr_pattern
-val eqT_pattern : unit -> constr_pattern
-val idT_pattern : unit -> constr_pattern
-
val find_eq_pattern : sorts -> sorts -> constr
val general_rewrite_bindings : bool -> (constr * constr substitution) -> tactic