aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/5019.v
blob: 09622097c5a6ed2154dabf4d9b65792f3134688d (plain)
1
2
3
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.