summaryrefslogtreecommitdiff
path: root/test-suite/success/PPFix.v8
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/PPFix.v8')
-rw-r--r--test-suite/success/PPFix.v88
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/success/PPFix.v8 b/test-suite/success/PPFix.v8
new file mode 100644
index 00000000..1ecbae3a
--- /dev/null
+++ b/test-suite/success/PPFix.v8
@@ -0,0 +1,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.