aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Cpo.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-15 19:48:24 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-15 19:48:24 +0000
commit3675bac6c38e0a26516e434be08bc100865b339b (patch)
tree87f8eb1905c7b508dea60b1e216f79120e9e772d /theories/Sets/Cpo.v
parentc881bc37b91a201f7555ee021ccb74adb360d131 (diff)
modif existentielle (exists | --> exists ,) + bug d'affichage des pt fixes
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5099 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Sets/Cpo.v')
-rwxr-xr-xtheories/Sets/Cpo.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/theories/Sets/Cpo.v b/theories/Sets/Cpo.v
index 0d77c0617..59f8fb2c8 100755
--- a/theories/Sets/Cpo.v
+++ b/theories/Sets/Cpo.v
@@ -67,7 +67,7 @@ Inductive Totally_ordered (B:Ensemble U) : Prop :=
Definition Compatible : Relation U :=
fun x y:U =>
In U C x ->
- In U C y -> exists z : _ | In U C z /\ Upper_Bound (Couple U x y) z.
+ In U C y -> exists z : _, In U C z /\ Upper_Bound (Couple U x y) z.
Inductive Directed (X:Ensemble U) : Prop :=
Definition_of_Directed :
@@ -75,21 +75,21 @@ Inductive Directed (X:Ensemble U) : Prop :=
Inhabited U X ->
(forall x1 x2:U,
Included U (Couple U x1 x2) X ->
- exists x3 : _ | In U X x3 /\ Upper_Bound (Couple U x1 x2) x3) ->
+ exists x3 : _, In U X x3 /\ Upper_Bound (Couple U x1 x2) x3) ->
Directed X.
Inductive Complete : Prop :=
Definition_of_Complete :
- ( exists bot : _ | Bottom bot) ->
- (forall X:Ensemble U, Directed X -> exists bsup : _ | Lub X bsup) ->
+ (exists bot : _, Bottom bot) ->
+ (forall X:Ensemble U, Directed X -> exists bsup : _, Lub X bsup) ->
Complete.
Inductive Conditionally_complete : Prop :=
Definition_of_Conditionally_complete :
(forall X:Ensemble U,
Included U X C ->
- ( exists maj : _ | Upper_Bound X maj) ->
- exists bsup : _ | Lub X bsup) -> Conditionally_complete.
+ (exists maj : _, Upper_Bound X maj) ->
+ exists bsup : _, Lub X bsup) -> Conditionally_complete.
End Bounds.
Hint Resolve Totally_ordered_definition Upper_Bound_definition
Lower_Bound_definition Lub_definition Glb_definition Bottom_definition