aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rtopology.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-15 11:58:37 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-15 11:58:37 +0000
commitd3c8ce6c19ffff8d53959f3f4bf41fef85172514 (patch)
tree7d9e33ad93c1080f49880af44fa906004a4873f4 /theories/Reals/Rtopology.v
parentf410308f7b300135d97b16ae3fbf776d8012bc61 (diff)
Pas d'associativite pour =_D
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3436 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rtopology.v')
-rw-r--r--theories/Reals/Rtopology.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Reals/Rtopology.v b/theories/Reals/Rtopology.v
index 98c2039eb..9909df51b 100644
--- a/theories/Reals/Rtopology.v
+++ b/theories/Reals/Rtopology.v
@@ -93,7 +93,7 @@ Qed.
Definition eq_Dom [D1,D2:R->Prop] : Prop := (inclus D1 D2)/\(inclus D2 D1).
-Infix 5 "=_D" eq_Dom.
+Infix "=_D" eq_Dom (at level 5, no associativity).
Lemma ouvert_P1 : (D:R->Prop) (ouvert D) <-> D =_D (interieur D).
Intro; Split.