aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Natural
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-28 23:30:21 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-28 23:30:21 +0000
commit00353bc0b970605ae092af594417a51a0cdf903f (patch)
tree24187302e7bc000e784af8e745d6da9d525f7e52 /theories/Numbers/Natural
parenta0b31c88aa2bcd50524cbc48d16eb78c62da3445 (diff)
Deletion of useless Zlog_def
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14246 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Numbers/Natural')
-rw-r--r--theories/Numbers/Natural/BigN/NMake.v2
-rw-r--r--theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v6
2 files changed, 4 insertions, 4 deletions
diff --git a/theories/Numbers/Natural/BigN/NMake.v b/theories/Numbers/Natural/BigN/NMake.v
index 66b39aca9..64b8ec844 100644
--- a/theories/Numbers/Natural/BigN/NMake.v
+++ b/theories/Numbers/Natural/BigN/NMake.v
@@ -1244,7 +1244,7 @@ Module Make (W0:CyclicType) <: NType.
apply ZnZ.spec_head0; auto with zarith.
Qed.
- Lemma spec_log2 : forall x, [log2 x] = Zlog2 [x].
+ Lemma spec_log2 : forall x, [log2 x] = Z.log2 [x].
Proof.
intros. destruct (Z_lt_ge_dec 0 [x]).
symmetry. apply Z.log2_unique. apply spec_pos.
diff --git a/theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v b/theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v
index 9bed794f2..225c0853e 100644
--- a/theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v
+++ b/theories/Numbers/Natural/SpecViaZ/NSigNAxioms.v
@@ -277,13 +277,13 @@ Qed.
Lemma log2_spec : forall n, 0<n ->
2^(log2 n) <= n /\ n < 2^(succ (log2 n)).
Proof.
- intros n. zify. change (Zlog2 [n]+1)%Z with (Zsucc (Zlog2 [n])).
- apply Zlog2_spec.
+ intros n. zify. change (Z.log2 [n]+1)%Z with (Z.succ (Z.log2 [n])).
+ apply Z.log2_spec.
Qed.
Lemma log2_nonpos : forall n, n<=0 -> log2 n == 0.
Proof.
- intros n. zify. apply Zlog2_nonpos.
+ intros n. zify. apply Z.log2_nonpos.
Qed.
(** Even / Odd *)