aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Even.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-04 16:08:36 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-04 16:08:36 +0000
commitb4ace8546bf9de05a8cdd4267e17c32ee6806f18 (patch)
tree5c402a955151e959d0642f79adedb60c4f07fd0d /theories/Arith/Even.v
parentbb02036b476d3a3e7b3b79568257ef3d28ea6a11 (diff)
Commit malencontreux sur précédente version
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@655 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Even.v')
-rw-r--r--theories/Arith/Even.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Even.v b/theories/Arith/Even.v
index e2ae8eed2..a79a4d267 100644
--- a/theories/Arith/Even.v
+++ b/theories/Arith/Even.v
@@ -30,7 +30,7 @@ Auto with arith.
Intros n' H. Elim H; Auto with arith.
Save.
-Lemma not_even_and_odd2 : (n:nat) (even n) -> (odd n) -> False.
+Lemma not_even_and_odd : (n:nat) (even n) -> (odd n) -> False.
Proof.
Induction n.
Intros. Inversion H0.