summaryrefslogtreecommitdiff
path: root/theories/Init/Tauto.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Init/Tauto.v')
-rw-r--r--theories/Init/Tauto.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Init/Tauto.v b/theories/Init/Tauto.v
index 1e409607..87b7a9a3 100644
--- a/theories/Init/Tauto.v
+++ b/theories/Init/Tauto.v
@@ -2,7 +2,7 @@ Require Import Notations.
Require Import Datatypes.
Require Import Logic.
-Local Declare ML Module "tauto".
+Declare ML Module "tauto_plugin".
Local Ltac not_dep_intros :=
repeat match goal with
@@ -27,7 +27,7 @@ Local Ltac simplif flags :=
| id: ?X1 |- _ => is_disj flags X1; elim id; intro; clear id
| id0: (forall (_: ?X1), ?X2), id1: ?X1|- _ =>
(* generalize (id0 id1); intro; clear id0 does not work
- (see Marco Maggiesi's bug PR#301)
+ (see Marco Maggiesi's BZ#301)
so we instead use Assert and exact. *)
assert X2; [exact (id0 id1) | clear id0]
| id: forall (_ : ?X1), ?X2|- _ =>