summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4103.v
blob: 92cc0279ac62023f8c5cefbdaab6f990d80a98ec (plain)
1
2
3
4
5
6
7
8
9
10
11
12
Set Primitive Projections.

CoInductive stream A := { hd : A; tl : stream A }.

CoFixpoint ticks (n : nat) : stream unit := {| hd := tt; tl := ticks n |}.

Lemma expand : exists n : nat, (ticks n) = (ticks n).(tl _).
Proof.
  eexists.
  (* Set Debug Tactic Unification. *)
  (* Set Debug RAKAM. *)
  reflexivity.