aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Raxioms.v
diff options
context:
space:
mode:
authorGravatar mayero <mayero@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-07-03 18:27:15 +0000
committerGravatar mayero <mayero@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-07-03 18:27:15 +0000
commit533d30df924cbdd9e0ef01e4d9fb8a48e201e6e8 (patch)
treefeeabb1b13161c34a88b41a6a4f59a62f9961f8b /theories/Reals/Raxioms.v
parent9013e6d80b26b177fbcd10a706f271ca4b576585 (diff)
ajouts
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@553 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Raxioms.v')
-rw-r--r--theories/Reals/Raxioms.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/theories/Reals/Raxioms.v b/theories/Reals/Raxioms.v
index 579672866..7b7ec3103 100644
--- a/theories/Reals/Raxioms.v
+++ b/theories/Reals/Raxioms.v
@@ -161,4 +161,7 @@ Definition is_lub:=[E:R->Prop][m:R]
(is_upper_bound E m)/\(b:R)(is_upper_bound E b)->(Rlt m b).
(**********)
-Axiom complet:(E:R->Prop)((bound E)->(ExT [m:R](is_lub E m))).
+Axiom complet:(E:R->Prop)(bound E)->
+ (ExT [x:R] (E x))->
+ (ExT [m:R](is_lub E m)).
+