aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-12-07 23:21:07 +0000
committerGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-12-07 23:21:07 +0000
commitd0f57e4e8b9d8feaadf96a241d3546ba061eb20c (patch)
treec5543fd14d187ccd6fe47d295718c802cb5b24e7 /proofs
parent47c78072c71b34c4c5469736367234f43203e7c9 (diff)
Adding the tactic "instantiate" (without argument), to force the
instantiation of evars in tacticals (cf r9985, r10294). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10356 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs')
-rw-r--r--proofs/refiner.ml7
-rw-r--r--proofs/refiner.mli4
2 files changed, 7 insertions, 4 deletions
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index 76fe0129f..7010153ba 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -223,9 +223,7 @@ let refiner = function
ref = Some(Daimon,[])})
-let local_Constraints gl = refiner (Prim Change_evars) gl
-
-let norm_evar_tac = local_Constraints
+let norm_evar_tac gl = refiner (Prim Change_evars) gl
let norm_evar_proof sigma pf =
let nf_subgoal i sgl =
@@ -312,6 +310,9 @@ let idtac_valid = function
(* [goal_goal_list : goal sigma -> goal list sigma] *)
let goal_goal_list gls = {it=[gls.it];sigma=gls.sigma}
+(* forces propagation of evar constraints *)
+let tclNORMEVAR = norm_evar_tac
+
(* identity tactic without any message *)
let tclIDTAC gls = (goal_goal_list gls, idtac_valid)
diff --git a/proofs/refiner.mli b/proofs/refiner.mli
index 530a72a37..ba092e89e 100644
--- a/proofs/refiner.mli
+++ b/proofs/refiner.mli
@@ -47,7 +47,6 @@ val frontier : transformation_tactic
val list_pf : proof_tree -> goal list
val unTAC : tactic -> goal sigma -> proof_tree sigma
-val local_Constraints : tactic
(* [frontier_map f n p] applies f on the n-th open subgoal of p and
rebuilds proof-tree.
@@ -61,6 +60,9 @@ val frontier_mapi :
(*s Tacticals. *)
+(* [tclNORMEVAR] forces propagation of evar constraints *)
+val tclNORMEVAR : tactic
+
(* [tclIDTAC] is the identity tactic without message printing*)
val tclIDTAC : tactic
val tclIDTAC_MESSAGE : Pp.std_ppcmds -> tactic