aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-05-30 12:11:28 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-06-01 03:55:05 -0400
commit4af77d01c434ff11f0899d504628f4ff91c49142 (patch)
tree28994111a58e9f823fdef25bb7f9d8089a72c60e
parente7e0946401aa931ddca90d616a7968d548ab060f (diff)
Add opened bug 5019
-rw-r--r--test-suite/bugs/opened/5019.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/test-suite/bugs/opened/5019.v b/test-suite/bugs/opened/5019.v
new file mode 100644
index 000000000..09622097c
--- /dev/null
+++ b/test-suite/bugs/opened/5019.v
@@ -0,0 +1,4 @@
+Require Import Coq.ZArith.ZArith.
+Goal forall (T0 : Z -> Type) (k : nat) d (P : T0 (Z.of_nat (S k)) -> Prop), P d.
+ clear; intros.
+ Fail Timeout 1 zify.