aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/MVT.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/MVT.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/MVT.v')
-rw-r--r--theories/Reals/MVT.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Reals/MVT.v b/theories/Reals/MVT.v
index d7531e49f..a6c2d115c 100644
--- a/theories/Reals/MVT.v
+++ b/theories/Reals/MVT.v
@@ -25,7 +25,7 @@ Theorem MVT :
(g b - g a) * derive_pt f c (pr1 c P) =
(f b - f a) * derive_pt g c (pr2 c P)).
intros; assert (H2 := Rlt_le _ _ H).
-pose (h := fun y:R => (g b - g a) * f y - (f b - f a) * g y).
+set (h := fun y:R => (g b - g a) * f y - (f b - f a) * g y).
cut (forall c:R, a < c < b -> derivable_pt h c).
intro; cut (forall c:R, a <= c <= b -> continuity_pt h c).
intro; assert (H4 := continuity_ab_maj h a b H2 H3).
@@ -33,7 +33,7 @@ assert (H5 := continuity_ab_min h a b H2 H3).
elim H4; intros Mx H6.
elim H5; intros mx H7.
cut (h a = h b).
-intro; pose (M := h Mx); pose (m := h mx).
+intro; set (M := h Mx); set (m := h mx).
cut
(forall (c:R) (P:a < c < b),
derive_pt h c (X c P) =