aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/tacmach.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-13 20:38:41 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:28:50 +0100
commit485bbfbed4ae4a28119c4e42c5e40fd77abf4f8a (patch)
treeab397f012c1d9ea53e041759309b08cccfeac817 /proofs/tacmach.mli
parent771be16883c8c47828f278ce49545716918764c4 (diff)
Tactics API using EConstr.
Diffstat (limited to 'proofs/tacmach.mli')
-rw-r--r--proofs/tacmach.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli
index 07d02212c..cfbfe12b1 100644
--- a/proofs/tacmach.mli
+++ b/proofs/tacmach.mli
@@ -67,8 +67,8 @@ val pf_whd_all : goal sigma -> EConstr.constr -> constr
val pf_hnf_constr : goal sigma -> EConstr.constr -> constr
val pf_nf : goal sigma -> EConstr.constr -> constr
val pf_nf_betaiota : goal sigma -> EConstr.constr -> constr
-val pf_reduce_to_quantified_ind : goal sigma -> EConstr.types -> pinductive * types
-val pf_reduce_to_atomic_ind : goal sigma -> EConstr.types -> pinductive * types
+val pf_reduce_to_quantified_ind : goal sigma -> EConstr.types -> pinductive * EConstr.types
+val pf_reduce_to_atomic_ind : goal sigma -> EConstr.types -> pinductive * EConstr.types
val pf_compute : goal sigma -> EConstr.constr -> constr
val pf_unfoldn : (occurrences * evaluable_global_reference) list
-> goal sigma -> EConstr.constr -> constr
@@ -121,7 +121,7 @@ module New : sig
val pf_last_hyp : ([ `NF ], 'r) Proofview.Goal.t -> Context.Named.Declaration.t
val pf_nf_concl : ([ `LZ ], 'r) Proofview.Goal.t -> types
- val pf_reduce_to_quantified_ind : ('a, 'r) Proofview.Goal.t -> EConstr.types -> pinductive * types
+ val pf_reduce_to_quantified_ind : ('a, 'r) Proofview.Goal.t -> EConstr.types -> pinductive * EConstr.types
val pf_hnf_constr : ('a, 'r) Proofview.Goal.t -> EConstr.constr -> types
val pf_hnf_type_of : ('a, 'r) Proofview.Goal.t -> EConstr.constr -> types