aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/5315.v
diff options
context:
space:
mode:
authorGravatar Julien Forest <forest@ensiie.fr>2017-06-16 16:45:47 +0200
committerGravatar Julien Forest <forest@ensiie.fr>2017-07-29 10:28:07 +0200
commit3810a76a85a83242a739bacdfd2c8485a8e4c9da (patch)
treef9c3b50a86f44c06e16aa74907e4050c5a609ecf /test-suite/bugs/closed/5315.v
parent17f37f42792b3150fcebb6236b9896845957b89d (diff)
closing bug 5315
Diffstat (limited to 'test-suite/bugs/closed/5315.v')
-rw-r--r--test-suite/bugs/closed/5315.v10
1 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5315.v b/test-suite/bugs/closed/5315.v
new file mode 100644
index 000000000..f1f1b8c05
--- /dev/null
+++ b/test-suite/bugs/closed/5315.v
@@ -0,0 +1,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. \ No newline at end of file