aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Znat.v
diff options
context:
space:
mode:
authorGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-03-28 18:15:23 +0000
committerGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-03-28 18:15:23 +0000
commit5bb2935198434eceea41e1b966b56a175def396d (patch)
tree1266f4bde8439fdcd33d6c1125a4e88622c2d8b8 /theories/ZArith/Znat.v
parentbca8775b49fd63c119cf2dd4f54c87676a93ed61 (diff)
Correction du bug 1816 (ajout d'un lemme dans Znat) et suppression
d'un test non significatif git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10726 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Znat.v')
-rw-r--r--theories/ZArith/Znat.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/theories/ZArith/Znat.v b/theories/ZArith/Znat.v
index ec37c1412..5d3b20160 100644
--- a/theories/ZArith/Znat.v
+++ b/theories/ZArith/Znat.v
@@ -29,6 +29,11 @@ Definition neq (x y:nat) := x <> y.
(** Injection and successor *)
+Theorem inj_0 : Z_of_nat 0 = 0%Z.
+Proof.
+ reflexivity.
+Qed.
+
Theorem inj_S : forall n:nat, Z_of_nat (S n) = Zsucc (Z_of_nat n).
Proof.
intro y; induction y as [| n H];