summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/5019.v
blob: 7c973f88b538417b82327aae5fee93cba4d18cad (plain)
1
2
3
4
5
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.
  Timeout 1 zify. (* used to loop forever; should take < 0.01 s *)
Admitted.