aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FSetAVL.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-05 16:31:16 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-05 16:31:16 +0000
commit316e114dd188f85ec657420989bf909ecfe9d006 (patch)
tree37229712b18593049740b28b6a18a5d9e7150faa /theories/FSets/FSetAVL.v
parent44cedab7be5a44a01d467fbd2dba24400d575206 (diff)
kill some useless module aliases E:=X (for better name printing, see Elie's 14097)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10511 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FSetAVL.v')
-rw-r--r--theories/FSets/FSetAVL.v9
1 files changed, 4 insertions, 5 deletions
diff --git a/theories/FSets/FSetAVL.v b/theories/FSets/FSetAVL.v
index 20fdae9fe..b6bcb6fb4 100644
--- a/theories/FSets/FSetAVL.v
+++ b/theories/FSets/FSetAVL.v
@@ -30,7 +30,6 @@ Module II:=MoreInt(I).
Import II.
Open Local Scope Int_scope.
-Module E := X.
Module MX := OrderedTypeFacts X.
Definition elt := X.t.
@@ -1647,7 +1646,7 @@ Fixpoint for_all (s:t) : bool := match s with
| Node l x r _ => f x && for_all l && for_all r
end.
-Lemma for_all_1 : forall s, compat_bool E.eq f ->
+Lemma for_all_1 : forall s, compat_bool X.eq f ->
For_all (fun x => f x = true) s -> for_all s = true.
Proof.
induction s; simpl; auto.
@@ -1658,7 +1657,7 @@ Proof.
destruct (f t); simpl; auto.
Qed.
-Lemma for_all_2 : forall s, compat_bool E.eq f ->
+Lemma for_all_2 : forall s, compat_bool X.eq f ->
for_all s = true -> For_all (fun x => f x = true) s.
Proof.
induction s; simpl; auto; intros; red; intros; inv In.
@@ -1676,7 +1675,7 @@ Fixpoint exists_ (s:t) : bool := match s with
| Node l x r _ => f x || exists_ l || exists_ r
end.
-Lemma exists_1 : forall s, compat_bool E.eq f ->
+Lemma exists_1 : forall s, compat_bool X.eq f ->
Exists (fun x => f x = true) s -> exists_ s = true.
Proof.
induction s; simpl; destruct 2 as (x,(U,V)); inv In.
@@ -1686,7 +1685,7 @@ Proof.
apply orb_true_intro; right; apply IHs2; firstorder.
Qed.
-Lemma exists_2 : forall s, compat_bool E.eq f ->
+Lemma exists_2 : forall s, compat_bool X.eq f ->
exists_ s = true -> Exists (fun x => f x = true) s.
Proof.
induction s; simpl; intros.