aboutsummaryrefslogtreecommitdiffhomepage
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.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5372.v b/test-suite/bugs/closed/5372.v
index 2dc78d4c7..e60244cd1 100644
--- a/test-suite/bugs/closed/5372.v
+++ b/test-suite/bugs/closed/5372.v
@@ -1,4 +1,5 @@
(* 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