aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Ensembles.v
diff options
context:
space:
mode:
authorGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-20 16:00:43 +0000
committerGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-20 16:00:43 +0000
commitd857c99c6c985eb36ce8a4b2667dc0b5ccca115c (patch)
tree2ea53c80dd3319b24c38b15cb5be5a582c9b302a /theories/Sets/Ensembles.v
parent4837b599b4f158decc91f615a25e3a636c6ced5d (diff)
Library doc adjustments (until page 140)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1655 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Sets/Ensembles.v')
-rwxr-xr-xtheories/Sets/Ensembles.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Sets/Ensembles.v b/theories/Sets/Ensembles.v
index 0ddad8578..40389087e 100755
--- a/theories/Sets/Ensembles.v
+++ b/theories/Sets/Ensembles.v
@@ -43,10 +43,10 @@ Inductive Full_set : Ensemble :=
Full_intro: (x: U) (In Full_set x).
(* NB The following definition builds-in equality of elements in U as
- Leibniz equality.
+ Leibniz equality. \\
This may have to be changed if we replace U by a Setoid on U with its own
- equality eqs, with
- [In_singleton: (y: U)(eqs x y) -> (In (Singleton x) y)]. *)
+ equality eqs, with
+ [In_singleton: (y: U)(eqs x y) -> (In (Singleton x) y)]. *)
Inductive Singleton [x:U] : Ensemble :=
In_singleton: (In (Singleton x) x).