aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/IntMap
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-21 10:19:59 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-21 10:19:59 +0000
commitf070d33f9822dac079e58a9920c9c9e0cade12f6 (patch)
tree9ddea6b144ca133d323d7ec2e6659a0bb3a650f8 /theories/IntMap
parentb7aa648034f73c390ba2b49c8d47c3c8277002ef (diff)
code mort dans tactinterp; plus de Debug On/Off dans Correctness
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2490 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/IntMap')
-rw-r--r--theories/IntMap/Adist.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/IntMap/Adist.v b/theories/IntMap/Adist.v
index 5c3296885..fbc2870f1 100644
--- a/theories/IntMap/Adist.v
+++ b/theories/IntMap/Adist.v
@@ -270,7 +270,7 @@ Qed.
d(a,a'')+d(a'',a')$,
but in fact $d(a,a')\leq max(d(a,a''),d(a'',a'))$.
This means that $min(pd(a,a''),pd(a'',a'))<=pd(a,a')$ (lemma [ad_pdist_ultra] below).
- This follows from the fact that $a \Ra |a| = 1/2^{\texttt{ad\_plength}}(a))$
+ This follows from the fact that $a ~Ra~|a| = 1/2^{\texttt{ad\_plength}}(a))$
is an ultrametric norm, i.e. that $|a-a'| \leq max (|a-a''|, |a''-a'|)$,
or equivalently that $|a+b|<=max(|a|,|b|)$, i.e. that
min $(\texttt{ad\_plength}(a), \texttt{ad\_plength}(b)) \leq