aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-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.