aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/clenvtac.mli
diff options
context:
space:
mode:
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