aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_4103.v
blob: 690511a86c780d4fbde890d3561cc1ff62bd89b4 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
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.
Abort.