summaryrefslogtreecommitdiff
path: root/test-suite/success/PPFix.v8
blob: 1ecbae3ab3b10dac4ba8e6e65fe41e7322a727d8 (plain)
1
2
3
4
5
6
7
8

(* To test PP of fixpoints *)
Require Import Arith.
Check fix a(n: nat): n<5 -> nat :=
  match n return n<5 -> nat with
    | 0 => fun _ => 0
    | S n => fun h => S (a n (lt_S_n _ _ (lt_S _ _ h)))
  end.