aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorHugo Herbelin2020-11-28 15:10:21 +0100
committerHugo Herbelin2021-01-18 15:25:26 +0100
commite56c65cf68c4055b4e1272b5a2afbf5803d93a42 (patch)
tree8ad85144180f8bd359afe078f846b66b8472e7c3 /test-suite
parentf44e65e0d209fdada20998d661ad10a5e82a0d92 (diff)
Fixes #13413: freshness issue with "%" introduction pattern.
We build earlier the final expected name at the end of a sequence of "%" introduction patterns.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/bug_13413.v20
-rw-r--r--test-suite/success/forward.v4
2 files changed, 24 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/bug_13413.v b/test-suite/bugs/closed/bug_13413.v
new file mode 100644
index 0000000000..b4414a6a1d
--- /dev/null
+++ b/test-suite/bugs/closed/bug_13413.v
@@ -0,0 +1,20 @@
+Goal forall (A B : Prop) (H : A -> B), A -> A -> B.
+intros A B H ?%H H0.
+exact H1.
+Qed.
+
+Goal forall (A B : Prop) (H : A -> B), A -> A -> B.
+intros A B H ?H%H H0.
+exact H1.
+Qed.
+
+Goal forall (A B : Prop) (H : A -> B), A -> A -> B.
+intros A B H J%H H0.
+exact J.
+Qed.
+
+Set Mangle Names.
+Goal forall (A B : Prop) (H : A -> B), A -> A -> B.
+intros A B H ?%H _0.
+assumption.
+Qed.
diff --git a/test-suite/success/forward.v b/test-suite/success/forward.v
index 4e36dec15b..62c788e910 100644
--- a/test-suite/success/forward.v
+++ b/test-suite/success/forward.v
@@ -27,3 +27,7 @@ Fail match goal with |- (?f ?a) => idtac end. (* should be beta-iota reduced *)
2:match goal with _: (?f ?a) |- _ => idtac end. (* should not be beta-iota reduced *)
Abort.
+Goal nat.
+assert nat as J%S by exact 0.
+exact J.
+Qed.