aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rsqrt_def.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-24 10:27:08 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-24 10:27:08 +0000
commit38734c5e122e9a38cf5b8afc586f47abced11361 (patch)
tree2227afa958bf809d9152b526e29f183b552e5e61 /theories/Reals/Rsqrt_def.v
parentc69ae2a1f05db124c19b7f326ca23e980f643198 (diff)
changement de pose en set (pose n'etait pas utilise avec la semantique
documentee). Reste a retablir la semantique de pose. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5141 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rsqrt_def.v')
-rw-r--r--theories/Reals/Rsqrt_def.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Reals/Rsqrt_def.v b/theories/Reals/Rsqrt_def.v
index b123f1bb7..932e40773 100644
--- a/theories/Reals/Rsqrt_def.v
+++ b/theories/Reals/Rsqrt_def.v
@@ -267,7 +267,7 @@ unfold cv_infty in |- *.
intro.
case (total_order_T 0 M); intro.
elim s; intro.
-pose (N := up M).
+set (N := up M).
cut (0 <= N)%Z.
intro.
elim (IZN N H0); intros N0 H1.
@@ -475,8 +475,8 @@ apply dicho_up_decreasing; assumption.
assumption.
right; reflexivity.
2: left; assumption.
-pose (Vn := fun n:nat => dicho_lb x y (fun z:R => cond_positivity (f z)) n).
-pose (Wn := fun n:nat => dicho_up x y (fun z:R => cond_positivity (f z)) n).
+set (Vn := fun n:nat => dicho_lb x y (fun z:R => cond_positivity (f z)) n).
+set (Wn := fun n:nat => dicho_up x y (fun z:R => cond_positivity (f z)) n).
cut ((forall n:nat, f (Vn n) <= 0) -> f x0 <= 0).
cut ((forall n:nat, 0 <= f (Wn n)) -> 0 <= f x0).
intros.
@@ -652,7 +652,7 @@ Qed.
Lemma Rsqrt_exists :
forall y:R, 0 <= y -> sigT (fun z:R => 0 <= z /\ y = Rsqr z).
intros.
-pose (f := fun x:R => Rsqr x - y).
+set (f := fun x:R => Rsqr x - y).
cut (f 0 <= 0).
intro.
cut (continuity f).