From ecb17841e955ca888010d72876381a86cdcf09ad Mon Sep 17 00:00:00 2001 From: clrenard Date: Mon, 12 Nov 2001 15:56:10 +0000 Subject: 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 --- proofs/proof_type.ml | 7 +------ 1 file changed, 1 insertion(+), 6 deletions(-) (limited to 'proofs/proof_type.ml') diff --git a/proofs/proof_type.ml b/proofs/proof_type.ml index 81c57e5390..9965488c9f 100644 --- a/proofs/proof_type.ml +++ b/proofs/proof_type.ml @@ -9,7 +9,6 @@ open Environ open Evd open Names -open Stamps open Term open Util (*i*) @@ -55,14 +54,10 @@ type prim_rule = { params : Coqast.t list; terms : constr list } -(* A global constraint is a mappings of existential variables - with some extra information for the program tactic *) -type global_constraints = evar_map timestamped - (* Signature useful to define the tactic type *) type 'a sigma = { it : 'a ; - sigma : global_constraints } + sigma : evar_map } (*s Proof trees. [ref] = [None] if the goal has still to be proved, -- cgit v1.2.3