aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/tacred.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-06 21:59:18 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:26:38 +0100
commitb77579ac873975a15978c5a4ecf312d577746d26 (patch)
tree772e41667e74c38582ff6f4645c73e7d7556f935 /pretyping/tacred.mli
parent258c8502eafd3e078a5c7478a452432b5c046f71 (diff)
Tacred API using EConstr.
Diffstat (limited to 'pretyping/tacred.mli')
-rw-r--r--pretyping/tacred.mli10
1 files changed, 5 insertions, 5 deletions
diff --git a/pretyping/tacred.mli b/pretyping/tacred.mli
index f8dfe1adf..d32fcf491 100644
--- a/pretyping/tacred.mli
+++ b/pretyping/tacred.mli
@@ -17,7 +17,7 @@ open Locus
open Univ
type reduction_tactic_error =
- InvalidAbstraction of env * evar_map * constr * (env * Type_errors.type_error)
+ InvalidAbstraction of env * evar_map * EConstr.constr * (env * Type_errors.type_error)
exception ReductionTacticError of reduction_tactic_error
@@ -58,10 +58,10 @@ val unfoldn :
(occurrences * evaluable_global_reference) list -> reduction_function
(** Fold *)
-val fold_commands : constr list -> reduction_function
+val fold_commands : EConstr.constr list -> reduction_function
(** Pattern *)
-val pattern_occs : (occurrences * constr) list -> e_reduction_function
+val pattern_occs : (occurrences * EConstr.constr) list -> e_reduction_function
(** Rem: Lazy strategies are defined in Reduction *)
@@ -85,10 +85,10 @@ val reduce_to_quantified_ind : env -> evar_map -> types -> pinductive * types
(** [reduce_to_quantified_ref env sigma ref t] try to put [t] in the form
[t'=(x1:A1)..(xn:An)(ref args)] and fails with user error if not possible *)
val reduce_to_quantified_ref :
- env -> evar_map -> global_reference -> types -> types
+ env -> evar_map -> global_reference -> EConstr.types -> types
val reduce_to_atomic_ref :
- env -> evar_map -> global_reference -> types -> types
+ env -> evar_map -> global_reference -> EConstr.types -> types
val find_hnf_rectype :
env -> evar_map -> types -> pinductive * constr list