summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/5315.v
blob: d8824bff875a5dab20cbb55fb99f2b374ea50e6a (plain)
1
2
3
4
5
6
7
8
9
10
Require Import Recdef.

Function dumb_works (a:nat) {struct a} :=
  match (fun x => x) a with O => O | S n' => dumb_works n' end.

Function dumb_nope (a:nat) {struct a} :=
  match (id (fun x => x)) a with O => O | S n' => dumb_nope n' end.

(* This check is just present to ensure Function worked well *)
Check R_dumb_nope_complete.