summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/5372.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/5372.v')
-rw-r--r--test-suite/bugs/closed/5372.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5372.v b/test-suite/bugs/closed/5372.v
new file mode 100644
index 00000000..e60244cd
--- /dev/null
+++ b/test-suite/bugs/closed/5372.v
@@ -0,0 +1,8 @@
+(* coq bug 5372: https://coq.inria.fr/bugs/show_bug.cgi?id=5372 *)
+Require Import FunInd.
+Function odd (n:nat) :=
+ match n with
+ | 0 => false
+ | S n => true
+ end
+with even (n:nat) := false.