aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets
diff options
context:
space:
mode:
authorGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2014-07-10 19:48:51 +0200
committerGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2014-07-10 19:48:51 +0200
commit39ef54919006741dba7c1860524b6800eb97a2c4 (patch)
tree33e0328265d9169f449379d84abaef711f8cbf43 /theories/MSets
parent6663052ccd613faf4282bd73121a44398bd3ba76 (diff)
MSetRBT: unfortunate typo in compare_height (fix #3413)
Diffstat (limited to 'theories/MSets')
-rw-r--r--theories/MSets/MSetRBT.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/MSets/MSetRBT.v b/theories/MSets/MSetRBT.v
index af67aa1ec..d7e56cdef 100644
--- a/theories/MSets/MSetRBT.v
+++ b/theories/MSets/MSetRBT.v
@@ -398,7 +398,7 @@ Definition skip_black t :=
Fixpoint compare_height (s1x s1 s2 s2x: tree) : comparison :=
match skip_red s1x, skip_red s1, skip_red s2, skip_red s2x with
| Node _ s1x' _ _, Node _ s1' _ _, Node _ s2' _ _, Node _ s2x' _ _ =>
- compare_height (skip_black s2x') s1' s2' (skip_black s2x')
+ compare_height (skip_black s1x') s1' s2' (skip_black s2x')
| _, Leaf, _, Node _ _ _ _ => Lt
| Node _ _ _ _, _, Leaf, _ => Gt
| Node _ s1x' _ _, Node _ s1' _ _, Node _ s2' _ _, Leaf =>