aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Uniset.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-07-01 10:20:57 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-07-01 10:20:57 +0000
commita90e3402f4033583d84000ea2baf63959067e171 (patch)
treeb572f748c4d313367f11838462ce3d83f9fa8fda /theories/Sets/Uniset.v
parent445171395557a2447e70d90bb793277639a9a01e (diff)
Séparation des caractères spéciaux par un blanc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@544 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Sets/Uniset.v')
-rw-r--r--theories/Sets/Uniset.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Sets/Uniset.v b/theories/Sets/Uniset.v
index f89cda344..5d9162fdb 100644
--- a/theories/Sets/Uniset.v
+++ b/theories/Sets/Uniset.v
@@ -28,7 +28,7 @@ Definition Fullset := (Charac [a:A]true).
Definition Singleton := [a:A](Charac [a':A]
Case (eqA_dec a a') of
[h:(eqA a a')] true
- [h:~(eqA a a')] false end).
+ [h: ~(eqA a a')] false end).
Definition In : uniset -> A -> Prop :=
[s:uniset][a:A](charac s a)=true.