| Metamath
Proof Explorer Theorem List (p. 488 of 494) | < Previous Next > | |
| Bad symbols? Try the
GIF version. |
||
|
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
||
| Color key: | (1-30884) |
(30885-32407) |
(32408-49320) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | mofsssn 48701* | There is at most one function into a subclass of a singleton. (Contributed by Zhi Wang, 24-Sep-2024.) |
| ⊢ (𝐵 ⊆ {𝑌} → ∃*𝑓 𝑓:𝐴⟶𝐵) | ||
| Theorem | mofmo 48702* | There is at most one function into a class containing at most one element. (Contributed by Zhi Wang, 19-Sep-2024.) |
| ⊢ (∃*𝑥 𝑥 ∈ 𝐵 → ∃*𝑓 𝑓:𝐴⟶𝐵) | ||
| Theorem | mofeu 48703* | The uniqueness of a function into a set with at most one element. (Contributed by Zhi Wang, 1-Oct-2024.) |
| ⊢ 𝐺 = (𝐴 × 𝐵) & ⊢ (𝜑 → (𝐵 = ∅ → 𝐴 = ∅)) & ⊢ (𝜑 → ∃*𝑥 𝑥 ∈ 𝐵) ⇒ ⊢ (𝜑 → (𝐹:𝐴⟶𝐵 ↔ 𝐹 = 𝐺)) | ||
| Theorem | elfvne0 48704 | If a function value has a member, then the function is not an empty set (An artifact of our function value definition.) (Contributed by Zhi Wang, 16-Sep-2024.) |
| ⊢ (𝐴 ∈ (𝐹‘𝐵) → 𝐹 ≠ ∅) | ||
| Theorem | fdomne0 48705 | A function with non-empty domain is non-empty and has non-empty codomain. (Contributed by Zhi Wang, 1-Oct-2024.) |
| ⊢ ((𝐹:𝑋⟶𝑌 ∧ 𝑋 ≠ ∅) → (𝐹 ≠ ∅ ∧ 𝑌 ≠ ∅)) | ||
| Theorem | f1sn2g 48706 | A function that maps a singleton to a class is injective. (Contributed by Zhi Wang, 1-Oct-2024.) |
| ⊢ ((𝐴 ∈ 𝑉 ∧ 𝐹:{𝐴}⟶𝐵) → 𝐹:{𝐴}–1-1→𝐵) | ||
| Theorem | f102g 48707 | A function that maps the empty set to a class is injective. (Contributed by Zhi Wang, 1-Oct-2024.) |
| ⊢ ((𝐴 = ∅ ∧ 𝐹:𝐴⟶𝐵) → 𝐹:𝐴–1-1→𝐵) | ||
| Theorem | f1mo 48708* | A function that maps a set with at most one element to a class is injective. (Contributed by Zhi Wang, 1-Oct-2024.) |
| ⊢ ((∃*𝑥 𝑥 ∈ 𝐴 ∧ 𝐹:𝐴⟶𝐵) → 𝐹:𝐴–1-1→𝐵) | ||
| Theorem | f002 48709 | A function with an empty codomain must have empty domain. (Contributed by Zhi Wang, 1-Oct-2024.) |
| ⊢ (𝜑 → 𝐹:𝐴⟶𝐵) ⇒ ⊢ (𝜑 → (𝐵 = ∅ → 𝐴 = ∅)) | ||
| Theorem | map0cor 48710* | A function exists iff an empty codomain is accompanied with an empty domain. (Contributed by Zhi Wang, 1-Oct-2024.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝐵 ∈ 𝑊) ⇒ ⊢ (𝜑 → ((𝐵 = ∅ → 𝐴 = ∅) ↔ ∃𝑓 𝑓:𝐴⟶𝐵)) | ||
| Theorem | fvconstr 48711 | Two ways of expressing 𝐴𝑅𝐵. (Contributed by Zhi Wang, 18-Sep-2024.) |
| ⊢ (𝜑 → 𝐹 = (𝑅 × {𝑌})) & ⊢ (𝜑 → 𝑌 ∈ 𝑉) & ⊢ (𝜑 → 𝑌 ≠ ∅) ⇒ ⊢ (𝜑 → (𝐴𝑅𝐵 ↔ (𝐴𝐹𝐵) = 𝑌)) | ||
| Theorem | fvconstrn0 48712 | Two ways of expressing 𝐴𝑅𝐵. (Contributed by Zhi Wang, 20-Sep-2024.) |
| ⊢ (𝜑 → 𝐹 = (𝑅 × {𝑌})) & ⊢ (𝜑 → 𝑌 ∈ 𝑉) & ⊢ (𝜑 → 𝑌 ≠ ∅) ⇒ ⊢ (𝜑 → (𝐴𝑅𝐵 ↔ (𝐴𝐹𝐵) ≠ ∅)) | ||
| Theorem | fvconstr2 48713 | Two ways of expressing 𝐴𝑅𝐵. (Contributed by Zhi Wang, 18-Sep-2024.) |
| ⊢ (𝜑 → 𝐹 = (𝑅 × {𝑌})) & ⊢ (𝜑 → 𝑋 ∈ (𝐴𝐹𝐵)) ⇒ ⊢ (𝜑 → 𝐴𝑅𝐵) | ||
| Theorem | ovmpt4d 48714* | Deduction version of ovmpt4g 7563. (This is the operation analogue of fvmpt2d 7010.) (Contributed by Zhi Wang, 9-Oct-2025.) |
| ⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐴, 𝑦 ∈ 𝐵 ↦ 𝐶)) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵)) → 𝐶 ∈ 𝑉) ⇒ ⊢ ((𝜑 ∧ (𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵)) → (𝑥𝐹𝑦) = 𝐶) | ||
| Theorem | fonex 48715 | The domain of a surjection is a proper class if the range is a proper class as well. Can be used to prove that if a structure component extractor restricted to a class maps onto a proper class, then the class is a proper class as well. (Contributed by Zhi Wang, 20-Oct-2025.) |
| ⊢ 𝐵 ∉ V & ⊢ 𝐹:𝐴–onto→𝐵 ⇒ ⊢ 𝐴 ∉ V | ||
| Theorem | fmpodg 48716* | Domain and codomain of the mapping operation; deduction form. (Contributed by Zhi Wang, 29-Sep-2025.) |
| ⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐴, 𝑦 ∈ 𝐵 ↦ 𝐶)) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵)) → 𝐶 ∈ 𝑆) & ⊢ (𝜑 → 𝑅 = (𝐴 × 𝐵)) ⇒ ⊢ (𝜑 → 𝐹:𝑅⟶𝑆) | ||
| Theorem | fmpod 48717* | Domain and codomain of the mapping operation; deduction form. (Contributed by Zhi Wang, 30-Sep-2025.) |
| ⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐴, 𝑦 ∈ 𝐵 ↦ 𝐶)) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵)) → 𝐶 ∈ 𝑆) ⇒ ⊢ (𝜑 → 𝐹:(𝐴 × 𝐵)⟶𝑆) | ||
| Theorem | resinsnlem 48718 | Lemma for resinsnALT 48720. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (𝜑 → (𝜒 ↔ ¬ 𝜓)) & ⊢ (¬ 𝜑 → 𝜒) ⇒ ⊢ ((𝜑 ∧ 𝜓) ↔ ¬ 𝜒) | ||
| Theorem | resinsn 48719 | Restriction to the intersection with a singleton. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ ((𝐹 ↾ (𝐴 ∩ {𝐵})) = ∅ ↔ ¬ 𝐵 ∈ (dom 𝐹 ∩ 𝐴)) | ||
| Theorem | resinsnALT 48720 | Restriction to the intersection with a singleton. (Contributed by Zhi Wang, 6-Oct-2025.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ ((𝐹 ↾ (𝐴 ∩ {𝐵})) = ∅ ↔ ¬ 𝐵 ∈ (dom 𝐹 ∩ 𝐴)) | ||
| Theorem | dftpos5 48721* | Alternate definition of tpos. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ tpos 𝐹 = (𝐹 ∘ ((𝑥 ∈ ◡dom 𝐹 ↦ ∪ ◡{𝑥}) ∪ {〈∅, ∅〉})) | ||
| Theorem | dftpos6 48722* | Alternate definition of tpos. The second half of the right hand side could apply ressn 6287 and become (𝐹 ↾ {∅}) (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ tpos 𝐹 = ((𝐹 ∘ (𝑥 ∈ ◡dom 𝐹 ↦ ∪ ◡{𝑥})) ∪ ({∅} × (𝐹 “ {∅}))) | ||
| Theorem | dmtposss 48723 | The domain of tpos 𝐹 is a subset. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ dom tpos 𝐹 ⊆ ((V × V) ∪ {∅}) | ||
| Theorem | tposres0 48724 | The transposition of a set restricted to the empty set is the set restricted to the empty set. See also ressn 6287 and dftpos6 48722 for an alternate proof. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (tpos 𝐹 ↾ {∅}) = (𝐹 ↾ {∅}) | ||
| Theorem | tposresg 48725 | The transposition restricted to a set. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (tpos 𝐹 ↾ 𝑅) = ((tpos 𝐹 ↾ ◡◡𝑅) ∪ (𝐹 ↾ (𝑅 ∩ {∅}))) | ||
| Theorem | tposrescnv 48726* | The transposition restricted to a converse is the transposition of the restricted class, with the empty set removed from the domain. Note that the right hand side is a more useful form of (tpos (𝐹 ↾ 𝑅) ↾ (V ∖ {∅})) by df-tpos 8234. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (tpos 𝐹 ↾ ◡𝑅) = (𝐹 ∘ (𝑥 ∈ ◡dom (𝐹 ↾ 𝑅) ↦ ∪ ◡{𝑥})) | ||
| Theorem | tposres2 48727 | The transposition restricted to a set. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (𝜑 → ¬ ∅ ∈ (dom 𝐹 ∩ 𝑅)) ⇒ ⊢ (𝜑 → (tpos 𝐹 ↾ 𝑅) = (tpos 𝐹 ↾ ◡◡𝑅)) | ||
| Theorem | tposres3 48728 | The transposition restricted to a set. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (𝜑 → ¬ ∅ ∈ (dom 𝐹 ∩ 𝑅)) ⇒ ⊢ (𝜑 → (tpos 𝐹 ↾ 𝑅) = tpos (𝐹 ↾ ◡𝑅)) | ||
| Theorem | tposres 48729 | The transposition restricted to a relation. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (Rel 𝑅 → (tpos 𝐹 ↾ 𝑅) = tpos (𝐹 ↾ ◡𝑅)) | ||
| Theorem | tposresxp 48730 | The transposition restricted to a Cartesian product. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (tpos 𝐹 ↾ (𝐴 × 𝐵)) = tpos (𝐹 ↾ (𝐵 × 𝐴)) | ||
| Theorem | tposf1o 48731 | Condition of a bijective transposition. (Contributed by Zhi Wang, 5-Oct-2025.) |
| ⊢ (𝐹:(𝐴 × 𝐵)–1-1-onto→𝐶 → tpos 𝐹:(𝐵 × 𝐴)–1-1-onto→𝐶) | ||
| Theorem | tposid 48732 | Swap an ordered pair. (Contributed by Zhi Wang, 5-Oct-2025.) |
| ⊢ (𝑋tpos I 𝑌) = 〈𝑌, 𝑋〉 | ||
| Theorem | tposidres 48733 | Swap an ordered pair. (Contributed by Zhi Wang, 5-Oct-2025.) |
| ⊢ (𝜑 → 𝑋 ∈ 𝐴) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) ⇒ ⊢ (𝜑 → (𝑌tpos ( I ↾ (𝐴 × 𝐵))𝑋) = 〈𝑋, 𝑌〉) | ||
| Theorem | tposidf1o 48734 | The swap function, or the twisting map, is bijective. (Contributed by Zhi Wang, 5-Oct-2025.) |
| ⊢ tpos ( I ↾ (𝐴 × 𝐵)):(𝐵 × 𝐴)–1-1-onto→(𝐴 × 𝐵) | ||
| Theorem | tposideq 48735* | Two ways of expressing the swap function. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ (Rel 𝑅 → (tpos I ↾ 𝑅) = (𝑥 ∈ 𝑅 ↦ ∪ ◡{𝑥})) | ||
| Theorem | tposideq2 48736* | Two ways of expressing the swap function. (Contributed by Zhi Wang, 6-Oct-2025.) |
| ⊢ 𝑅 = (𝐴 × 𝐵) ⇒ ⊢ (tpos I ↾ 𝑅) = (𝑥 ∈ 𝑅 ↦ ∪ ◡{𝑥}) | ||
| Theorem | fvconst0ci 48737 | A constant function's value is either the constant or the empty set. (An artifact of our function value definition.) (Contributed by Zhi Wang, 18-Sep-2024.) |
| ⊢ 𝐵 ∈ V & ⊢ 𝑌 = ((𝐴 × {𝐵})‘𝑋) ⇒ ⊢ (𝑌 = ∅ ∨ 𝑌 = 𝐵) | ||
| Theorem | fvconstdomi 48738 | A constant function's value is dominated by the constant. (An artifact of our function value definition.) (Contributed by Zhi Wang, 18-Sep-2024.) |
| ⊢ 𝐵 ∈ V ⇒ ⊢ ((𝐴 × {𝐵})‘𝑋) ≼ 𝐵 | ||
| Theorem | f1omo 48739* | There is at most one element in the function value of a constant function whose output is 1o. (An artifact of our function value definition.) Proof could be significantly shortened by fvconstdomi 48738 assuming ax-un 7738 (see f1omoALT 48740). (Contributed by Zhi Wang, 19-Sep-2024.) |
| ⊢ (𝜑 → 𝐹 = (𝐴 × {1o})) ⇒ ⊢ (𝜑 → ∃*𝑦 𝑦 ∈ (𝐹‘𝑋)) | ||
| Theorem | f1omoALT 48740* | There is at most one element in the function value of a constant function whose output is 1o. (An artifact of our function value definition.) Use f1omo 48739 without assuming ax-un 7738. (Contributed by Zhi Wang, 18-Sep-2024.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ (𝜑 → 𝐹 = (𝐴 × {1o})) ⇒ ⊢ (𝜑 → ∃*𝑦 𝑦 ∈ (𝐹‘𝑋)) | ||
| Theorem | iccin 48741 | Intersection of two closed intervals of extended reals. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ (((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*) ∧ (𝐶 ∈ ℝ* ∧ 𝐷 ∈ ℝ*)) → ((𝐴[,]𝐵) ∩ (𝐶[,]𝐷)) = (if(𝐴 ≤ 𝐶, 𝐶, 𝐴)[,]if(𝐵 ≤ 𝐷, 𝐵, 𝐷))) | ||
| Theorem | iccdisj2 48742 | If the upper bound of one closed interval is less than the lower bound of the other, the intervals are disjoint. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ ((𝐴 ∈ ℝ* ∧ 𝐷 ∈ ℝ* ∧ 𝐵 < 𝐶) → ((𝐴[,]𝐵) ∩ (𝐶[,]𝐷)) = ∅) | ||
| Theorem | iccdisj 48743 | If the upper bound of one closed interval is less than the lower bound of the other, the intervals are disjoint. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ ((((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*) ∧ (𝐶 ∈ ℝ* ∧ 𝐷 ∈ ℝ*)) ∧ 𝐵 < 𝐶) → ((𝐴[,]𝐵) ∩ (𝐶[,]𝐷)) = ∅) | ||
| Theorem | slotresfo 48744* | The condition of a structure component extractor restricted to a class being a surjection. This combined with fonex 48715 can be used to prove a class being proper. (Contributed by Zhi Wang, 20-Oct-2025.) |
| ⊢ 𝐸 Fn V & ⊢ (𝑘 ∈ 𝐴 → (𝐸‘𝑘) ∈ 𝑉) & ⊢ (𝑏 ∈ 𝑉 → 𝐾 ∈ 𝐴) & ⊢ (𝑏 ∈ 𝑉 → 𝑏 = (𝐸‘𝐾)) ⇒ ⊢ (𝐸 ↾ 𝐴):𝐴–onto→𝑉 | ||
| Theorem | mreuniss 48745 | The union of a collection of closed sets is a subset. (Contributed by Zhi Wang, 29-Sep-2024.) |
| ⊢ ((𝐶 ∈ (Moore‘𝑋) ∧ 𝑆 ⊆ 𝐶) → ∪ 𝑆 ⊆ 𝑋) | ||
Additional contents for topology. | ||
| Theorem | clduni 48746 | The union of closed sets is the underlying set of the topology (the union of open sets). (Contributed by Zhi Wang, 6-Sep-2024.) |
| ⊢ (𝐽 ∈ Top → ∪ (Clsd‘𝐽) = ∪ 𝐽) | ||
| Theorem | opncldeqv 48747* | Conditions on open sets are equivalent to conditions on closed sets. (Contributed by Zhi Wang, 30-Aug-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ ((𝜑 ∧ 𝑥 = (∪ 𝐽 ∖ 𝑦)) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∀𝑥 ∈ 𝐽 𝜓 ↔ ∀𝑦 ∈ (Clsd‘𝐽)𝜒)) | ||
| Theorem | opndisj 48748 | Two ways of saying that two open sets are disjoint, if 𝐽 is a topology and 𝑋 is an open set. (Contributed by Zhi Wang, 6-Sep-2024.) |
| ⊢ (𝑍 = (∪ 𝐽 ∖ 𝑋) → (𝑌 ∈ (𝐽 ∩ 𝒫 𝑍) ↔ (𝑌 ∈ 𝐽 ∧ (𝑋 ∩ 𝑌) = ∅))) | ||
| Theorem | clddisj 48749 | Two ways of saying that two closed sets are disjoint, if 𝐽 is a topology and 𝑋 is a closed set. An alternative proof is similar to that of opndisj 48748 with elssuni 4919 replaced by the combination of cldss 23002 and eqid 2734. (Contributed by Zhi Wang, 6-Sep-2024.) |
| ⊢ (𝑍 = (∪ 𝐽 ∖ 𝑋) → (𝑌 ∈ ((Clsd‘𝐽) ∩ 𝒫 𝑍) ↔ (𝑌 ∈ (Clsd‘𝐽) ∧ (𝑋 ∩ 𝑌) = ∅))) | ||
| Theorem | neircl 48750 | Reverse closure of the neighborhood operation. (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 Zhi Wang, 16-Sep-2024.) |
| ⊢ (𝑁 ∈ ((nei‘𝐽)‘𝑆) → 𝐽 ∈ Top) | ||
| Theorem | opnneilem 48751* | Lemma factoring out common proof steps of opnneil 48755 and opnneirv 48753. (Contributed by Zhi Wang, 31-Aug-2024.) |
| ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ 𝐽 (𝑆 ⊆ 𝑥 ∧ 𝜓) ↔ ∃𝑦 ∈ 𝐽 (𝑆 ⊆ 𝑦 ∧ 𝜒))) | ||
| Theorem | opnneir 48752* | If something is true for an open neighborhood, it must be true for a neighborhood. (Contributed by Zhi Wang, 31-Aug-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ 𝐽 (𝑆 ⊆ 𝑥 ∧ 𝜓) → ∃𝑥 ∈ ((nei‘𝐽)‘𝑆)𝜓)) | ||
| Theorem | opnneirv 48753* | A variant of opnneir 48752 with different dummy variables. (Contributed by Zhi Wang, 31-Aug-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ 𝐽 (𝑆 ⊆ 𝑥 ∧ 𝜓) → ∃𝑦 ∈ ((nei‘𝐽)‘𝑆)𝜒)) | ||
| Theorem | opnneilv 48754* | The converse of opnneir 48752 with different dummy variables. Note that the second hypothesis could be generalized by adding 𝑦 ∈ 𝐽 to the antecedent. See the proof for details. Although 𝐽 ∈ Top might be redundant here (see neircl 48750), it is listed for explicitness. (Contributed by Zhi Wang, 31-Aug-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ ((𝜑 ∧ 𝑦 ⊆ 𝑥) → (𝜓 → 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ ((nei‘𝐽)‘𝑆)𝜓 → ∃𝑦 ∈ 𝐽 (𝑆 ⊆ 𝑦 ∧ 𝜒))) | ||
| Theorem | opnneil 48755* | A variant of opnneilv 48754. (Contributed by Zhi Wang, 31-Aug-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ ((𝜑 ∧ 𝑦 ⊆ 𝑥) → (𝜓 → 𝜒)) & ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ ((nei‘𝐽)‘𝑆)𝜓 → ∃𝑥 ∈ 𝐽 (𝑆 ⊆ 𝑥 ∧ 𝜓))) | ||
| Theorem | opnneieqv 48756* | The equivalence between neighborhood and open neighborhood. See opnneieqvv 48757 for different dummy variables. (Contributed by Zhi Wang, 31-Aug-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ ((𝜑 ∧ 𝑦 ⊆ 𝑥) → (𝜓 → 𝜒)) & ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ ((nei‘𝐽)‘𝑆)𝜓 ↔ ∃𝑥 ∈ 𝐽 (𝑆 ⊆ 𝑥 ∧ 𝜓))) | ||
| Theorem | opnneieqvv 48757* | The equivalence between neighborhood and open neighborhood. A variant of opnneieqv 48756 with two dummy variables. (Contributed by Zhi Wang, 31-Aug-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ ((𝜑 ∧ 𝑦 ⊆ 𝑥) → (𝜓 → 𝜒)) & ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ ((nei‘𝐽)‘𝑆)𝜓 ↔ ∃𝑦 ∈ 𝐽 (𝑆 ⊆ 𝑦 ∧ 𝜒))) | ||
| Theorem | restcls2lem 48758 | A closed set in a subspace topology is a subset of the subspace. (Contributed by Zhi Wang, 2-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑋 = ∪ 𝐽) & ⊢ (𝜑 → 𝑌 ⊆ 𝑋) & ⊢ (𝜑 → 𝐾 = (𝐽 ↾t 𝑌)) & ⊢ (𝜑 → 𝑆 ∈ (Clsd‘𝐾)) ⇒ ⊢ (𝜑 → 𝑆 ⊆ 𝑌) | ||
| Theorem | restcls2 48759 | A closed set in a subspace topology is the closure in the original topology intersecting with the subspace. (Contributed by Zhi Wang, 2-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑋 = ∪ 𝐽) & ⊢ (𝜑 → 𝑌 ⊆ 𝑋) & ⊢ (𝜑 → 𝐾 = (𝐽 ↾t 𝑌)) & ⊢ (𝜑 → 𝑆 ∈ (Clsd‘𝐾)) ⇒ ⊢ (𝜑 → 𝑆 = (((cls‘𝐽)‘𝑆) ∩ 𝑌)) | ||
| Theorem | restclsseplem 48760 | Lemma for restclssep 48761. (Contributed by Zhi Wang, 2-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑋 = ∪ 𝐽) & ⊢ (𝜑 → 𝑌 ⊆ 𝑋) & ⊢ (𝜑 → 𝐾 = (𝐽 ↾t 𝑌)) & ⊢ (𝜑 → 𝑆 ∈ (Clsd‘𝐾)) & ⊢ (𝜑 → (𝑆 ∩ 𝑇) = ∅) & ⊢ (𝜑 → 𝑇 ⊆ 𝑌) ⇒ ⊢ (𝜑 → (((cls‘𝐽)‘𝑆) ∩ 𝑇) = ∅) | ||
| Theorem | restclssep 48761 | Two disjoint closed sets in a subspace topology are separated in the original topology. (Contributed by Zhi Wang, 2-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑋 = ∪ 𝐽) & ⊢ (𝜑 → 𝑌 ⊆ 𝑋) & ⊢ (𝜑 → 𝐾 = (𝐽 ↾t 𝑌)) & ⊢ (𝜑 → 𝑆 ∈ (Clsd‘𝐾)) & ⊢ (𝜑 → (𝑆 ∩ 𝑇) = ∅) & ⊢ (𝜑 → 𝑇 ∈ (Clsd‘𝐾)) ⇒ ⊢ (𝜑 → ((𝑆 ∩ ((cls‘𝐽)‘𝑇)) = ∅ ∧ (((cls‘𝐽)‘𝑆) ∩ 𝑇) = ∅)) | ||
| Theorem | cnneiima 48762 | Given a continuous function, the preimage of a neighborhood is a neighborhood. To be precise, the preimage of a neighborhood of a subset 𝑇 of the codomain of a continuous function is a neighborhood of any subset of the preimage of 𝑇. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ (𝜑 → 𝐹 ∈ (𝐽 Cn 𝐾)) & ⊢ (𝜑 → 𝑁 ∈ ((nei‘𝐾)‘𝑇)) & ⊢ (𝜑 → 𝑆 ⊆ (◡𝐹 “ 𝑇)) ⇒ ⊢ (𝜑 → (◡𝐹 “ 𝑁) ∈ ((nei‘𝐽)‘𝑆)) | ||
| Theorem | iooii 48763 | Open intervals are open sets of II. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ ((0 ≤ 𝐴 ∧ 𝐵 ≤ 1) → (𝐴(,)𝐵) ∈ II) | ||
| Theorem | icccldii 48764 | Closed intervals are closed sets of II. Note that iccss 13438, iccordt 23187, and ordtresticc 23196 are proved from ixxss12 13390, ordtcld3 23172, and ordtrest2 23177, respectively. An alternate proof uses restcldi 23146, dfii2 24863, and icccld 24742. (Contributed by Zhi Wang, 8-Sep-2024.) |
| ⊢ ((0 ≤ 𝐴 ∧ 𝐵 ≤ 1) → (𝐴[,]𝐵) ∈ (Clsd‘II)) | ||
| Theorem | i0oii 48765 | (0[,)𝐴) is open in II. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ (𝐴 ≤ 1 → (0[,)𝐴) ∈ II) | ||
| Theorem | io1ii 48766 | (𝐴(,]1) is open in II. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ (0 ≤ 𝐴 → (𝐴(,]1) ∈ II) | ||
| Theorem | sepnsepolem1 48767* | Lemma for sepnsepo 48769. (Contributed by Zhi Wang, 1-Sep-2024.) |
| ⊢ (∃𝑥 ∈ 𝐽 ∃𝑦 ∈ 𝐽 (𝜑 ∧ 𝜓 ∧ 𝜒) ↔ ∃𝑥 ∈ 𝐽 (𝜑 ∧ ∃𝑦 ∈ 𝐽 (𝜓 ∧ 𝜒))) | ||
| Theorem | sepnsepolem2 48768* | Open neighborhood and neighborhood is equivalent regarding disjointness. Lemma for sepnsepo 48769. Proof could be shortened by 1 step using ssdisjdr 48674. (Contributed by Zhi Wang, 1-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) ⇒ ⊢ (𝜑 → (∃𝑦 ∈ ((nei‘𝐽)‘𝐷)(𝑥 ∩ 𝑦) = ∅ ↔ ∃𝑦 ∈ 𝐽 (𝐷 ⊆ 𝑦 ∧ (𝑥 ∩ 𝑦) = ∅))) | ||
| Theorem | sepnsepo 48769* | Open neighborhood and neighborhood is equivalent regarding disjointness for both sides. Namely, separatedness by open neighborhoods is equivalent to separatedness by neighborhoods. (Contributed by Zhi Wang, 1-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ ((nei‘𝐽)‘𝐶)∃𝑦 ∈ ((nei‘𝐽)‘𝐷)(𝑥 ∩ 𝑦) = ∅ ↔ ∃𝑥 ∈ 𝐽 ∃𝑦 ∈ 𝐽 (𝐶 ⊆ 𝑥 ∧ 𝐷 ⊆ 𝑦 ∧ (𝑥 ∩ 𝑦) = ∅))) | ||
| Theorem | sepdisj 48770 | Separated sets are disjoint. Note that in general separatedness also requires 𝑇 ⊆ ∪ 𝐽 and (𝑆 ∩ ((cls‘𝐽)‘𝑇)) = ∅ as well but they are unnecessary here. (Contributed by Zhi Wang, 7-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑆 ⊆ ∪ 𝐽) & ⊢ (𝜑 → (((cls‘𝐽)‘𝑆) ∩ 𝑇) = ∅) ⇒ ⊢ (𝜑 → (𝑆 ∩ 𝑇) = ∅) | ||
| Theorem | seposep 48771* | If two sets are separated by (open) neighborhoods, then they are separated subsets of the underlying set. Note that separatedness by open neighborhoods is equivalent to separatedness by neighborhoods. See sepnsepo 48769. The relationship between separatedness and closure is also seen in isnrm 23308, isnrm2 23331, isnrm3 23332. (Contributed by Zhi Wang, 7-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → ∃𝑛 ∈ 𝐽 ∃𝑚 ∈ 𝐽 (𝑆 ⊆ 𝑛 ∧ 𝑇 ⊆ 𝑚 ∧ (𝑛 ∩ 𝑚) = ∅)) ⇒ ⊢ (𝜑 → ((𝑆 ⊆ ∪ 𝐽 ∧ 𝑇 ⊆ ∪ 𝐽) ∧ ((𝑆 ∩ ((cls‘𝐽)‘𝑇)) = ∅ ∧ (((cls‘𝐽)‘𝑆) ∩ 𝑇) = ∅))) | ||
| Theorem | sepcsepo 48772* | If two sets are separated by closed neighborhoods, then they are separated by (open) neighborhoods. See sepnsepo 48769 for the equivalence between separatedness by open neighborhoods and separatedness by neighborhoods. Although 𝐽 ∈ Top might be redundant here, it is listed for explicitness. 𝐽 ∈ Top can be obtained from neircl 48750, adantr 480, and rexlimiva 3134. (Contributed by Zhi Wang, 8-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → ∃𝑛 ∈ ((nei‘𝐽)‘𝑆)∃𝑚 ∈ ((nei‘𝐽)‘𝑇)(𝑛 ∈ (Clsd‘𝐽) ∧ 𝑚 ∈ (Clsd‘𝐽) ∧ (𝑛 ∩ 𝑚) = ∅)) ⇒ ⊢ (𝜑 → ∃𝑛 ∈ 𝐽 ∃𝑚 ∈ 𝐽 (𝑆 ⊆ 𝑛 ∧ 𝑇 ⊆ 𝑚 ∧ (𝑛 ∩ 𝑚) = ∅)) | ||
| Theorem | sepfsepc 48773* | If two sets are separated by a continuous function, then they are separated by closed neighborhoods. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ (𝜑 → ∃𝑓 ∈ (𝐽 Cn II)(𝑆 ⊆ (◡𝑓 “ {0}) ∧ 𝑇 ⊆ (◡𝑓 “ {1}))) ⇒ ⊢ (𝜑 → ∃𝑛 ∈ ((nei‘𝐽)‘𝑆)∃𝑚 ∈ ((nei‘𝐽)‘𝑇)(𝑛 ∈ (Clsd‘𝐽) ∧ 𝑚 ∈ (Clsd‘𝐽) ∧ (𝑛 ∩ 𝑚) = ∅)) | ||
| Theorem | seppsepf 48774 | If two sets are precisely separated by a continuous function, then they are separated by the continuous function. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ (𝜑 → ∃𝑓 ∈ (𝐽 Cn II)(𝑆 = (◡𝑓 “ {0}) ∧ 𝑇 = (◡𝑓 “ {1}))) ⇒ ⊢ (𝜑 → ∃𝑓 ∈ (𝐽 Cn II)(𝑆 ⊆ (◡𝑓 “ {0}) ∧ 𝑇 ⊆ (◡𝑓 “ {1}))) | ||
| Theorem | seppcld 48775* | If two sets are precisely separated by a continuous function, then they are closed. An alternate proof involves II ∈ Fre. (Contributed by Zhi Wang, 9-Sep-2024.) |
| ⊢ (𝜑 → ∃𝑓 ∈ (𝐽 Cn II)(𝑆 = (◡𝑓 “ {0}) ∧ 𝑇 = (◡𝑓 “ {1}))) ⇒ ⊢ (𝜑 → (𝑆 ∈ (Clsd‘𝐽) ∧ 𝑇 ∈ (Clsd‘𝐽))) | ||
| Theorem | isnrm4 48776* | A topological space is normal iff any two disjoint closed sets are separated by neighborhoods. (Contributed by Zhi Wang, 1-Sep-2024.) |
| ⊢ (𝐽 ∈ Nrm ↔ (𝐽 ∈ Top ∧ ∀𝑐 ∈ (Clsd‘𝐽)∀𝑑 ∈ (Clsd‘𝐽)((𝑐 ∩ 𝑑) = ∅ → ∃𝑥 ∈ ((nei‘𝐽)‘𝑐)∃𝑦 ∈ ((nei‘𝐽)‘𝑑)(𝑥 ∩ 𝑦) = ∅))) | ||
| Theorem | dfnrm2 48777* | A topological space is normal if any disjoint closed sets can be separated by open neighborhoods. An alternate definition of df-nrm 23290. (Contributed by Zhi Wang, 30-Aug-2024.) |
| ⊢ Nrm = {𝑗 ∈ Top ∣ ∀𝑐 ∈ (Clsd‘𝑗)∀𝑑 ∈ (Clsd‘𝑗)((𝑐 ∩ 𝑑) = ∅ → ∃𝑥 ∈ 𝑗 ∃𝑦 ∈ 𝑗 (𝑐 ⊆ 𝑥 ∧ 𝑑 ⊆ 𝑦 ∧ (𝑥 ∩ 𝑦) = ∅))} | ||
| Theorem | dfnrm3 48778* | A topological space is normal if any disjoint closed sets can be separated by neighborhoods. An alternate definition of df-nrm 23290. (Contributed by Zhi Wang, 2-Sep-2024.) |
| ⊢ Nrm = {𝑗 ∈ Top ∣ ∀𝑐 ∈ (Clsd‘𝑗)∀𝑑 ∈ (Clsd‘𝑗)((𝑐 ∩ 𝑑) = ∅ → ∃𝑥 ∈ ((nei‘𝑗)‘𝑐)∃𝑦 ∈ ((nei‘𝑗)‘𝑑)(𝑥 ∩ 𝑦) = ∅)} | ||
| Theorem | iscnrm3lem1 48779* | Lemma for iscnrm3 48797. Subspace topology is a topology. (Contributed by Zhi Wang, 3-Sep-2024.) |
| ⊢ (𝐽 ∈ Top → (∀𝑥 ∈ 𝐴 𝜑 ↔ ∀𝑥 ∈ 𝐴 ((𝐽 ↾t 𝑥) ∈ Top ∧ 𝜑))) | ||
| Theorem | iscnrm3lem2 48780* | Lemma for iscnrm3 48797 proving a biconditional on restricted universal quantifications. (Contributed by Zhi Wang, 3-Sep-2024.) |
| ⊢ (𝜑 → (∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 ∀𝑧 ∈ 𝐶 𝜓 → ((𝑤 ∈ 𝐷 ∧ 𝑣 ∈ 𝐸) → 𝜒))) & ⊢ (𝜑 → (∀𝑤 ∈ 𝐷 ∀𝑣 ∈ 𝐸 𝜒 → ((𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵 ∧ 𝑧 ∈ 𝐶) → 𝜓))) ⇒ ⊢ (𝜑 → (∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 ∀𝑧 ∈ 𝐶 𝜓 ↔ ∀𝑤 ∈ 𝐷 ∀𝑣 ∈ 𝐸 𝜒)) | ||
| Theorem | iscnrm3lem4 48781 | Lemma for iscnrm3lem5 48782 and iscnrm3r 48793. (Contributed by Zhi Wang, 4-Sep-2024.) |
| ⊢ (𝜂 → (𝜓 → 𝜁)) & ⊢ ((𝜑 ∧ 𝜒 ∧ 𝜃) → 𝜂) & ⊢ ((𝜑 ∧ 𝜒 ∧ 𝜃) → (𝜁 → 𝜏)) ⇒ ⊢ (𝜑 → (𝜓 → (𝜒 → (𝜃 → 𝜏)))) | ||
| Theorem | iscnrm3lem5 48782* | Lemma for iscnrm3l 48796. (Contributed by Zhi Wang, 3-Sep-2024.) |
| ⊢ ((𝑥 = 𝑆 ∧ 𝑦 = 𝑇) → (𝜑 ↔ 𝜓)) & ⊢ ((𝑥 = 𝑆 ∧ 𝑦 = 𝑇) → (𝜒 ↔ 𝜃)) & ⊢ ((𝜏 ∧ 𝜂 ∧ 𝜁) → (𝑆 ∈ 𝑉 ∧ 𝑇 ∈ 𝑊)) & ⊢ ((𝜏 ∧ 𝜂 ∧ 𝜁) → ((𝜓 → 𝜃) → 𝜎)) ⇒ ⊢ (𝜏 → (∀𝑥 ∈ 𝑉 ∀𝑦 ∈ 𝑊 (𝜑 → 𝜒) → (𝜂 → (𝜁 → 𝜎)))) | ||
| Theorem | iscnrm3lem6 48783* | Lemma for iscnrm3lem7 48784. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑉 ∧ 𝑦 ∈ 𝑊) ∧ 𝜓) → 𝜒) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ 𝑉 ∃𝑦 ∈ 𝑊 𝜓 → 𝜒)) | ||
| Theorem | iscnrm3lem7 48784* | Lemma for iscnrm3rlem8 48792 and iscnrm3llem2 48795 involving restricted existential quantifications. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝑧 = 𝑍 → (𝜒 ↔ 𝜃)) & ⊢ (𝑤 = 𝑊 → (𝜃 ↔ 𝜏)) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵) ∧ 𝜓) → (𝑍 ∈ 𝐶 ∧ 𝑊 ∈ 𝐷 ∧ 𝜏)) ⇒ ⊢ (𝜑 → (∃𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝜓 → ∃𝑧 ∈ 𝐶 ∃𝑤 ∈ 𝐷 𝜒)) | ||
| Theorem | iscnrm3rlem1 48785 | Lemma for iscnrm3rlem2 48786. The hypothesis could be generalized to (𝜑 → (𝑆 ∖ 𝑇) ⊆ 𝑋). (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝜑 → 𝑆 ⊆ 𝑋) ⇒ ⊢ (𝜑 → (𝑆 ∖ 𝑇) = (𝑆 ∩ (𝑋 ∖ (𝑆 ∩ 𝑇)))) | ||
| Theorem | iscnrm3rlem2 48786 | Lemma for iscnrm3rlem3 48787. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑆 ⊆ ∪ 𝐽) ⇒ ⊢ (𝜑 → (((cls‘𝐽)‘𝑆) ∖ 𝑇) ∈ (Clsd‘(𝐽 ↾t (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ 𝑇))))) | ||
| Theorem | iscnrm3rlem3 48787 | Lemma for iscnrm3r 48793. The designed subspace is a subset of the original set; the two sets are closed sets in the subspace. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ ((𝐽 ∈ Top ∧ (𝑆 ∈ 𝒫 ∪ 𝐽 ∧ 𝑇 ∈ 𝒫 ∪ 𝐽)) → ((∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇))) ∈ 𝒫 ∪ 𝐽 ∧ (((cls‘𝐽)‘𝑆) ∖ ((cls‘𝐽)‘𝑇)) ∈ (Clsd‘(𝐽 ↾t (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇))))) ∧ (((cls‘𝐽)‘𝑇) ∖ ((cls‘𝐽)‘𝑆)) ∈ (Clsd‘(𝐽 ↾t (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇))))))) | ||
| Theorem | iscnrm3rlem4 48788 | Lemma for iscnrm3rlem8 48792. Given two disjoint subsets 𝑆 and 𝑇 of the underlying set of a topology 𝐽, if 𝑁 is a superset of (((cls‘𝐽)‘𝑆) ∖ 𝑇), then it is a superset of 𝑆. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑆 ⊆ ∪ 𝐽) & ⊢ (𝜑 → (𝑆 ∩ 𝑇) = ∅) & ⊢ (𝜑 → (((cls‘𝐽)‘𝑆) ∖ 𝑇) ⊆ 𝑁) ⇒ ⊢ (𝜑 → 𝑆 ⊆ 𝑁) | ||
| Theorem | iscnrm3rlem5 48789 | Lemma for iscnrm3rlem6 48790. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑆 ⊆ ∪ 𝐽) & ⊢ (𝜑 → 𝑇 ⊆ ∪ 𝐽) ⇒ ⊢ (𝜑 → (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇))) ∈ 𝐽) | ||
| Theorem | iscnrm3rlem6 48790 | Lemma for iscnrm3rlem7 48791. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑆 ⊆ ∪ 𝐽) & ⊢ (𝜑 → 𝑇 ⊆ ∪ 𝐽) & ⊢ (𝜑 → 𝑂 ⊆ (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇)))) ⇒ ⊢ (𝜑 → (𝑂 ∈ (𝐽 ↾t (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇)))) ↔ 𝑂 ∈ 𝐽)) | ||
| Theorem | iscnrm3rlem7 48791 | Lemma for iscnrm3rlem8 48792. Open neighborhoods in the subspace topology are open neighborhoods in the original topology given that the subspace is an open set in the original topology. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝜑 → 𝐽 ∈ Top) & ⊢ (𝜑 → 𝑆 ⊆ ∪ 𝐽) & ⊢ (𝜑 → 𝑇 ⊆ ∪ 𝐽) & ⊢ (𝜑 → 𝑂 ∈ (𝐽 ↾t (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇))))) ⇒ ⊢ (𝜑 → 𝑂 ∈ 𝐽) | ||
| Theorem | iscnrm3rlem8 48792* | Lemma for iscnrm3r 48793. Disjoint open neighborhoods in the subspace topology are disjoint open neighborhoods in the original topology given that the subspace is an open set in the original topology. Therefore, given any two sets separated in the original topology and separated by open neighborhoods in the subspace topology, they must be separated by open neighborhoods in the original topology. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ ((𝐽 ∈ Top ∧ (𝑆 ∈ 𝒫 ∪ 𝐽 ∧ 𝑇 ∈ 𝒫 ∪ 𝐽) ∧ ((𝑆 ∩ ((cls‘𝐽)‘𝑇)) = ∅ ∧ (((cls‘𝐽)‘𝑆) ∩ 𝑇) = ∅)) → (∃𝑙 ∈ (𝐽 ↾t (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇))))∃𝑘 ∈ (𝐽 ↾t (∪ 𝐽 ∖ (((cls‘𝐽)‘𝑆) ∩ ((cls‘𝐽)‘𝑇))))((((cls‘𝐽)‘𝑆) ∖ ((cls‘𝐽)‘𝑇)) ⊆ 𝑙 ∧ (((cls‘𝐽)‘𝑇) ∖ ((cls‘𝐽)‘𝑆)) ⊆ 𝑘 ∧ (𝑙 ∩ 𝑘) = ∅) → ∃𝑛 ∈ 𝐽 ∃𝑚 ∈ 𝐽 (𝑆 ⊆ 𝑛 ∧ 𝑇 ⊆ 𝑚 ∧ (𝑛 ∩ 𝑚) = ∅))) | ||
| Theorem | iscnrm3r 48793* | Lemma for iscnrm3 48797. If all subspaces of a topology are normal, i.e., two disjoint closed sets can be separated by open neighborhoods, then in the original topology two separated sets can be separated by open neighborhoods. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝐽 ∈ Top → (∀𝑧 ∈ 𝒫 ∪ 𝐽∀𝑐 ∈ (Clsd‘(𝐽 ↾t 𝑧))∀𝑑 ∈ (Clsd‘(𝐽 ↾t 𝑧))((𝑐 ∩ 𝑑) = ∅ → ∃𝑙 ∈ (𝐽 ↾t 𝑧)∃𝑘 ∈ (𝐽 ↾t 𝑧)(𝑐 ⊆ 𝑙 ∧ 𝑑 ⊆ 𝑘 ∧ (𝑙 ∩ 𝑘) = ∅)) → ((𝑆 ∈ 𝒫 ∪ 𝐽 ∧ 𝑇 ∈ 𝒫 ∪ 𝐽) → (((𝑆 ∩ ((cls‘𝐽)‘𝑇)) = ∅ ∧ (((cls‘𝐽)‘𝑆) ∩ 𝑇) = ∅) → ∃𝑛 ∈ 𝐽 ∃𝑚 ∈ 𝐽 (𝑆 ⊆ 𝑛 ∧ 𝑇 ⊆ 𝑚 ∧ (𝑛 ∩ 𝑚) = ∅))))) | ||
| Theorem | iscnrm3llem1 48794 | Lemma for iscnrm3l 48796. Closed sets in the subspace are subsets of the underlying set of the original topology. (Contributed by Zhi Wang, 4-Sep-2024.) |
| ⊢ ((𝐽 ∈ Top ∧ (𝑍 ∈ 𝒫 ∪ 𝐽 ∧ 𝐶 ∈ (Clsd‘(𝐽 ↾t 𝑍)) ∧ 𝐷 ∈ (Clsd‘(𝐽 ↾t 𝑍))) ∧ (𝐶 ∩ 𝐷) = ∅) → (𝐶 ∈ 𝒫 ∪ 𝐽 ∧ 𝐷 ∈ 𝒫 ∪ 𝐽)) | ||
| Theorem | iscnrm3llem2 48795* | Lemma for iscnrm3l 48796. If there exist disjoint open neighborhoods in the original topology for two disjoint closed sets in a subspace, then they can be separated by open neighborhoods in the subspace topology. (Could shorten proof with ssin0 45005.) (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ ((𝐽 ∈ Top ∧ (𝑍 ∈ 𝒫 ∪ 𝐽 ∧ 𝐶 ∈ (Clsd‘(𝐽 ↾t 𝑍)) ∧ 𝐷 ∈ (Clsd‘(𝐽 ↾t 𝑍))) ∧ (𝐶 ∩ 𝐷) = ∅) → (∃𝑛 ∈ 𝐽 ∃𝑚 ∈ 𝐽 (𝐶 ⊆ 𝑛 ∧ 𝐷 ⊆ 𝑚 ∧ (𝑛 ∩ 𝑚) = ∅) → ∃𝑙 ∈ (𝐽 ↾t 𝑍)∃𝑘 ∈ (𝐽 ↾t 𝑍)(𝐶 ⊆ 𝑙 ∧ 𝐷 ⊆ 𝑘 ∧ (𝑙 ∩ 𝑘) = ∅))) | ||
| Theorem | iscnrm3l 48796* | Lemma for iscnrm3 48797. Given a topology 𝐽, if two separated sets can be separated by open neighborhoods, then all subspaces of the topology 𝐽 are normal, i.e., two disjoint closed sets can be separated by open neighborhoods. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝐽 ∈ Top → (∀𝑠 ∈ 𝒫 ∪ 𝐽∀𝑡 ∈ 𝒫 ∪ 𝐽(((𝑠 ∩ ((cls‘𝐽)‘𝑡)) = ∅ ∧ (((cls‘𝐽)‘𝑠) ∩ 𝑡) = ∅) → ∃𝑛 ∈ 𝐽 ∃𝑚 ∈ 𝐽 (𝑠 ⊆ 𝑛 ∧ 𝑡 ⊆ 𝑚 ∧ (𝑛 ∩ 𝑚) = ∅)) → ((𝑍 ∈ 𝒫 ∪ 𝐽 ∧ 𝐶 ∈ (Clsd‘(𝐽 ↾t 𝑍)) ∧ 𝐷 ∈ (Clsd‘(𝐽 ↾t 𝑍))) → ((𝐶 ∩ 𝐷) = ∅ → ∃𝑙 ∈ (𝐽 ↾t 𝑍)∃𝑘 ∈ (𝐽 ↾t 𝑍)(𝐶 ⊆ 𝑙 ∧ 𝐷 ⊆ 𝑘 ∧ (𝑙 ∩ 𝑘) = ∅))))) | ||
| Theorem | iscnrm3 48797* | A completely normal topology is a topology in which two separated sets can be separated by open neighborhoods. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝐽 ∈ CNrm ↔ (𝐽 ∈ Top ∧ ∀𝑠 ∈ 𝒫 ∪ 𝐽∀𝑡 ∈ 𝒫 ∪ 𝐽(((𝑠 ∩ ((cls‘𝐽)‘𝑡)) = ∅ ∧ (((cls‘𝐽)‘𝑠) ∩ 𝑡) = ∅) → ∃𝑛 ∈ 𝐽 ∃𝑚 ∈ 𝐽 (𝑠 ⊆ 𝑛 ∧ 𝑡 ⊆ 𝑚 ∧ (𝑛 ∩ 𝑚) = ∅)))) | ||
| Theorem | iscnrm3v 48798* | A topology is completely normal iff two separated sets can be separated by open neighborhoods. (Contributed by Zhi Wang, 10-Sep-2024.) |
| ⊢ (𝐽 ∈ Top → (𝐽 ∈ CNrm ↔ ∀𝑠 ∈ 𝒫 ∪ 𝐽∀𝑡 ∈ 𝒫 ∪ 𝐽(((𝑠 ∩ ((cls‘𝐽)‘𝑡)) = ∅ ∧ (((cls‘𝐽)‘𝑠) ∩ 𝑡) = ∅) → ∃𝑛 ∈ 𝐽 ∃𝑚 ∈ 𝐽 (𝑠 ⊆ 𝑛 ∧ 𝑡 ⊆ 𝑚 ∧ (𝑛 ∩ 𝑚) = ∅)))) | ||
| Theorem | iscnrm4 48799* | A completely normal topology is a topology in which two separated sets can be separated by neighborhoods. (Contributed by Zhi Wang, 5-Sep-2024.) |
| ⊢ (𝐽 ∈ CNrm ↔ (𝐽 ∈ Top ∧ ∀𝑠 ∈ 𝒫 ∪ 𝐽∀𝑡 ∈ 𝒫 ∪ 𝐽(((𝑠 ∩ ((cls‘𝐽)‘𝑡)) = ∅ ∧ (((cls‘𝐽)‘𝑠) ∩ 𝑡) = ∅) → ∃𝑛 ∈ ((nei‘𝐽)‘𝑠)∃𝑚 ∈ ((nei‘𝐽)‘𝑡)(𝑛 ∩ 𝑚) = ∅))) | ||
| Theorem | isprsd 48800* | Property of being a preordered set (deduction form). (Contributed by Zhi Wang, 18-Sep-2024.) |
| ⊢ (𝜑 → 𝐵 = (Base‘𝐾)) & ⊢ (𝜑 → ≤ = (le‘𝐾)) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) ⇒ ⊢ (𝜑 → (𝐾 ∈ Proset ↔ ∀𝑥 ∈ 𝐵 ∀𝑦 ∈ 𝐵 ∀𝑧 ∈ 𝐵 (𝑥 ≤ 𝑥 ∧ ((𝑥 ≤ 𝑦 ∧ 𝑦 ≤ 𝑧) → 𝑥 ≤ 𝑧)))) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |