aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-03-05 10:58:08 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-03-05 10:58:08 +0000
commit4dbf6842e0b2b43c5f8c15817942dfecaab5cd2e (patch)
treef81b47df039aed8471726bfb635b6a675602ecab /theories/ZArith
parent21cd39996cabdf280f4cc99557c54f6c7c73bbc8 (diff)
petits changements afin de profiter du nouveau Rewrite/in
(l'unification marche mieux) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2512 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/Zcomplements.v2
-rw-r--r--theories/ZArith/Zlogarithm.v12
-rw-r--r--theories/ZArith/auxiliary.v2
3 files changed, 8 insertions, 8 deletions
diff --git a/theories/ZArith/Zcomplements.v b/theories/ZArith/Zcomplements.v
index ce9691450..ef479c831 100644
--- a/theories/ZArith/Zcomplements.v
+++ b/theories/ZArith/Zcomplements.v
@@ -51,7 +51,7 @@ Intros.
Generalize (Zeq_Zminus H0).
Intro.
Apply Zminus_Zeq.
-Rewrite <- (Zmult_Zminus_distr_r x y z) in H1.
+Rewrite <- Zmult_Zminus_distr_r in H1.
Elim (Zmult_zero H1).
Omega.
Trivial.
diff --git a/theories/ZArith/Zlogarithm.v b/theories/ZArith/Zlogarithm.v
index e219e0eae..c33b1f157 100644
--- a/theories/ZArith/Zlogarithm.v
+++ b/theories/ZArith/Zlogarithm.v
@@ -54,15 +54,15 @@ Theorem log_inf_correct : (x:positive) ` 0 <= (log_inf x)` /\
Induction x; Intros; Simpl;
[ Elim H; Intros Hp HR; Clear H; Split;
[ Auto with zarith
- | Rewrite (two_p_S (Zs (log_inf p)) (Zle_le_S `0` (log_inf p) Hp));
- Rewrite (two_p_S (log_inf p) Hp);
- Rewrite (two_p_S (log_inf p) Hp) in HR;
+ | Conditional (Apply Zle_le_S; Trivial) Rewrite two_p_S with x:=(Zs (log_inf p));
+ Conditional Trivial Rewrite two_p_S;
+ Conditional Trivial Rewrite two_p_S in HR;
Rewrite (POS_xI p); Omega ]
| Elim H; Intros Hp HR; Clear H; Split;
[ Auto with zarith
- | Rewrite (two_p_S (Zs (log_inf p)) (Zle_le_S `0` (log_inf p) Hp));
- Rewrite (two_p_S (log_inf p) Hp);
- Rewrite (two_p_S (log_inf p) Hp) in HR;
+ | Conditional (Apply Zle_le_S; Trivial) Rewrite two_p_S with x:=(Zs (log_inf p));
+ Conditional Trivial Rewrite two_p_S;
+ Conditional Trivial Rewrite two_p_S in HR;
Rewrite (POS_xO p); Omega ]
| Unfold two_power_pos; Unfold shift_pos; Simpl; Omega
].
diff --git a/theories/ZArith/auxiliary.v b/theories/ZArith/auxiliary.v
index e6edf81a5..b6505d6bb 100644
--- a/theories/ZArith/auxiliary.v
+++ b/theories/ZArith/auxiliary.v
@@ -713,7 +713,7 @@ Theorem OMEGA20:
(x,y,z:Z)(Zne x ZERO) -> (y=ZERO) -> (Zne (Zplus x (Zmult y z)) ZERO).
Unfold Zne not; Intros x y z H1 H2 H3; Apply H1; Rewrite H2 in H3;
-Simpl in H3; Rewrite (Zero_right x) in H3; Trivial with arith.
+Simpl in H3; Rewrite Zero_right in H3; Trivial with arith.
Save.
Definition fast_Zplus_sym :=