Theorem List for Intuitionistic Logic Explorer - 12701-12800 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
Theorem | bastg 12701 |
A member of a basis is a subset of the topology it generates.
(Contributed by NM, 16-Jul-2006.) (Revised by Mario Carneiro,
10-Jan-2015.)
|
⊢ (𝐵 ∈ 𝑉 → 𝐵 ⊆ (topGen‘𝐵)) |
|
Theorem | unitg 12702 |
The topology generated by a basis 𝐵 is a topology on ∪ 𝐵.
Importantly, this theorem means that we don't have to specify separately
the base set for the topological space generated by a basis. In other
words, any member of the class TopBases
completely specifies the
basis it corresponds to. (Contributed by NM, 16-Jul-2006.) (Proof
shortened by OpenAI, 30-Mar-2020.)
|
⊢ (𝐵 ∈ 𝑉 → ∪
(topGen‘𝐵) = ∪ 𝐵) |
|
Theorem | tgss 12703 |
Subset relation for generated topologies. (Contributed by NM,
7-May-2007.)
|
⊢ ((𝐶 ∈ 𝑉 ∧ 𝐵 ⊆ 𝐶) → (topGen‘𝐵) ⊆ (topGen‘𝐶)) |
|
Theorem | tgcl 12704 |
Show that a basis generates a topology. Remark in [Munkres] p. 79.
(Contributed by NM, 17-Jul-2006.)
|
⊢ (𝐵 ∈ TopBases → (topGen‘𝐵) ∈ Top) |
|
Theorem | tgclb 12705 |
The property tgcl 12704 can be reversed: if the topology generated
by 𝐵
is actually a topology, then 𝐵 must be a topological basis. This
yields an alternative definition of TopBases.
(Contributed by
Mario Carneiro, 2-Sep-2015.)
|
⊢ (𝐵 ∈ TopBases ↔ (topGen‘𝐵) ∈ Top) |
|
Theorem | tgtopon 12706 |
A basis generates a topology on ∪
𝐵. (Contributed by
Mario
Carneiro, 14-Aug-2015.)
|
⊢ (𝐵 ∈ TopBases → (topGen‘𝐵) ∈ (TopOn‘∪ 𝐵)) |
|
Theorem | topbas 12707 |
A topology is its own basis. (Contributed by NM, 17-Jul-2006.)
|
⊢ (𝐽 ∈ Top → 𝐽 ∈ TopBases) |
|
Theorem | tgtop 12708 |
A topology is its own basis. (Contributed by NM, 18-Jul-2006.)
|
⊢ (𝐽 ∈ Top → (topGen‘𝐽) = 𝐽) |
|
Theorem | eltop 12709 |
Membership in a topology, expressed without quantifiers. (Contributed
by NM, 19-Jul-2006.)
|
⊢ (𝐽 ∈ Top → (𝐴 ∈ 𝐽 ↔ 𝐴 ⊆ ∪
(𝐽 ∩ 𝒫 𝐴))) |
|
Theorem | eltop2 12710* |
Membership in a topology. (Contributed by NM, 19-Jul-2006.)
|
⊢ (𝐽 ∈ Top → (𝐴 ∈ 𝐽 ↔ ∀𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐽 (𝑥 ∈ 𝑦 ∧ 𝑦 ⊆ 𝐴))) |
|
Theorem | eltop3 12711* |
Membership in a topology. (Contributed by NM, 19-Jul-2006.)
|
⊢ (𝐽 ∈ Top → (𝐴 ∈ 𝐽 ↔ ∃𝑥(𝑥 ⊆ 𝐽 ∧ 𝐴 = ∪ 𝑥))) |
|
Theorem | tgdom 12712 |
A space has no more open sets than subsets of a basis. (Contributed by
Stefan O'Rear, 22-Feb-2015.) (Revised by Mario Carneiro,
9-Apr-2015.)
|
⊢ (𝐵 ∈ 𝑉 → (topGen‘𝐵) ≼ 𝒫 𝐵) |
|
Theorem | tgiun 12713* |
The indexed union of a set of basic open sets is in the generated
topology. (Contributed by Mario Carneiro, 2-Sep-2015.)
|
⊢ ((𝐵 ∈ 𝑉 ∧ ∀𝑥 ∈ 𝐴 𝐶 ∈ 𝐵) → ∪ 𝑥 ∈ 𝐴 𝐶 ∈ (topGen‘𝐵)) |
|
Theorem | tgidm 12714 |
The topology generator function is idempotent. (Contributed by NM,
18-Jul-2006.) (Revised by Mario Carneiro, 2-Sep-2015.)
|
⊢ (𝐵 ∈ 𝑉 → (topGen‘(topGen‘𝐵)) = (topGen‘𝐵)) |
|
Theorem | bastop 12715 |
Two ways to express that a basis is a topology. (Contributed by NM,
18-Jul-2006.)
|
⊢ (𝐵 ∈ TopBases → (𝐵 ∈ Top ↔ (topGen‘𝐵) = 𝐵)) |
|
Theorem | tgtop11 12716 |
The topology generation function is one-to-one when applied to completed
topologies. (Contributed by NM, 18-Jul-2006.)
|
⊢ ((𝐽 ∈ Top ∧ 𝐾 ∈ Top ∧ (topGen‘𝐽) = (topGen‘𝐾)) → 𝐽 = 𝐾) |
|
Theorem | en1top 12717 |
{∅} is the only topology with one element.
(Contributed by FL,
18-Aug-2008.)
|
⊢ (𝐽 ∈ Top → (𝐽 ≈ 1o ↔ 𝐽 = {∅})) |
|
Theorem | tgss3 12718 |
A criterion for determining whether one topology is finer than another.
Lemma 2.2 of [Munkres] p. 80 using
abbreviations. (Contributed by NM,
20-Jul-2006.) (Proof shortened by Mario Carneiro, 2-Sep-2015.)
|
⊢ ((𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑊) → ((topGen‘𝐵) ⊆ (topGen‘𝐶) ↔ 𝐵 ⊆ (topGen‘𝐶))) |
|
Theorem | tgss2 12719* |
A criterion for determining whether one topology is finer than another,
based on a comparison of their bases. Lemma 2.2 of [Munkres] p. 80.
(Contributed by NM, 20-Jul-2006.) (Proof shortened by Mario Carneiro,
2-Sep-2015.)
|
⊢ ((𝐵 ∈ 𝑉 ∧ ∪ 𝐵 = ∪
𝐶) →
((topGen‘𝐵) ⊆
(topGen‘𝐶) ↔
∀𝑥 ∈ ∪ 𝐵∀𝑦 ∈ 𝐵 (𝑥 ∈ 𝑦 → ∃𝑧 ∈ 𝐶 (𝑥 ∈ 𝑧 ∧ 𝑧 ⊆ 𝑦)))) |
|
Theorem | basgen 12720 |
Given a topology 𝐽, show that a subset 𝐵
satisfying the third
antecedent is a basis for it. Lemma 2.3 of [Munkres] p. 81 using
abbreviations. (Contributed by NM, 22-Jul-2006.) (Revised by Mario
Carneiro, 2-Sep-2015.)
|
⊢ ((𝐽 ∈ Top ∧ 𝐵 ⊆ 𝐽 ∧ 𝐽 ⊆ (topGen‘𝐵)) → (topGen‘𝐵) = 𝐽) |
|
Theorem | basgen2 12721* |
Given a topology 𝐽, show that a subset 𝐵
satisfying the third
antecedent is a basis for it. Lemma 2.3 of [Munkres] p. 81.
(Contributed by NM, 20-Jul-2006.) (Proof shortened by Mario Carneiro,
2-Sep-2015.)
|
⊢ ((𝐽 ∈ Top ∧ 𝐵 ⊆ 𝐽 ∧ ∀𝑥 ∈ 𝐽 ∀𝑦 ∈ 𝑥 ∃𝑧 ∈ 𝐵 (𝑦 ∈ 𝑧 ∧ 𝑧 ⊆ 𝑥)) → (topGen‘𝐵) = 𝐽) |
|
Theorem | 2basgeng 12722 |
Conditions that determine the equality of two generated topologies.
(Contributed by NM, 8-May-2007.) (Revised by Jim Kingdon,
5-Mar-2023.)
|
⊢ ((𝐵 ∈ 𝑉 ∧ 𝐵 ⊆ 𝐶 ∧ 𝐶 ⊆ (topGen‘𝐵)) → (topGen‘𝐵) = (topGen‘𝐶)) |
|
Theorem | bastop1 12723* |
A subset of a topology is a basis for the topology iff every member of
the topology is a union of members of the basis. We use the
idiom "(topGen‘𝐵) = 𝐽 " to express "𝐵 is a
basis for
topology 𝐽 " since we do not have a
separate notation for this.
Definition 15.35 of [Schechter] p.
428. (Contributed by NM,
2-Feb-2008.) (Proof shortened by Mario Carneiro, 2-Sep-2015.)
|
⊢ ((𝐽 ∈ Top ∧ 𝐵 ⊆ 𝐽) → ((topGen‘𝐵) = 𝐽 ↔ ∀𝑥 ∈ 𝐽 ∃𝑦(𝑦 ⊆ 𝐵 ∧ 𝑥 = ∪ 𝑦))) |
|
Theorem | bastop2 12724* |
A version of bastop1 12723 that doesn't have 𝐵 ⊆ 𝐽 in the antecedent.
(Contributed by NM, 3-Feb-2008.)
|
⊢ (𝐽 ∈ Top → ((topGen‘𝐵) = 𝐽 ↔ (𝐵 ⊆ 𝐽 ∧ ∀𝑥 ∈ 𝐽 ∃𝑦(𝑦 ⊆ 𝐵 ∧ 𝑥 = ∪ 𝑦)))) |
|
8.1.3 Examples of topologies
|
|
Theorem | distop 12725 |
The discrete topology on a set 𝐴. Part of Example 2 in [Munkres]
p. 77. (Contributed by FL, 17-Jul-2006.) (Revised by Mario Carneiro,
19-Mar-2015.)
|
⊢ (𝐴 ∈ 𝑉 → 𝒫 𝐴 ∈ Top) |
|
Theorem | topnex 12726 |
The class of all topologies is a proper class. The proof uses
discrete topologies and pwnex 4427. (Contributed by BJ, 2-May-2021.)
|
⊢ Top ∉ V |
|
Theorem | distopon 12727 |
The discrete topology on a set 𝐴, with base set. (Contributed by
Mario Carneiro, 13-Aug-2015.)
|
⊢ (𝐴 ∈ 𝑉 → 𝒫 𝐴 ∈ (TopOn‘𝐴)) |
|
Theorem | sn0topon 12728 |
The singleton of the empty set is a topology on the empty set.
(Contributed by Mario Carneiro, 13-Aug-2015.)
|
⊢ {∅} ∈
(TopOn‘∅) |
|
Theorem | sn0top 12729 |
The singleton of the empty set is a topology. (Contributed by Stefan
Allan, 3-Mar-2006.) (Proof shortened by Mario Carneiro,
13-Aug-2015.)
|
⊢ {∅} ∈ Top |
|
Theorem | epttop 12730* |
The excluded point topology. (Contributed by Mario Carneiro,
3-Sep-2015.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝑃 ∈ 𝐴) → {𝑥 ∈ 𝒫 𝐴 ∣ (𝑃 ∈ 𝑥 → 𝑥 = 𝐴)} ∈ (TopOn‘𝐴)) |
|
Theorem | distps 12731 |
The discrete topology on a set 𝐴 expressed as a topological space.
(Contributed by FL, 20-Aug-2006.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐾 = {〈(Base‘ndx),
𝐴〉,
〈(TopSet‘ndx), 𝒫 𝐴〉} ⇒ ⊢ 𝐾 ∈ TopSp |
|
8.1.4 Closure and interior
|
|
Syntax | ccld 12732 |
Extend class notation with the set of closed sets of a topology.
|
class Clsd |
|
Syntax | cnt 12733 |
Extend class notation with interior of a subset of a topology base set.
|
class int |
|
Syntax | ccl 12734 |
Extend class notation with closure of a subset of a topology base set.
|
class cls |
|
Definition | df-cld 12735* |
Define a function on topologies whose value is the set of closed sets of
the topology. (Contributed by NM, 2-Oct-2006.)
|
⊢ Clsd = (𝑗 ∈ Top ↦ {𝑥 ∈ 𝒫 ∪ 𝑗
∣ (∪ 𝑗 ∖ 𝑥) ∈ 𝑗}) |
|
Definition | df-ntr 12736* |
Define a function on topologies whose value is the interior function on
the subsets of the base set. See ntrval 12750. (Contributed by NM,
10-Sep-2006.)
|
⊢ int = (𝑗 ∈ Top ↦ (𝑥 ∈ 𝒫 ∪ 𝑗
↦ ∪ (𝑗 ∩ 𝒫 𝑥))) |
|
Definition | df-cls 12737* |
Define a function on topologies whose value is the closure function on
the subsets of the base set. See clsval 12751. (Contributed by NM,
3-Oct-2006.)
|
⊢ cls = (𝑗 ∈ Top ↦ (𝑥 ∈ 𝒫 ∪ 𝑗
↦ ∩ {𝑦 ∈ (Clsd‘𝑗) ∣ 𝑥 ⊆ 𝑦})) |
|
Theorem | fncld 12738 |
The closed-set generator is a well-behaved function. (Contributed by
Stefan O'Rear, 1-Feb-2015.)
|
⊢ Clsd Fn Top |
|
Theorem | cldval 12739* |
The set of closed sets of a topology. (Note that the set of open sets
is just the topology itself, so we don't have a separate definition.)
(Contributed by NM, 2-Oct-2006.) (Revised by Mario Carneiro,
11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → (Clsd‘𝐽) = {𝑥 ∈ 𝒫 𝑋 ∣ (𝑋 ∖ 𝑥) ∈ 𝐽}) |
|
Theorem | ntrfval 12740* |
The interior function on the subsets of a topology's base set.
(Contributed by NM, 10-Sep-2006.) (Revised by Mario Carneiro,
11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → (int‘𝐽) = (𝑥 ∈ 𝒫 𝑋 ↦ ∪
(𝐽 ∩ 𝒫 𝑥))) |
|
Theorem | clsfval 12741* |
The closure function on the subsets of a topology's base set.
(Contributed by NM, 3-Oct-2006.) (Revised by Mario Carneiro,
11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → (cls‘𝐽) = (𝑥 ∈ 𝒫 𝑋 ↦ ∩
{𝑦 ∈
(Clsd‘𝐽) ∣
𝑥 ⊆ 𝑦})) |
|
Theorem | cldrcl 12742 |
Reverse closure of the closed set operation. (Contributed by Stefan
O'Rear, 22-Feb-2015.)
|
⊢ (𝐶 ∈ (Clsd‘𝐽) → 𝐽 ∈ Top) |
|
Theorem | iscld 12743 |
The predicate "the class 𝑆 is a closed set". (Contributed
by NM,
2-Oct-2006.) (Revised by Mario Carneiro, 11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → (𝑆 ∈ (Clsd‘𝐽) ↔ (𝑆 ⊆ 𝑋 ∧ (𝑋 ∖ 𝑆) ∈ 𝐽))) |
|
Theorem | iscld2 12744 |
A subset of the underlying set of a topology is closed iff its
complement is open. (Contributed by NM, 4-Oct-2006.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → (𝑆 ∈ (Clsd‘𝐽) ↔ (𝑋 ∖ 𝑆) ∈ 𝐽)) |
|
Theorem | cldss 12745 |
A closed set is a subset of the underlying set of a topology.
(Contributed by NM, 5-Oct-2006.) (Revised by Stefan O'Rear,
22-Feb-2015.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝑆 ∈ (Clsd‘𝐽) → 𝑆 ⊆ 𝑋) |
|
Theorem | cldss2 12746 |
The set of closed sets is contained in the powerset of the base.
(Contributed by Mario Carneiro, 6-Jan-2014.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (Clsd‘𝐽) ⊆ 𝒫 𝑋 |
|
Theorem | cldopn 12747 |
The complement of a closed set is open. (Contributed by NM,
5-Oct-2006.) (Revised by Stefan O'Rear, 22-Feb-2015.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝑆 ∈ (Clsd‘𝐽) → (𝑋 ∖ 𝑆) ∈ 𝐽) |
|
Theorem | difopn 12748 |
The difference of a closed set with an open set is open. (Contributed
by Mario Carneiro, 6-Jan-2014.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐴 ∈ 𝐽 ∧ 𝐵 ∈ (Clsd‘𝐽)) → (𝐴 ∖ 𝐵) ∈ 𝐽) |
|
Theorem | topcld 12749 |
The underlying set of a topology is closed. Part of Theorem 6.1(1) of
[Munkres] p. 93. (Contributed by NM,
3-Oct-2006.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → 𝑋 ∈ (Clsd‘𝐽)) |
|
Theorem | ntrval 12750 |
The interior of a subset of a topology's base set is the union of all
the open sets it includes. Definition of interior of [Munkres] p. 94.
(Contributed by NM, 10-Sep-2006.) (Revised by Mario Carneiro,
11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → ((int‘𝐽)‘𝑆) = ∪ (𝐽 ∩ 𝒫 𝑆)) |
|
Theorem | clsval 12751* |
The closure of a subset of a topology's base set is the intersection of
all the closed sets that include it. Definition of closure of [Munkres]
p. 94. (Contributed by NM, 10-Sep-2006.) (Revised by Mario Carneiro,
11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → ((cls‘𝐽)‘𝑆) = ∩ {𝑥 ∈ (Clsd‘𝐽) ∣ 𝑆 ⊆ 𝑥}) |
|
Theorem | 0cld 12752 |
The empty set is closed. Part of Theorem 6.1(1) of [Munkres] p. 93.
(Contributed by NM, 4-Oct-2006.)
|
⊢ (𝐽 ∈ Top → ∅ ∈
(Clsd‘𝐽)) |
|
Theorem | uncld 12753 |
The union of two closed sets is closed. Equivalent to Theorem 6.1(3) of
[Munkres] p. 93. (Contributed by NM,
5-Oct-2006.)
|
⊢ ((𝐴 ∈ (Clsd‘𝐽) ∧ 𝐵 ∈ (Clsd‘𝐽)) → (𝐴 ∪ 𝐵) ∈ (Clsd‘𝐽)) |
|
Theorem | cldcls 12754 |
A closed subset equals its own closure. (Contributed by NM,
15-Mar-2007.)
|
⊢ (𝑆 ∈ (Clsd‘𝐽) → ((cls‘𝐽)‘𝑆) = 𝑆) |
|
Theorem | iuncld 12755* |
A finite indexed union of closed sets is closed. (Contributed by Mario
Carneiro, 19-Sep-2015.) (Revised by Jim Kingdon, 10-Mar-2023.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝐴 ∈ Fin ∧ ∀𝑥 ∈ 𝐴 𝐵 ∈ (Clsd‘𝐽)) → ∪ 𝑥 ∈ 𝐴 𝐵 ∈ (Clsd‘𝐽)) |
|
Theorem | unicld 12756 |
A finite union of closed sets is closed. (Contributed by Mario
Carneiro, 19-Sep-2015.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝐴 ∈ Fin ∧ 𝐴 ⊆ (Clsd‘𝐽)) → ∪
𝐴 ∈ (Clsd‘𝐽)) |
|
Theorem | ntropn 12757 |
The interior of a subset of a topology's underlying set is open.
(Contributed by NM, 11-Sep-2006.) (Revised by Mario Carneiro,
11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → ((int‘𝐽)‘𝑆) ∈ 𝐽) |
|
Theorem | clsss 12758 |
Subset relationship for closure. (Contributed by NM, 10-Feb-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋 ∧ 𝑇 ⊆ 𝑆) → ((cls‘𝐽)‘𝑇) ⊆ ((cls‘𝐽)‘𝑆)) |
|
Theorem | ntrss 12759 |
Subset relationship for interior. (Contributed by NM, 3-Oct-2007.)
(Revised by Jim Kingdon, 11-Mar-2023.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋 ∧ 𝑇 ⊆ 𝑆) → ((int‘𝐽)‘𝑇) ⊆ ((int‘𝐽)‘𝑆)) |
|
Theorem | sscls 12760 |
A subset of a topology's underlying set is included in its closure.
(Contributed by NM, 22-Feb-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → 𝑆 ⊆ ((cls‘𝐽)‘𝑆)) |
|
Theorem | ntrss2 12761 |
A subset includes its interior. (Contributed by NM, 3-Oct-2007.)
(Revised by Mario Carneiro, 11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → ((int‘𝐽)‘𝑆) ⊆ 𝑆) |
|
Theorem | ssntr 12762 |
An open subset of a set is a subset of the set's interior. (Contributed
by Jeff Hankins, 31-Aug-2009.) (Revised by Mario Carneiro,
11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) ∧ (𝑂 ∈ 𝐽 ∧ 𝑂 ⊆ 𝑆)) → 𝑂 ⊆ ((int‘𝐽)‘𝑆)) |
|
Theorem | ntrss3 12763 |
The interior of a subset of a topological space is included in the
space. (Contributed by NM, 1-Oct-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → ((int‘𝐽)‘𝑆) ⊆ 𝑋) |
|
Theorem | ntrin 12764 |
A pairwise intersection of interiors is the interior of the
intersection. This does not always hold for arbitrary intersections.
(Contributed by Jeff Hankins, 31-Aug-2009.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝐴 ⊆ 𝑋 ∧ 𝐵 ⊆ 𝑋) → ((int‘𝐽)‘(𝐴 ∩ 𝐵)) = (((int‘𝐽)‘𝐴) ∩ ((int‘𝐽)‘𝐵))) |
|
Theorem | isopn3 12765 |
A subset is open iff it equals its own interior. (Contributed by NM,
9-Oct-2006.) (Revised by Mario Carneiro, 11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → (𝑆 ∈ 𝐽 ↔ ((int‘𝐽)‘𝑆) = 𝑆)) |
|
Theorem | ntridm 12766 |
The interior operation is idempotent. (Contributed by NM,
2-Oct-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → ((int‘𝐽)‘((int‘𝐽)‘𝑆)) = ((int‘𝐽)‘𝑆)) |
|
Theorem | clstop 12767 |
The closure of a topology's underlying set is the entire set.
(Contributed by NM, 5-Oct-2007.) (Proof shortened by Jim Kingdon,
11-Mar-2023.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → ((cls‘𝐽)‘𝑋) = 𝑋) |
|
Theorem | ntrtop 12768 |
The interior of a topology's underlying set is the entire set.
(Contributed by NM, 12-Sep-2006.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → ((int‘𝐽)‘𝑋) = 𝑋) |
|
Theorem | clsss2 12769 |
If a subset is included in a closed set, so is the subset's closure.
(Contributed by NM, 22-Feb-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐶 ∈ (Clsd‘𝐽) ∧ 𝑆 ⊆ 𝐶) → ((cls‘𝐽)‘𝑆) ⊆ 𝐶) |
|
Theorem | clsss3 12770 |
The closure of a subset of a topological space is included in the space.
(Contributed by NM, 26-Feb-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → ((cls‘𝐽)‘𝑆) ⊆ 𝑋) |
|
Theorem | ntrcls0 12771 |
A subset whose closure has an empty interior also has an empty interior.
(Contributed by NM, 4-Oct-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋 ∧ ((int‘𝐽)‘((cls‘𝐽)‘𝑆)) = ∅) → ((int‘𝐽)‘𝑆) = ∅) |
|
Theorem | ntreq0 12772* |
Two ways to say that a subset has an empty interior. (Contributed by
NM, 3-Oct-2007.) (Revised by Jim Kingdon, 11-Mar-2023.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → (((int‘𝐽)‘𝑆) = ∅ ↔ ∀𝑥 ∈ 𝐽 (𝑥 ⊆ 𝑆 → 𝑥 = ∅))) |
|
Theorem | cls0 12773 |
The closure of the empty set. (Contributed by NM, 2-Oct-2007.) (Proof
shortened by Jim Kingdon, 12-Mar-2023.)
|
⊢ (𝐽 ∈ Top → ((cls‘𝐽)‘∅) =
∅) |
|
Theorem | ntr0 12774 |
The interior of the empty set. (Contributed by NM, 2-Oct-2007.)
|
⊢ (𝐽 ∈ Top → ((int‘𝐽)‘∅) =
∅) |
|
Theorem | isopn3i 12775 |
An open subset equals its own interior. (Contributed by Mario Carneiro,
30-Dec-2016.)
|
⊢ ((𝐽 ∈ Top ∧ 𝑆 ∈ 𝐽) → ((int‘𝐽)‘𝑆) = 𝑆) |
|
Theorem | discld 12776 |
The open sets of a discrete topology are closed and its closed sets are
open. (Contributed by FL, 7-Jun-2007.) (Revised by Mario Carneiro,
7-Apr-2015.)
|
⊢ (𝐴 ∈ 𝑉 → (Clsd‘𝒫 𝐴) = 𝒫 𝐴) |
|
Theorem | sn0cld 12777 |
The closed sets of the topology {∅}.
(Contributed by FL,
5-Jan-2009.)
|
⊢ (Clsd‘{∅}) =
{∅} |
|
8.1.5 Neighborhoods
|
|
Syntax | cnei 12778 |
Extend class notation with neighborhood relation for topologies.
|
class nei |
|
Definition | df-nei 12779* |
Define a function on topologies whose value is a map from a subset to
its neighborhoods. (Contributed by NM, 11-Feb-2007.)
|
⊢ nei = (𝑗 ∈ Top ↦ (𝑥 ∈ 𝒫 ∪ 𝑗
↦ {𝑦 ∈
𝒫 ∪ 𝑗 ∣ ∃𝑔 ∈ 𝑗 (𝑥 ⊆ 𝑔 ∧ 𝑔 ⊆ 𝑦)})) |
|
Theorem | neifval 12780* |
Value of the neighborhood function on the subsets of the base set of a
topology. (Contributed by NM, 11-Feb-2007.) (Revised by Mario
Carneiro, 11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → (nei‘𝐽) = (𝑥 ∈ 𝒫 𝑋 ↦ {𝑣 ∈ 𝒫 𝑋 ∣ ∃𝑔 ∈ 𝐽 (𝑥 ⊆ 𝑔 ∧ 𝑔 ⊆ 𝑣)})) |
|
Theorem | neif 12781 |
The neighborhood function is a function from the set of the subsets of
the base set of a topology. (Contributed by NM, 12-Feb-2007.) (Revised
by Mario Carneiro, 11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → (nei‘𝐽) Fn 𝒫 𝑋) |
|
Theorem | neiss2 12782 |
A set with a neighborhood is a subset of the base set of a topology.
(This theorem depends on a function's value being empty outside of its
domain, but it will make later theorems simpler to state.) (Contributed
by NM, 12-Feb-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑁 ∈ ((nei‘𝐽)‘𝑆)) → 𝑆 ⊆ 𝑋) |
|
Theorem | neival 12783* |
Value of the set of neighborhoods of a subset of the base set of a
topology. (Contributed by NM, 11-Feb-2007.) (Revised by Mario
Carneiro, 11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → ((nei‘𝐽)‘𝑆) = {𝑣 ∈ 𝒫 𝑋 ∣ ∃𝑔 ∈ 𝐽 (𝑆 ⊆ 𝑔 ∧ 𝑔 ⊆ 𝑣)}) |
|
Theorem | isnei 12784* |
The predicate "the class 𝑁 is a neighborhood of 𝑆".
(Contributed by FL, 25-Sep-2006.) (Revised by Mario Carneiro,
11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋) → (𝑁 ∈ ((nei‘𝐽)‘𝑆) ↔ (𝑁 ⊆ 𝑋 ∧ ∃𝑔 ∈ 𝐽 (𝑆 ⊆ 𝑔 ∧ 𝑔 ⊆ 𝑁)))) |
|
Theorem | neiint 12785 |
An intuitive definition of a neighborhood in terms of interior.
(Contributed by Szymon Jaroszewicz, 18-Dec-2007.) (Revised by Mario
Carneiro, 11-Nov-2013.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋 ∧ 𝑁 ⊆ 𝑋) → (𝑁 ∈ ((nei‘𝐽)‘𝑆) ↔ 𝑆 ⊆ ((int‘𝐽)‘𝑁))) |
|
Theorem | isneip 12786* |
The predicate "the class 𝑁 is a neighborhood of point 𝑃".
(Contributed by NM, 26-Feb-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑃 ∈ 𝑋) → (𝑁 ∈ ((nei‘𝐽)‘{𝑃}) ↔ (𝑁 ⊆ 𝑋 ∧ ∃𝑔 ∈ 𝐽 (𝑃 ∈ 𝑔 ∧ 𝑔 ⊆ 𝑁)))) |
|
Theorem | neii1 12787 |
A neighborhood is included in the topology's base set. (Contributed by
NM, 12-Feb-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑁 ∈ ((nei‘𝐽)‘𝑆)) → 𝑁 ⊆ 𝑋) |
|
Theorem | neisspw 12788 |
The neighborhoods of any set are subsets of the base set. (Contributed
by Stefan O'Rear, 6-Aug-2015.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → ((nei‘𝐽)‘𝑆) ⊆ 𝒫 𝑋) |
|
Theorem | neii2 12789* |
Property of a neighborhood. (Contributed by NM, 12-Feb-2007.)
|
⊢ ((𝐽 ∈ Top ∧ 𝑁 ∈ ((nei‘𝐽)‘𝑆)) → ∃𝑔 ∈ 𝐽 (𝑆 ⊆ 𝑔 ∧ 𝑔 ⊆ 𝑁)) |
|
Theorem | neiss 12790 |
Any neighborhood of a set 𝑆 is also a neighborhood of any subset
𝑅
⊆ 𝑆. Similar
to Proposition 1 of [BourbakiTop1] p.
I.2.
(Contributed by FL, 25-Sep-2006.)
|
⊢ ((𝐽 ∈ Top ∧ 𝑁 ∈ ((nei‘𝐽)‘𝑆) ∧ 𝑅 ⊆ 𝑆) → 𝑁 ∈ ((nei‘𝐽)‘𝑅)) |
|
Theorem | ssnei 12791 |
A set is included in any of its neighborhoods. Generalization to
subsets of elnei 12792. (Contributed by FL, 16-Nov-2006.)
|
⊢ ((𝐽 ∈ Top ∧ 𝑁 ∈ ((nei‘𝐽)‘𝑆)) → 𝑆 ⊆ 𝑁) |
|
Theorem | elnei 12792 |
A point belongs to any of its neighborhoods. Property Viii of
[BourbakiTop1] p. I.3. (Contributed
by FL, 28-Sep-2006.)
|
⊢ ((𝐽 ∈ Top ∧ 𝑃 ∈ 𝐴 ∧ 𝑁 ∈ ((nei‘𝐽)‘{𝑃})) → 𝑃 ∈ 𝑁) |
|
Theorem | 0nnei 12793 |
The empty set is not a neighborhood of a nonempty set. (Contributed by
FL, 18-Sep-2007.)
|
⊢ ((𝐽 ∈ Top ∧ 𝑆 ≠ ∅) → ¬ ∅ ∈
((nei‘𝐽)‘𝑆)) |
|
Theorem | neipsm 12794* |
A neighborhood of a set is a neighborhood of every point in the set.
Proposition 1 of [BourbakiTop1] p.
I.2. (Contributed by FL,
16-Nov-2006.) (Revised by Jim Kingdon, 22-Mar-2023.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ⊆ 𝑋 ∧ ∃𝑥 𝑥 ∈ 𝑆) → (𝑁 ∈ ((nei‘𝐽)‘𝑆) ↔ ∀𝑝 ∈ 𝑆 𝑁 ∈ ((nei‘𝐽)‘{𝑝}))) |
|
Theorem | opnneissb 12795 |
An open set is a neighborhood of any of its subsets. (Contributed by
FL, 2-Oct-2006.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑁 ∈ 𝐽 ∧ 𝑆 ⊆ 𝑋) → (𝑆 ⊆ 𝑁 ↔ 𝑁 ∈ ((nei‘𝐽)‘𝑆))) |
|
Theorem | opnssneib 12796 |
Any superset of an open set is a neighborhood of it. (Contributed by
NM, 14-Feb-2007.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ ((𝐽 ∈ Top ∧ 𝑆 ∈ 𝐽 ∧ 𝑁 ⊆ 𝑋) → (𝑆 ⊆ 𝑁 ↔ 𝑁 ∈ ((nei‘𝐽)‘𝑆))) |
|
Theorem | ssnei2 12797 |
Any subset 𝑀 of 𝑋 containing a
neighborhood 𝑁 of a set 𝑆
is a neighborhood of this set. Generalization to subsets of Property
Vi of [BourbakiTop1] p. I.3. (Contributed by FL,
2-Oct-2006.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (((𝐽 ∈ Top ∧ 𝑁 ∈ ((nei‘𝐽)‘𝑆)) ∧ (𝑁 ⊆ 𝑀 ∧ 𝑀 ⊆ 𝑋)) → 𝑀 ∈ ((nei‘𝐽)‘𝑆)) |
|
Theorem | opnneiss 12798 |
An open set is a neighborhood of any of its subsets. (Contributed by NM,
13-Feb-2007.)
|
⊢ ((𝐽 ∈ Top ∧ 𝑁 ∈ 𝐽 ∧ 𝑆 ⊆ 𝑁) → 𝑁 ∈ ((nei‘𝐽)‘𝑆)) |
|
Theorem | opnneip 12799 |
An open set is a neighborhood of any of its members. (Contributed by NM,
8-Mar-2007.)
|
⊢ ((𝐽 ∈ Top ∧ 𝑁 ∈ 𝐽 ∧ 𝑃 ∈ 𝑁) → 𝑁 ∈ ((nei‘𝐽)‘{𝑃})) |
|
Theorem | tpnei 12800 |
The underlying set of a topology is a neighborhood of any of its
subsets. Special case of opnneiss 12798. (Contributed by FL,
2-Oct-2006.)
|
⊢ 𝑋 = ∪ 𝐽 ⇒ ⊢ (𝐽 ∈ Top → (𝑆 ⊆ 𝑋 ↔ 𝑋 ∈ ((nei‘𝐽)‘𝑆))) |