summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/5372.v
blob: e60244cd1d28139859ca209b563489619cb2e3d3 (plain)
1
2
3
4
5
6
7
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.