aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4453.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-12-17 20:32:09 +0100
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-12-17 20:35:15 +0100
commit840cefca77a48ad68641539cd26d8d2e8c9dc031 (patch)
tree809abc3414582db2fa55b8675a6a78c50293deb3 /test-suite/bugs/closed/4453.v
parenta17891fdc314d0fe5246ab785268e2005a8c98b2 (diff)
(Partial) fix for bug #4453: raise an error instead of an anomaly.
Diffstat (limited to 'test-suite/bugs/closed/4453.v')
-rw-r--r--test-suite/bugs/closed/4453.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4453.v b/test-suite/bugs/closed/4453.v
new file mode 100644
index 000000000..009dd5e3c
--- /dev/null
+++ b/test-suite/bugs/closed/4453.v
@@ -0,0 +1,8 @@
+
+Section Foo.
+Variable A : Type.
+Lemma foo : A -> True. now intros _. Qed.
+Goal Type -> True.
+rename A into B.
+intros A.
+Fail apply foo.