summaryrefslogtreecommitdiff
path: root/theories/MSets/MSetAVL.v
diff options
context:
space:
mode:
authorGravatar Stephane Glondu <steph@glondu.net>2011-04-19 16:47:51 +0200
committerGravatar Stephane Glondu <steph@glondu.net>2011-04-19 16:47:51 +0200
commitaa33547c764a229e22d323ca213d46ea221b903e (patch)
tree3894cb190f34bc1d2deee4322a674db641562ee0 /theories/MSets/MSetAVL.v
parent50dc9067e98ca001ad2e875011abab5da6fdb621 (diff)
parent9d27ae09786866b6e3d7b79d1fa7667e5e2aa309 (diff)
Remove non-DFSG contentsupstream/8.3.pl2+dfsg
Diffstat (limited to 'theories/MSets/MSetAVL.v')
-rw-r--r--theories/MSets/MSetAVL.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/MSets/MSetAVL.v b/theories/MSets/MSetAVL.v
index c41df7c2..96580749 100644
--- a/theories/MSets/MSetAVL.v
+++ b/theories/MSets/MSetAVL.v
@@ -82,9 +82,9 @@ Definition empty := Leaf.
Definition is_empty s :=
match s with Leaf => true | _ => false end.
-(** ** Appartness *)
+(** ** Membership *)
-(** The [mem] function is deciding appartness. It exploits the
+(** The [mem] function is deciding membership. It exploits the
binary search tree invariant to achieve logarithmic complexity. *)
Fixpoint mem x s :=
@@ -792,7 +792,7 @@ Proof.
split; auto. try discriminate. intro H; elim (H x); auto.
Qed.
-(** * Appartness *)
+(** * Membership *)
Lemma mem_spec : forall s x `{Ok s}, mem x s = true <-> InT x s.
Proof.