summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/5618.v
blob: 47e0e92d2ac2e70f2ff830f203da5dcc4eb990b9 (plain)
1
2
3
4
5
6
7
8
9
Require Import FunInd.

Function test {T} (v : T) (x : nat) : nat :=
  match x with
  | 0 => 0
  | S x' => test v x'
  end.

Check R_test_complete.