aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-18 10:41:19 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-18 10:41:19 +0000
commit51ca3f46d2afd7f5e261e5147119526f2950a53b (patch)
tree1ca4bd8633caf6cb39baf50f26a1a296cedda0c4
parent8dbc29de13c5cb91bff356d7c729f0d30d6b46ad (diff)
Un nouveau lemme redondant ...
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4934 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--theories/ZArith/Zbinary.v27
1 files changed, 6 insertions, 21 deletions
diff --git a/theories/ZArith/Zbinary.v b/theories/ZArith/Zbinary.v
index e1b3019c4..142bfdef6 100644
--- a/theories/ZArith/Zbinary.v
+++ b/theories/ZArith/Zbinary.v
@@ -105,16 +105,10 @@ Definition Zmod2 := [z:Z] Cases z of
end
end.
-Lemma double_moins_un_add_un : (p:positive)
- (xI p)=(double_moins_un (add_un p)).
-Proof.
- Induction p; Simpl; Intros.
- Rewrite H; Auto.
-
- Trivial.
-
- Trivial.
-Save.
+V7only [
+Notation double_moins_un_add_un :=
+ [p](sym_eq ? ? ? (double_moins_un_add_un_xI p)).
+].
Lemma Zmod2_twice : (z:Z)
`z = (2*(Zmod2 z) + (bit_value (Zodd_bool z)))`.
@@ -126,7 +120,7 @@ Proof.
NewDestruct p; Simpl.
NewDestruct p as [p|p|]; Simpl.
- Rewrite (double_moins_un_add_un p); Trivial.
+ Rewrite <- (double_moins_un_add_un_xI p); Trivial.
Trivial.
@@ -216,16 +210,7 @@ Proof.
Auto with zarith.
Save.
-Lemma add_un_double_moins_un_xO : (p:positive)
- (add_un (double_moins_un p))=(xO p).
-Proof.
- NewInduction p as [|p H|]; Simpl.
- Trivial.
-
- Rewrite H; Trivial.
-
- Trivial.
-Save.
+V7only [Notation add_un_double_moins_un_xO := is_double_moins_un.].
Lemma two_compl_value_Sn : (n:nat) (bv : (Bvector (S n))) (b:bool)
(two_compl_value (S n) (Bcons b (S n) bv)) =