aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/tacmach.mli
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-10-24 17:38:59 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-10-24 17:42:14 +0200
commit884b6cc6c12bd557085cdaa4972d593684c9cc1a (patch)
treef3ba143e41d8d053d4369ffcba7ae294b001beb5 /proofs/tacmach.mli
parent1556c6b8f77d16814ff1c53fb14fc9b06574ec4b (diff)
Change reduction_of_red_expr to return an e_reduction_function returning
an updated evar_map, as pattern is working up to universe equalities that must be kept. Straightforward adaptation of the code depending on this.
Diffstat (limited to 'proofs/tacmach.mli')
-rw-r--r--proofs/tacmach.mli5
1 files changed, 4 insertions, 1 deletions
diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli
index b754f6f40..3ee970c1f 100644
--- a/proofs/tacmach.mli
+++ b/proofs/tacmach.mli
@@ -50,7 +50,7 @@ val pf_get_hyp_typ : goal sigma -> Id.t -> types
val pf_get_new_id : Id.t -> goal sigma -> Id.t
val pf_get_new_ids : Id.t list -> goal sigma -> Id.t list
-val pf_reduction_of_red_expr : goal sigma -> red_expr -> constr -> constr
+val pf_reduction_of_red_expr : goal sigma -> red_expr -> constr -> evar_map * constr
val pf_apply : (env -> evar_map -> 'a) -> goal sigma -> 'a
@@ -59,6 +59,9 @@ val pf_eapply : (env -> evar_map -> 'a -> evar_map * 'b) ->
val pf_reduce :
(env -> evar_map -> constr -> constr) ->
goal sigma -> constr -> constr
+val pf_e_reduce :
+ (env -> evar_map -> constr -> evar_map * constr) ->
+ goal sigma -> constr -> evar_map * constr
val pf_whd_betadeltaiota : goal sigma -> constr -> constr
val pf_hnf_constr : goal sigma -> constr -> constr