aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar clrenard <clrenard@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-11-12 15:56:10 +0000
committerGravatar clrenard <clrenard@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-11-12 15:56:10 +0000
commitecb17841e955ca888010d72876381a86cdcf09ad (patch)
tree4c6c24f6ce5a8221f8632fceb0f6717948cdca8d /tactics
parent2f611e10fb3dc42fc00d80b1e087fa33f6fc846e (diff)
Suppression des stamps et donc des *_constraints
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2186 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics')
-rw-r--r--tactics/tacticals.ml2
-rw-r--r--tactics/tactics.ml1
-rw-r--r--tactics/tactics.mli3
-rw-r--r--tactics/wcclausenv.ml2
-rw-r--r--tactics/wcclausenv.mli2
5 files changed, 5 insertions, 5 deletions
diff --git a/tactics/tacticals.ml b/tactics/tacticals.ml
index b71f7ab2a..70f30187d 100644
--- a/tactics/tacticals.ml
+++ b/tactics/tacticals.ml
@@ -129,7 +129,7 @@ let pf_is_matching gls pat n =
is_matching_conv (w_env wc) (w_Underlying wc) pat n
let pf_matches gls pat n =
- matches_conv (pf_env gls) (Stamps.ts_it (sig_sig gls)) pat n
+ matches_conv (pf_env gls) (project gls) pat n
(* [OnCL clausefinder clausetac]
* executes the clausefinder to find the clauses, and then executes the
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 804555583..c9247c09e 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -10,7 +10,6 @@
open Pp
open Util
-open Stamps
open Names
open Nameops
open Sign
diff --git a/tactics/tactics.mli b/tactics/tactics.mli
index 60d48530c..b91aa09e6 100644
--- a/tactics/tactics.mli
+++ b/tactics/tactics.mli
@@ -12,6 +12,7 @@
open Names
open Term
open Environ
+open Sign
open Tacmach
open Proof_type
open Reduction
@@ -27,7 +28,7 @@ open Nametab
(*s General functions. *)
-val type_clenv_binding : walking_constraints ->
+val type_clenv_binding : named_context sigma ->
constr * constr -> constr substitution -> constr
val string_of_inductive : constr -> string
diff --git a/tactics/wcclausenv.ml b/tactics/wcclausenv.ml
index 0df646c0c..3b93cce07 100644
--- a/tactics/wcclausenv.ml
+++ b/tactics/wcclausenv.ml
@@ -28,7 +28,7 @@ open Evar_refiner
write to Eduardo.Gimenez@inria.fr and ask for the prize :-)
-- Eduardo (11/8/97) *)
-type wc = walking_constraints
+type wc = named_context sigma
let pf_get_new_id id gls =
next_ident_away id (pf_ids_of_hyps gls)
diff --git a/tactics/wcclausenv.mli b/tactics/wcclausenv.mli
index cd88cc1b5..24174e508 100644
--- a/tactics/wcclausenv.mli
+++ b/tactics/wcclausenv.mli
@@ -32,7 +32,7 @@ type arg_binder =
type arg_bindings = (arg_binder * constr) list
-type wc = walking_constraints
+type wc = named_context sigma
val clenv_constrain_with_bindings : arg_bindings -> wc clausenv -> wc clausenv