aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-02-14 15:55:35 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-02-14 15:55:35 +0000
commita7de8633c23fe66ee32463d78dae89661805c2d1 (patch)
tree641c081a3e43215a62970c882a5cf93276ff39c6 /tactics
parenta0ea7fc67d18598e88559a133cac6b1d993ec66c (diff)
Centralisation des références à des globaux de Coq dans Coqlib (ex-Stdlib) et suppression Stock
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1386 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics')
-rw-r--r--tactics/equality.mli16
1 files changed, 0 insertions, 16 deletions
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