aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zmisc.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-13 11:03:04 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-13 11:03:04 +0000
commitfb7e6748d9b02fff8da1335dc3f4dedeb23a8f5d (patch)
treeb92404c5d75b2bae8fa574a8b61e3992acb30b03 /theories/ZArith/Zmisc.v
parent4ea5e9e7a3c08adabb0fb5113f849ffdd48ed172 (diff)
suite changements ZArith en vu de librairie FSet
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4149 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zmisc.v')
-rw-r--r--theories/ZArith/Zmisc.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/theories/ZArith/Zmisc.v b/theories/ZArith/Zmisc.v
index 9b5eb9260..a4cf3a9b3 100644
--- a/theories/ZArith/Zmisc.v
+++ b/theories/ZArith/Zmisc.v
@@ -298,25 +298,25 @@ Proof.
NewDestruct z; [ Idtac | NewDestruct p | NewDestruct p ]; Compute; Trivial.
Qed.
-Lemma Zeven_Sn : (z:Z)(Zeven z) -> (Zodd (Zs z)).
+Lemma Zeven_Sn : (z:Z)(Zodd z) -> (Zeven (Zs z)).
Proof.
NewDestruct z; Unfold Zs; [ Idtac | NewDestruct p | NewDestruct p ]; Simpl; Trivial.
Unfold double_moins_un; Case p; Simpl; Auto.
Qed.
-Lemma Zodd_Sn : (z:Z)(Zodd z) -> (Zeven (Zs z)).
+Lemma Zodd_Sn : (z:Z)(Zeven z) -> (Zodd (Zs z)).
Proof.
NewDestruct z; Unfold Zs; [ Idtac | NewDestruct p | NewDestruct p ]; Simpl; Trivial.
Unfold double_moins_un; Case p; Simpl; Auto.
Qed.
-Lemma Zeven_pred : (z:Z)(Zeven z) -> (Zodd (Zpred z)).
+Lemma Zeven_pred : (z:Z)(Zodd z) -> (Zeven (Zpred z)).
Proof.
NewDestruct z; Unfold Zpred; [ Idtac | NewDestruct p | NewDestruct p ]; Simpl; Trivial.
Unfold double_moins_un; Case p; Simpl; Auto.
Qed.
-Lemma Zodd_pred : (z:Z)(Zodd z) -> (Zeven (Zpred z)).
+Lemma Zodd_pred : (z:Z)(Zeven z) -> (Zodd (Zpred z)).
Proof.
NewDestruct z; Unfold Zpred; [ Idtac | NewDestruct p | NewDestruct p ]; Simpl; Trivial.
Unfold double_moins_un; Case p; Simpl; Auto.
@@ -384,7 +384,7 @@ Intro p; Split with (Zdiv2 (Zpred (NEG p))).
Pattern 1 (NEG p); Rewrite (Zs_pred (NEG p)).
Pattern 1 (Zpred (NEG p)); Rewrite (Zeven_div2 (Zpred (NEG p))).
Reflexivity.
-Apply Zodd_pred; Assumption.
+Apply Zeven_pred; Assumption.
Qed.
Lemma Zsplit2 : (x:Z) { p : Z*Z | let (x1,x2)=p in (`x=x1+x2` /\ (x1=x2 \/ `x2=x1+1`)) }.