summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_8794.v
blob: 5ff0b30260f0d52b7467195a73e778aec2dd65e0 (plain)
1
2
3
4
5
6
7
8
9
10
11
(* This used to raise an anomaly in 8.8 *)

Inductive T := Tau (t : T).

Notation idT t := (match t with Tau t => Tau t end).

Lemma match_itree : forall (t : T), t = idT t.
Proof. destruct t; auto. Qed.

Lemma what (k : unit -> T) : k tt = k tt.
Proof. rewrite match_itree. Abort.