aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/clenvtac.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-10-12 15:36:17 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-10-13 19:12:34 +0200
commite9c25b3368a73737553821d2e954383c57698a86 (patch)
tree30374a292fcbb373862cae80d6288be4783aa77a /proofs/clenvtac.mli
parent267d7a63e9c24573226d0890bedb783f10dcb235 (diff)
Add support for deactivating type class inference from induction/destruct.
Diffstat (limited to 'proofs/clenvtac.mli')
-rw-r--r--proofs/clenvtac.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/proofs/clenvtac.mli b/proofs/clenvtac.mli
index bede509e7..6a7e12a35 100644
--- a/proofs/clenvtac.mli
+++ b/proofs/clenvtac.mli
@@ -15,7 +15,7 @@ open Unification
(** Tactics *)
val unify : ?flags:unify_flags -> constr -> unit Proofview.tactic
val clenv_refine : evars_flag -> ?with_classes:bool -> clausenv -> unit Proofview.tactic
-val res_pf : ?with_evars:evars_flag -> ?flags:unify_flags -> clausenv -> unit Proofview.tactic
+val res_pf : ?with_evars:evars_flag -> ?with_classes:bool -> ?flags:unify_flags -> clausenv -> unit Proofview.tactic
val clenv_pose_dependent_evars : evars_flag -> clausenv -> clausenv
val clenv_value_cast_meta : clausenv -> constr