aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Integer
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-28 23:30:10 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-28 23:30:10 +0000
commita0b31c88aa2bcd50524cbc48d16eb78c62da3445 (patch)
treeebf4533e46fb630e520a745f2b3df41d489a33ec /theories/Numbers/Integer
parent2941378aee6586bcff9f8a117f11e5c5c2327607 (diff)
Deletion of useless Zsqrt_def
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14245 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Numbers/Integer')
-rw-r--r--theories/Numbers/Integer/BigZ/ZMake.v4
-rw-r--r--theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v4
2 files changed, 4 insertions, 4 deletions
diff --git a/theories/Numbers/Integer/BigZ/ZMake.v b/theories/Numbers/Integer/BigZ/ZMake.v
index 173a8f177..0bcf22e32 100644
--- a/theories/Numbers/Integer/BigZ/ZMake.v
+++ b/theories/Numbers/Integer/BigZ/ZMake.v
@@ -383,13 +383,13 @@ Module Make (N:NType) <: ZType.
| Neg nx => Neg N.zero
end.
- Theorem spec_sqrt: forall x, to_Z (sqrt x) = Zsqrt (to_Z x).
+ Theorem spec_sqrt: forall x, to_Z (sqrt x) = Z.sqrt (to_Z x).
Proof.
destruct x as [p|p]; simpl.
apply N.spec_sqrt.
rewrite N.spec_0.
destruct (Z_le_lt_eq_dec _ _ (N.spec_pos p)) as [LT|EQ].
- rewrite Zsqrt_neg; auto with zarith.
+ rewrite Z.sqrt_neg; auto with zarith.
now rewrite <- EQ.
Qed.
diff --git a/theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v b/theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v
index 390b52ebe..dd83b65da 100644
--- a/theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v
+++ b/theories/Numbers/Integer/SpecViaZ/ZSigZAxioms.v
@@ -311,12 +311,12 @@ Qed.
Lemma sqrt_spec : forall n, 0<=n ->
(sqrt n)*(sqrt n) <= n /\ n < (succ (sqrt n))*(succ (sqrt n)).
Proof.
- intros n. zify. apply Zsqrt_spec.
+ intros n. zify. apply Z.sqrt_spec.
Qed.
Lemma sqrt_neg : forall n, n<0 -> sqrt n == 0.
Proof.
- intros n. zify. apply Zsqrt_neg.
+ intros n. zify. apply Z.sqrt_neg.
Qed.
(** Log2 *)