aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_5372.v
blob: e36b7a5d70b05583f86a8701b7c95e2ec611a0f1 (plain)
1
2
3
4
5
6
7
8
9
(* 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.
Reset odd.