aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Raxioms.v
diff options
context:
space:
mode:
authorGravatar mayero <mayero@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-07-04 17:06:33 +0000
committerGravatar mayero <mayero@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-07-04 17:06:33 +0000
commitfae615defa0fca136dc7d1f6208d38333327d133 (patch)
treeffac7d7f8352c776f6865378663139dfa0375ee6 /theories/Reals/Raxioms.v
parent533d30df924cbdd9e0ef01e4d9fb8a48e201e6e8 (diff)
correction
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@554 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Raxioms.v')
-rw-r--r--theories/Reals/Raxioms.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Reals/Raxioms.v b/theories/Reals/Raxioms.v
index 7b7ec3103..2297e7d7b 100644
--- a/theories/Reals/Raxioms.v
+++ b/theories/Reals/Raxioms.v
@@ -158,7 +158,7 @@ Definition bound:=[E:R->Prop](ExT [m:R](is_upper_bound E m)).
(**********)
Definition is_lub:=[E:R->Prop][m:R]
- (is_upper_bound E m)/\(b:R)(is_upper_bound E b)->(Rlt m b).
+ (is_upper_bound E m)/\(b:R)(is_upper_bound E b)->(Rle m b).
(**********)
Axiom complet:(E:R->Prop)(bound E)->