summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4366.v
blob: 403c2d202687f886c69efa9877284f74b655b4a2 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
Fixpoint stupid (n : nat) : unit :=
match n with
| 0 => tt
| S n =>
  let () := stupid n in
  let () := stupid n in
  tt
end.

Goal True.
Proof.
pose (v := stupid 24).
Timeout 4 vm_compute in v.
exact I.
Qed.