aboutsummaryrefslogtreecommitdiff
path: root/tactics/tactics.mli
diff options
context:
space:
mode:
authorEnrico Tassi2018-05-28 17:02:46 +0200
committerEnrico Tassi2018-05-28 17:02:46 +0200
commitb7d58843654963754593b0c9e44c0a5b7b7af16e (patch)
tree712844638f82eee8fd8cafd1a21da390d4e5b3df /tactics/tactics.mli
parent81535edc4b21015bd63d23e57ca9d707b4b71f6b (diff)
Tactics.introduction: remove dangerous option ~check
In locally nameless mode (proof mode) names in the context *must* be distinct otherwise the term representation makes no sense.
Diffstat (limited to 'tactics/tactics.mli')
-rw-r--r--tactics/tactics.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/tactics/tactics.mli b/tactics/tactics.mli
index ddf78b1d4e..b17330f133 100644
--- a/tactics/tactics.mli
+++ b/tactics/tactics.mli
@@ -34,7 +34,7 @@ val is_quantified_hypothesis : Id.t -> Proofview.Goal.t -> bool
(** {6 Primitive tactics. } *)
-val introduction : ?check:bool -> Id.t -> unit Proofview.tactic
+val introduction : Id.t -> unit Proofview.tactic
val convert_concl : ?check:bool -> types -> cast_kind -> unit Proofview.tactic
val convert_hyp : ?check:bool -> named_declaration -> unit Proofview.tactic
val convert_concl_no_check : types -> cast_kind -> unit Proofview.tactic