HomeHome Intuitionistic Logic Explorer
Theorem List (p. 132 of 145)
< Previous  Next >
Bad symbols? Try the
GIF version.

Mirrors  >  Metamath Home Page  >  ILE Home Page  >  Theorem List Contents  >  Recent Proofs       This page: Page List

Theorem List for Intuitionistic Logic Explorer - 13101-13200   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theorem1unit 13101 The multiplicative identity is a unit. (Contributed by Mario Carneiro, 1-Dec-2014.)
𝑈 = (Unit‘𝑅)    &    1 = (1r𝑅)       (𝑅 ∈ Ring → 1𝑈)
 
Theoremunitcld 13102 A unit is an element of the base set. (Contributed by Mario Carneiro, 1-Dec-2014.)
(𝜑𝐵 = (Base‘𝑅))    &   (𝜑𝑈 = (Unit‘𝑅))    &   (𝜑𝑅 ∈ SRing)    &   (𝜑𝑋𝑈)       (𝜑𝑋𝐵)
 
Theoremunitssd 13103 The set of units is contained in the base set. (Contributed by Mario Carneiro, 5-Oct-2015.)
(𝜑𝐵 = (Base‘𝑅))    &   (𝜑𝑈 = (Unit‘𝑅))    &   (𝜑𝑅 ∈ SRing)       (𝜑𝑈𝐵)
 
Theoremopprunitd 13104 Being a unit is a symmetric property, so it transfers to the opposite ring. (Contributed by Mario Carneiro, 4-Dec-2014.)
(𝜑𝑈 = (Unit‘𝑅))    &   (𝜑𝑆 = (oppr𝑅))    &   (𝜑𝑅 ∈ Ring)       (𝜑𝑈 = (Unit‘𝑆))
 
Theoremcrngunit 13105 Property of being a unit in a commutative ring. (Contributed by Mario Carneiro, 18-Apr-2016.)
𝑈 = (Unit‘𝑅)    &    1 = (1r𝑅)    &    = (∥r𝑅)       (𝑅 ∈ CRing → (𝑋𝑈𝑋 1 ))
 
Theoremdvdsunit 13106 A divisor of a unit is a unit. (Contributed by Mario Carneiro, 18-Apr-2016.)
𝑈 = (Unit‘𝑅)    &    = (∥r𝑅)       ((𝑅 ∈ CRing ∧ 𝑌 𝑋𝑋𝑈) → 𝑌𝑈)
 
Theoremunitmulcl 13107 The product of units is a unit. (Contributed by Mario Carneiro, 2-Dec-2014.)
𝑈 = (Unit‘𝑅)    &    · = (.r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈𝑌𝑈) → (𝑋 · 𝑌) ∈ 𝑈)
 
Theoremunitmulclb 13108 Reversal of unitmulcl 13107 in a commutative ring. (Contributed by Mario Carneiro, 18-Apr-2016.)
𝑈 = (Unit‘𝑅)    &    · = (.r𝑅)    &   𝐵 = (Base‘𝑅)       ((𝑅 ∈ CRing ∧ 𝑋𝐵𝑌𝐵) → ((𝑋 · 𝑌) ∈ 𝑈 ↔ (𝑋𝑈𝑌𝑈)))
 
Theoremunitgrpbasd 13109 The base set of the group of units. (Contributed by Mario Carneiro, 25-Dec-2014.)
(𝜑𝑈 = (Unit‘𝑅))    &   (𝜑𝐺 = ((mulGrp‘𝑅) ↾s 𝑈))    &   (𝜑𝑅 ∈ SRing)       (𝜑𝑈 = (Base‘𝐺))
 
Theoremunitgrp 13110 The group of units is a group under multiplication. (Contributed by Mario Carneiro, 2-Dec-2014.)
𝑈 = (Unit‘𝑅)    &   𝐺 = ((mulGrp‘𝑅) ↾s 𝑈)       (𝑅 ∈ Ring → 𝐺 ∈ Grp)
 
Theoremunitabl 13111 The group of units of a commutative ring is abelian. (Contributed by Mario Carneiro, 19-Apr-2016.)
𝑈 = (Unit‘𝑅)    &   𝐺 = ((mulGrp‘𝑅) ↾s 𝑈)       (𝑅 ∈ CRing → 𝐺 ∈ Abel)
 
Theoremunitgrpid 13112 The identity of the group of units of a ring is the ring unity. (Contributed by Mario Carneiro, 2-Dec-2014.)
𝑈 = (Unit‘𝑅)    &   𝐺 = ((mulGrp‘𝑅) ↾s 𝑈)    &    1 = (1r𝑅)       (𝑅 ∈ Ring → 1 = (0g𝐺))
 
Theoremunitsubm 13113 The group of units is a submonoid of the multiplicative monoid of the ring. (Contributed by Mario Carneiro, 18-Jun-2015.)
𝑈 = (Unit‘𝑅)    &   𝑀 = (mulGrp‘𝑅)       (𝑅 ∈ Ring → 𝑈 ∈ (SubMnd‘𝑀))
 
Syntaxcinvr 13114 Extend class notation with multiplicative inverse.
class invr
 
Definitiondf-invr 13115 Define multiplicative inverse. (Contributed by NM, 21-Sep-2011.)
invr = (𝑟 ∈ V ↦ (invg‘((mulGrp‘𝑟) ↾s (Unit‘𝑟))))
 
Theoreminvrfvald 13116 Multiplicative inverse function for a ring. (Contributed by NM, 21-Sep-2011.) (Revised by Mario Carneiro, 25-Dec-2014.)
(𝜑𝑈 = (Unit‘𝑅))    &   (𝜑𝐺 = ((mulGrp‘𝑅) ↾s 𝑈))    &   (𝜑𝐼 = (invr𝑅))    &   (𝜑𝑅 ∈ Ring)       (𝜑𝐼 = (invg𝐺))
 
Theoremunitinvcl 13117 The inverse of a unit exists and is a unit. (Contributed by Mario Carneiro, 2-Dec-2014.)
𝑈 = (Unit‘𝑅)    &   𝐼 = (invr𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈) → (𝐼𝑋) ∈ 𝑈)
 
Theoremunitinvinv 13118 The inverse of the inverse of a unit is the same element. (Contributed by Mario Carneiro, 4-Dec-2014.)
𝑈 = (Unit‘𝑅)    &   𝐼 = (invr𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈) → (𝐼‘(𝐼𝑋)) = 𝑋)
 
Theoremringinvcl 13119 The inverse of a unit is an element of the ring. (Contributed by Mario Carneiro, 2-Dec-2014.)
𝑈 = (Unit‘𝑅)    &   𝐼 = (invr𝑅)    &   𝐵 = (Base‘𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈) → (𝐼𝑋) ∈ 𝐵)
 
Theoremunitlinv 13120 A unit times its inverse is the ring unity. (Contributed by Mario Carneiro, 2-Dec-2014.)
𝑈 = (Unit‘𝑅)    &   𝐼 = (invr𝑅)    &    · = (.r𝑅)    &    1 = (1r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈) → ((𝐼𝑋) · 𝑋) = 1 )
 
Theoremunitrinv 13121 A unit times its inverse is the ring unity. (Contributed by Mario Carneiro, 2-Dec-2014.)
𝑈 = (Unit‘𝑅)    &   𝐼 = (invr𝑅)    &    · = (.r𝑅)    &    1 = (1r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈) → (𝑋 · (𝐼𝑋)) = 1 )
 
Theorem1rinv 13122 The inverse of the ring unity is the ring unity. (Contributed by Mario Carneiro, 18-Jun-2015.)
𝐼 = (invr𝑅)    &    1 = (1r𝑅)       (𝑅 ∈ Ring → (𝐼1 ) = 1 )
 
Theorem0unit 13123 The additive identity is a unit if and only if 1 = 0, i.e. we are in the zero ring. (Contributed by Mario Carneiro, 4-Dec-2014.)
𝑈 = (Unit‘𝑅)    &    0 = (0g𝑅)    &    1 = (1r𝑅)       (𝑅 ∈ Ring → ( 0𝑈1 = 0 ))
 
Theoremunitnegcl 13124 The negative of a unit is a unit. (Contributed by Mario Carneiro, 4-Dec-2014.)
𝑈 = (Unit‘𝑅)    &   𝑁 = (invg𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈) → (𝑁𝑋) ∈ 𝑈)
 
Syntaxcdvr 13125 Extend class notation with ring division.
class /r
 
Definitiondf-dvr 13126* Define ring division. (Contributed by Mario Carneiro, 2-Jul-2014.)
/r = (𝑟 ∈ V ↦ (𝑥 ∈ (Base‘𝑟), 𝑦 ∈ (Unit‘𝑟) ↦ (𝑥(.r𝑟)((invr𝑟)‘𝑦))))
 
Theoremdvrfvald 13127* Division operation in a ring. (Contributed by Mario Carneiro, 2-Jul-2014.) (Revised by Mario Carneiro, 2-Dec-2014.) (Proof shortened by AV, 2-Mar-2024.)
(𝜑𝐵 = (Base‘𝑅))    &   (𝜑· = (.r𝑅))    &   (𝜑𝑈 = (Unit‘𝑅))    &   (𝜑𝐼 = (invr𝑅))    &   (𝜑/ = (/r𝑅))    &   (𝜑𝑅 ∈ SRing)       (𝜑/ = (𝑥𝐵, 𝑦𝑈 ↦ (𝑥 · (𝐼𝑦))))
 
Theoremdvrvald 13128 Division operation in a ring. (Contributed by Mario Carneiro, 2-Jul-2014.) (Revised by Mario Carneiro, 2-Dec-2014.)
(𝜑𝐵 = (Base‘𝑅))    &   (𝜑· = (.r𝑅))    &   (𝜑𝑈 = (Unit‘𝑅))    &   (𝜑𝐼 = (invr𝑅))    &   (𝜑/ = (/r𝑅))    &   (𝜑𝑅 ∈ Ring)    &   (𝜑𝑋𝐵)    &   (𝜑𝑌𝑈)       (𝜑 → (𝑋 / 𝑌) = (𝑋 · (𝐼𝑌)))
 
Theoremdvrcl 13129 Closure of division operation. (Contributed by Mario Carneiro, 2-Jul-2014.)
𝐵 = (Base‘𝑅)    &   𝑈 = (Unit‘𝑅)    &    / = (/r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝐵𝑌𝑈) → (𝑋 / 𝑌) ∈ 𝐵)
 
Theoremunitdvcl 13130 The units are closed under division. (Contributed by Mario Carneiro, 2-Jul-2014.)
𝑈 = (Unit‘𝑅)    &    / = (/r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈𝑌𝑈) → (𝑋 / 𝑌) ∈ 𝑈)
 
Theoremdvrid 13131 A ring element divided by itself is the ring unity. (dividap 8647 analog.) (Contributed by Mario Carneiro, 18-Jun-2015.)
𝑈 = (Unit‘𝑅)    &    / = (/r𝑅)    &    1 = (1r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈) → (𝑋 / 𝑋) = 1 )
 
Theoremdvr1 13132 A ring element divided by the ring unity is itself. (div1 8649 analog.) (Contributed by Mario Carneiro, 18-Jun-2015.)
𝐵 = (Base‘𝑅)    &    / = (/r𝑅)    &    1 = (1r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝐵) → (𝑋 / 1 ) = 𝑋)
 
Theoremdvrass 13133 An associative law for division. (divassap 8636 analog.) (Contributed by Mario Carneiro, 4-Dec-2014.)
𝐵 = (Base‘𝑅)    &   𝑈 = (Unit‘𝑅)    &    / = (/r𝑅)    &    · = (.r𝑅)       ((𝑅 ∈ Ring ∧ (𝑋𝐵𝑌𝐵𝑍𝑈)) → ((𝑋 · 𝑌) / 𝑍) = (𝑋 · (𝑌 / 𝑍)))
 
Theoremdvrcan1 13134 A cancellation law for division. (divcanap1 8627 analog.) (Contributed by Mario Carneiro, 2-Jul-2014.) (Revised by Mario Carneiro, 2-Dec-2014.)
𝐵 = (Base‘𝑅)    &   𝑈 = (Unit‘𝑅)    &    / = (/r𝑅)    &    · = (.r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝐵𝑌𝑈) → ((𝑋 / 𝑌) · 𝑌) = 𝑋)
 
Theoremdvrcan3 13135 A cancellation law for division. (divcanap3 8644 analog.) (Contributed by Mario Carneiro, 2-Jul-2014.) (Revised by Mario Carneiro, 18-Jun-2015.)
𝐵 = (Base‘𝑅)    &   𝑈 = (Unit‘𝑅)    &    / = (/r𝑅)    &    · = (.r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝐵𝑌𝑈) → ((𝑋 · 𝑌) / 𝑌) = 𝑋)
 
Theoremdvreq1 13136 Equality in terms of ratio equal to ring unity. (diveqap1 8651 analog.) (Contributed by Mario Carneiro, 28-Apr-2016.)
𝐵 = (Base‘𝑅)    &   𝑈 = (Unit‘𝑅)    &    / = (/r𝑅)    &    1 = (1r𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝐵𝑌𝑈) → ((𝑋 / 𝑌) = 1𝑋 = 𝑌))
 
Theoremringinvdv 13137 Write the inverse function in terms of division. (Contributed by Mario Carneiro, 2-Jul-2014.)
𝐵 = (Base‘𝑅)    &   𝑈 = (Unit‘𝑅)    &    / = (/r𝑅)    &    1 = (1r𝑅)    &   𝐼 = (invr𝑅)       ((𝑅 ∈ Ring ∧ 𝑋𝑈) → (𝐼𝑋) = ( 1 / 𝑋))
 
Theoremrngidpropdg 13138* The ring unity depends only on the ring's base set and multiplication operation. (Contributed by Mario Carneiro, 26-Dec-2014.)
(𝜑𝐵 = (Base‘𝐾))    &   (𝜑𝐵 = (Base‘𝐿))    &   ((𝜑 ∧ (𝑥𝐵𝑦𝐵)) → (𝑥(.r𝐾)𝑦) = (𝑥(.r𝐿)𝑦))    &   (𝜑𝐾𝑉)    &   (𝜑𝐿𝑊)       (𝜑 → (1r𝐾) = (1r𝐿))
 
Theoremdvdsrpropdg 13139* The divisibility relation depends only on the ring's base set and multiplication operation. (Contributed by Mario Carneiro, 26-Dec-2014.)
(𝜑𝐵 = (Base‘𝐾))    &   (𝜑𝐵 = (Base‘𝐿))    &   ((𝜑 ∧ (𝑥𝐵𝑦𝐵)) → (𝑥(.r𝐾)𝑦) = (𝑥(.r𝐿)𝑦))    &   (𝜑𝐾 ∈ SRing)    &   (𝜑𝐿 ∈ SRing)       (𝜑 → (∥r𝐾) = (∥r𝐿))
 
Theoremunitpropdg 13140* The set of units depends only on the ring's base set and multiplication operation. (Contributed by Mario Carneiro, 26-Dec-2014.)
(𝜑𝐵 = (Base‘𝐾))    &   (𝜑𝐵 = (Base‘𝐿))    &   ((𝜑 ∧ (𝑥𝐵𝑦𝐵)) → (𝑥(.r𝐾)𝑦) = (𝑥(.r𝐿)𝑦))    &   (𝜑𝐾 ∈ Ring)    &   (𝜑𝐿 ∈ Ring)       (𝜑 → (Unit‘𝐾) = (Unit‘𝐿))
 
Theoreminvrpropdg 13141* The ring inverse function depends only on the ring's base set and multiplication operation. (Contributed by Mario Carneiro, 26-Dec-2014.) (Revised by Mario Carneiro, 5-Oct-2015.)
(𝜑𝐵 = (Base‘𝐾))    &   (𝜑𝐵 = (Base‘𝐿))    &   ((𝜑 ∧ (𝑥𝐵𝑦𝐵)) → (𝑥(.r𝐾)𝑦) = (𝑥(.r𝐿)𝑦))    &   (𝜑𝐾 ∈ Ring)    &   (𝜑𝐿 ∈ Ring)       (𝜑 → (invr𝐾) = (invr𝐿))
 
7.3.7  Ring homomorphisms
 
Syntaxcrh 13142 Extend class notation with the ring homomorphisms.
class RingHom
 
Syntaxcrs 13143 Extend class notation with the ring isomorphisms.
class RingIso
 
Definitiondf-rnghom 13144* Define the set of ring homomorphisms from 𝑟 to 𝑠. (Contributed by Stefan O'Rear, 7-Mar-2015.)
RingHom = (𝑟 ∈ Ring, 𝑠 ∈ Ring ↦ (Base‘𝑟) / 𝑣(Base‘𝑠) / 𝑤{𝑓 ∈ (𝑤𝑚 𝑣) ∣ ((𝑓‘(1r𝑟)) = (1r𝑠) ∧ ∀𝑥𝑣𝑦𝑣 ((𝑓‘(𝑥(+g𝑟)𝑦)) = ((𝑓𝑥)(+g𝑠)(𝑓𝑦)) ∧ (𝑓‘(𝑥(.r𝑟)𝑦)) = ((𝑓𝑥)(.r𝑠)(𝑓𝑦))))})
 
Definitiondf-rngiso 13145* Define the set of ring isomorphisms from 𝑟 to 𝑠. (Contributed by Stefan O'Rear, 7-Mar-2015.)
RingIso = (𝑟 ∈ V, 𝑠 ∈ V ↦ {𝑓 ∈ (𝑟 RingHom 𝑠) ∣ 𝑓 ∈ (𝑠 RingHom 𝑟)})
 
7.4  The complex numbers as an algebraic extensible structure
 
7.4.1  Definition and basic properties
 
Syntaxcpsmet 13146 Extend class notation with the class of all pseudometric spaces.
class PsMet
 
Syntaxcxmet 13147 Extend class notation with the class of all extended metric spaces.
class ∞Met
 
Syntaxcmet 13148 Extend class notation with the class of all metrics.
class Met
 
Syntaxcbl 13149 Extend class notation with the metric space ball function.
class ball
 
Syntaxcfbas 13150 Extend class definition to include the class of filter bases.
class fBas
 
Syntaxcfg 13151 Extend class definition to include the filter generating function.
class filGen
 
Syntaxcmopn 13152 Extend class notation with a function mapping each metric space to the family of its open sets.
class MetOpen
 
Syntaxcmetu 13153 Extend class notation with the function mapping metrics to the uniform structure generated by that metric.
class metUnif
 
Definitiondf-psmet 13154* Define the set of all pseudometrics on a given base set. In a pseudo metric, two distinct points may have a distance zero. (Contributed by Thierry Arnoux, 7-Feb-2018.)
PsMet = (𝑥 ∈ V ↦ {𝑑 ∈ (ℝ*𝑚 (𝑥 × 𝑥)) ∣ ∀𝑦𝑥 ((𝑦𝑑𝑦) = 0 ∧ ∀𝑧𝑥𝑤𝑥 (𝑦𝑑𝑧) ≤ ((𝑤𝑑𝑦) +𝑒 (𝑤𝑑𝑧)))})
 
Definitiondf-xmet 13155* Define the set of all extended metrics on a given base set. The definition is similar to df-met 13156, but we also allow the metric to take on the value +∞. (Contributed by Mario Carneiro, 20-Aug-2015.)
∞Met = (𝑥 ∈ V ↦ {𝑑 ∈ (ℝ*𝑚 (𝑥 × 𝑥)) ∣ ∀𝑦𝑥𝑧𝑥 (((𝑦𝑑𝑧) = 0 ↔ 𝑦 = 𝑧) ∧ ∀𝑤𝑥 (𝑦𝑑𝑧) ≤ ((𝑤𝑑𝑦) +𝑒 (𝑤𝑑𝑧)))})
 
Definitiondf-met 13156* Define the (proper) class of all metrics. (A metric space is the metric's base set paired with the metric. However, we will often also call the metric itself a "metric space".) Equivalent to Definition 14-1.1 of [Gleason] p. 223. (Contributed by NM, 25-Aug-2006.)
Met = (𝑥 ∈ V ↦ {𝑑 ∈ (ℝ ↑𝑚 (𝑥 × 𝑥)) ∣ ∀𝑦𝑥𝑧𝑥 (((𝑦𝑑𝑧) = 0 ↔ 𝑦 = 𝑧) ∧ ∀𝑤𝑥 (𝑦𝑑𝑧) ≤ ((𝑤𝑑𝑦) + (𝑤𝑑𝑧)))})
 
Definitiondf-bl 13157* Define the metric space ball function. (Contributed by NM, 30-Aug-2006.) (Revised by Thierry Arnoux, 11-Feb-2018.)
ball = (𝑑 ∈ V ↦ (𝑥 ∈ dom dom 𝑑, 𝑧 ∈ ℝ* ↦ {𝑦 ∈ dom dom 𝑑 ∣ (𝑥𝑑𝑦) < 𝑧}))
 
Definitiondf-mopn 13158 Define a function whose value is the family of open sets of a metric space. (Contributed by NM, 1-Sep-2006.)
MetOpen = (𝑑 ran ∞Met ↦ (topGen‘ran (ball‘𝑑)))
 
Definitiondf-fbas 13159* Define the class of all filter bases. Note that a filter base on one set is also a filter base for any superset, so there is not a unique base set that can be recovered. (Contributed by Jeff Hankins, 1-Sep-2009.) (Revised by Stefan O'Rear, 11-Jul-2015.)
fBas = (𝑤 ∈ V ↦ {𝑥 ∈ 𝒫 𝒫 𝑤 ∣ (𝑥 ≠ ∅ ∧ ∅ ∉ 𝑥 ∧ ∀𝑦𝑥𝑧𝑥 (𝑥 ∩ 𝒫 (𝑦𝑧)) ≠ ∅)})
 
Definitiondf-fg 13160* Define the filter generating function. (Contributed by Jeff Hankins, 3-Sep-2009.) (Revised by Stefan O'Rear, 11-Jul-2015.)
filGen = (𝑤 ∈ V, 𝑥 ∈ (fBas‘𝑤) ↦ {𝑦 ∈ 𝒫 𝑤 ∣ (𝑥 ∩ 𝒫 𝑦) ≠ ∅})
 
Definitiondf-metu 13161* Define the function mapping metrics to the uniform structure generated by that metric. (Contributed by Thierry Arnoux, 1-Dec-2017.) (Revised by Thierry Arnoux, 11-Feb-2018.)
metUnif = (𝑑 ran PsMet ↦ ((dom dom 𝑑 × dom dom 𝑑)filGenran (𝑎 ∈ ℝ+ ↦ (𝑑 “ (0[,)𝑎)))))
 
PART 8  BASIC TOPOLOGY
 
8.1  Topology
 
8.1.1  Topological spaces

A topology on a set is a set of subsets of that set, called open sets, which satisfy certain conditions. One condition is that the whole set be an open set. Therefore, a set is recoverable from a topology on it (as its union), and it may sometimes be more convenient to consider topologies without reference to the underlying set.

 
8.1.1.1  Topologies
 
Syntaxctop 13162 Syntax for the class of topologies.
class Top
 
Definitiondf-top 13163* Define the class of topologies. It is a proper class. See istopg 13164 and istopfin 13165 for the corresponding characterizations, using respectively binary intersections like in this definition and nonempty finite intersections.

The final form of the definition is due to Bourbaki (Def. 1 of [BourbakiTop1] p. I.1), while the idea of defining a topology in terms of its open sets is due to Aleksandrov. For the convoluted history of the definitions of these notions, see

Gregory H. Moore, The emergence of open sets, closed sets, and limit points in analysis and topology, Historia Mathematica 35 (2008) 220--241.

(Contributed by NM, 3-Mar-2006.) (Revised by BJ, 20-Oct-2018.)

Top = {𝑥 ∣ (∀𝑦 ∈ 𝒫 𝑥 𝑦𝑥 ∧ ∀𝑦𝑥𝑧𝑥 (𝑦𝑧) ∈ 𝑥)}
 
Theoremistopg 13164* Express the predicate "𝐽 is a topology". See istopfin 13165 for another characterization using nonempty finite intersections instead of binary intersections.

Note: In the literature, a topology is often represented by a calligraphic letter T, which resembles the letter J. This confusion may have led to J being used by some authors (e.g., K. D. Joshi, Introduction to General Topology (1983), p. 114) and it is convenient for us since we later use 𝑇 to represent linear transformations (operators). (Contributed by Stefan Allan, 3-Mar-2006.) (Revised by Mario Carneiro, 11-Nov-2013.)

(𝐽𝐴 → (𝐽 ∈ Top ↔ (∀𝑥(𝑥𝐽 𝑥𝐽) ∧ ∀𝑥𝐽𝑦𝐽 (𝑥𝑦) ∈ 𝐽)))
 
Theoremistopfin 13165* Express the predicate "𝐽 is a topology" using nonempty finite intersections instead of binary intersections as in istopg 13164. It is not clear we can prove the converse without adding additional conditions. (Contributed by NM, 19-Jul-2006.) (Revised by Jim Kingdon, 14-Jan-2023.)
(𝐽 ∈ Top → (∀𝑥(𝑥𝐽 𝑥𝐽) ∧ ∀𝑥((𝑥𝐽𝑥 ≠ ∅ ∧ 𝑥 ∈ Fin) → 𝑥𝐽)))
 
Theoremuniopn 13166 The union of a subset of a topology (that is, the union of any family of open sets of a topology) is an open set. (Contributed by Stefan Allan, 27-Feb-2006.)
((𝐽 ∈ Top ∧ 𝐴𝐽) → 𝐴𝐽)
 
Theoremiunopn 13167* The indexed union of a subset of a topology is an open set. (Contributed by NM, 5-Oct-2006.)
((𝐽 ∈ Top ∧ ∀𝑥𝐴 𝐵𝐽) → 𝑥𝐴 𝐵𝐽)
 
Theoreminopn 13168 The intersection of two open sets of a topology is an open set. (Contributed by NM, 17-Jul-2006.)
((𝐽 ∈ Top ∧ 𝐴𝐽𝐵𝐽) → (𝐴𝐵) ∈ 𝐽)
 
Theoremfiinopn 13169 The intersection of a nonempty finite family of open sets is open. (Contributed by FL, 20-Apr-2012.)
(𝐽 ∈ Top → ((𝐴𝐽𝐴 ≠ ∅ ∧ 𝐴 ∈ Fin) → 𝐴𝐽))
 
Theoremunopn 13170 The union of two open sets is open. (Contributed by Jeff Madsen, 2-Sep-2009.)
((𝐽 ∈ Top ∧ 𝐴𝐽𝐵𝐽) → (𝐴𝐵) ∈ 𝐽)
 
Theorem0opn 13171 The empty set is an open subset of any topology. (Contributed by Stefan Allan, 27-Feb-2006.)
(𝐽 ∈ Top → ∅ ∈ 𝐽)
 
Theorem0ntop 13172 The empty set is not a topology. (Contributed by FL, 1-Jun-2008.)
¬ ∅ ∈ Top
 
Theoremtopopn 13173 The underlying set of a topology is an open set. (Contributed by NM, 17-Jul-2006.)
𝑋 = 𝐽       (𝐽 ∈ Top → 𝑋𝐽)
 
Theoremeltopss 13174 A member of a topology is a subset of its underlying set. (Contributed by NM, 12-Sep-2006.)
𝑋 = 𝐽       ((𝐽 ∈ Top ∧ 𝐴𝐽) → 𝐴𝑋)
 
8.1.1.2  Topologies on sets
 
Syntaxctopon 13175 Syntax for the function of topologies on sets.
class TopOn
 
Definitiondf-topon 13176* Define the function that associates with a set the set of topologies on it. (Contributed by Stefan O'Rear, 31-Jan-2015.)
TopOn = (𝑏 ∈ V ↦ {𝑗 ∈ Top ∣ 𝑏 = 𝑗})
 
Theoremfuntopon 13177 The class TopOn is a function. (Contributed by BJ, 29-Apr-2021.)
Fun TopOn
 
Theoremistopon 13178 Property of being a topology with a given base set. (Contributed by Stefan O'Rear, 31-Jan-2015.) (Revised by Mario Carneiro, 13-Aug-2015.)
(𝐽 ∈ (TopOn‘𝐵) ↔ (𝐽 ∈ Top ∧ 𝐵 = 𝐽))
 
Theoremtopontop 13179 A topology on a given base set is a topology. (Contributed by Mario Carneiro, 13-Aug-2015.)
(𝐽 ∈ (TopOn‘𝐵) → 𝐽 ∈ Top)
 
Theoremtoponuni 13180 The base set of a topology on a given base set. (Contributed by Mario Carneiro, 13-Aug-2015.)
(𝐽 ∈ (TopOn‘𝐵) → 𝐵 = 𝐽)
 
Theoremtopontopi 13181 A topology on a given base set is a topology. (Contributed by Mario Carneiro, 13-Aug-2015.)
𝐽 ∈ (TopOn‘𝐵)       𝐽 ∈ Top
 
Theoremtoponunii 13182 The base set of a topology on a given base set. (Contributed by Mario Carneiro, 13-Aug-2015.)
𝐽 ∈ (TopOn‘𝐵)       𝐵 = 𝐽
 
Theoremtoptopon 13183 Alternative definition of Top in terms of TopOn. (Contributed by Mario Carneiro, 13-Aug-2015.)
𝑋 = 𝐽       (𝐽 ∈ Top ↔ 𝐽 ∈ (TopOn‘𝑋))
 
Theoremtoptopon2 13184 A topology is the same thing as a topology on the union of its open sets. (Contributed by BJ, 27-Apr-2021.)
(𝐽 ∈ Top ↔ 𝐽 ∈ (TopOn‘ 𝐽))
 
Theoremtopontopon 13185 A topology on a set is a topology on the union of its open sets. (Contributed by BJ, 27-Apr-2021.)
(𝐽 ∈ (TopOn‘𝑋) → 𝐽 ∈ (TopOn‘ 𝐽))
 
Theoremtoponrestid 13186 Given a topology on a set, restricting it to that same set has no effect. (Contributed by Jim Kingdon, 6-Jul-2022.)
𝐴 ∈ (TopOn‘𝐵)       𝐴 = (𝐴t 𝐵)
 
Theoremtoponsspwpwg 13187 The set of topologies on a set is included in the double power set of that set. (Contributed by BJ, 29-Apr-2021.) (Revised by Jim Kingdon, 16-Jan-2023.)
(𝐴𝑉 → (TopOn‘𝐴) ⊆ 𝒫 𝒫 𝐴)
 
Theoremdmtopon 13188 The domain of TopOn is V. (Contributed by BJ, 29-Apr-2021.)
dom TopOn = V
 
Theoremfntopon 13189 The class TopOn is a function with domain V. (Contributed by BJ, 29-Apr-2021.)
TopOn Fn V
 
Theoremtoponmax 13190 The base set of a topology is an open set. (Contributed by Mario Carneiro, 13-Aug-2015.)
(𝐽 ∈ (TopOn‘𝐵) → 𝐵𝐽)
 
Theoremtoponss 13191 A member of a topology is a subset of its underlying set. (Contributed by Mario Carneiro, 21-Aug-2015.)
((𝐽 ∈ (TopOn‘𝑋) ∧ 𝐴𝐽) → 𝐴𝑋)
 
Theoremtoponcom 13192 If 𝐾 is a topology on the base set of topology 𝐽, then 𝐽 is a topology on the base of 𝐾. (Contributed by Mario Carneiro, 22-Aug-2015.)
((𝐽 ∈ Top ∧ 𝐾 ∈ (TopOn‘ 𝐽)) → 𝐽 ∈ (TopOn‘ 𝐾))
 
Theoremtoponcomb 13193 Biconditional form of toponcom 13192. (Contributed by BJ, 5-Dec-2021.)
((𝐽 ∈ Top ∧ 𝐾 ∈ Top) → (𝐽 ∈ (TopOn‘ 𝐾) ↔ 𝐾 ∈ (TopOn‘ 𝐽)))
 
Theoremtopgele 13194 The topologies over the same set have the greatest element (the discrete topology) and the least element (the indiscrete topology). (Contributed by FL, 18-Apr-2010.) (Revised by Mario Carneiro, 16-Sep-2015.)
(𝐽 ∈ (TopOn‘𝑋) → ({∅, 𝑋} ⊆ 𝐽𝐽 ⊆ 𝒫 𝑋))
 
8.1.1.3  Topological spaces
 
Syntaxctps 13195 Syntax for the class of topological spaces.
class TopSp
 
Definitiondf-topsp 13196 Define the class of topological spaces (as extensible structures). (Contributed by Stefan O'Rear, 13-Aug-2015.)
TopSp = {𝑓 ∣ (TopOpen‘𝑓) ∈ (TopOn‘(Base‘𝑓))}
 
Theoremistps 13197 Express the predicate "is a topological space". (Contributed by Mario Carneiro, 13-Aug-2015.)
𝐴 = (Base‘𝐾)    &   𝐽 = (TopOpen‘𝐾)       (𝐾 ∈ TopSp ↔ 𝐽 ∈ (TopOn‘𝐴))
 
Theoremistps2 13198 Express the predicate "is a topological space". (Contributed by NM, 20-Oct-2012.)
𝐴 = (Base‘𝐾)    &   𝐽 = (TopOpen‘𝐾)       (𝐾 ∈ TopSp ↔ (𝐽 ∈ Top ∧ 𝐴 = 𝐽))
 
Theoremtpsuni 13199 The base set of a topological space. (Contributed by FL, 27-Jun-2014.)
𝐴 = (Base‘𝐾)    &   𝐽 = (TopOpen‘𝐾)       (𝐾 ∈ TopSp → 𝐴 = 𝐽)
 
Theoremtpstop 13200 The topology extractor on a topological space is a topology. (Contributed by FL, 27-Jun-2014.)
𝐽 = (TopOpen‘𝐾)       (𝐾 ∈ TopSp → 𝐽 ∈ Top)
    < Previous  Next >

Page List
Jump to page: Contents  1 1-100 2 101-200 3 201-300 4 301-400 5 401-500 6 501-600 7 601-700 8 701-800 9 801-900 10 901-1000 11 1001-1100 12 1101-1200 13 1201-1300 14 1301-1400 15 1401-1500 16 1501-1600 17 1601-1700 18 1701-1800 19 1801-1900 20 1901-2000 21 2001-2100 22 2101-2200 23 2201-2300 24 2301-2400 25 2401-2500 26 2501-2600 27 2601-2700 28 2701-2800 29 2801-2900 30 2901-3000 31 3001-3100 32 3101-3200 33 3201-3300 34 3301-3400 35 3401-3500 36 3501-3600 37 3601-3700 38 3701-3800 39 3801-3900 40 3901-4000 41 4001-4100 42 4101-4200 43 4201-4300 44 4301-4400 45 4401-4500 46 4501-4600 47 4601-4700 48 4701-4800 49 4801-4900 50 4901-5000 51 5001-5100 52 5101-5200 53 5201-5300 54 5301-5400 55 5401-5500 56 5501-5600 57 5601-5700 58 5701-5800 59 5801-5900 60 5901-6000 61 6001-6100 62 6101-6200 63 6201-6300 64 6301-6400 65 6401-6500 66 6501-6600 67 6601-6700 68 6701-6800 69 6801-6900 70 6901-7000 71 7001-7100 72 7101-7200 73 7201-7300 74 7301-7400 75 7401-7500 76 7501-7600 77 7601-7700 78 7701-7800 79 7801-7900 80 7901-8000 81 8001-8100 82 8101-8200 83 8201-8300 84 8301-8400 85 8401-8500 86 8501-8600 87 8601-8700 88 8701-8800 89 8801-8900 90 8901-9000 91 9001-9100 92 9101-9200 93 9201-9300 94 9301-9400 95 9401-9500 96 9501-9600 97 9601-9700 98 9701-9800 99 9801-9900 100 9901-10000 101 10001-10100 102 10101-10200 103 10201-10300 104 10301-10400 105 10401-10500 106 10501-10600 107 10601-10700 108 10701-10800 109 10801-10900 110 10901-11000 111 11001-11100 112 11101-11200 113 11201-11300 114 11301-11400 115 11401-11500 116 11501-11600 117 11601-11700 118 11701-11800 119 11801-11900 120 11901-12000 121 12001-12100 122 12101-12200 123 12201-12300 124 12301-12400 125 12401-12500 126 12501-12600 127 12601-12700 128 12701-12800 129 12801-12900 130 12901-13000 131 13001-13100 132 13101-13200 133 13201-13300 134 13301-13400 135 13401-13500 136 13501-13600 137 13601-13700 138 13701-13800 139 13801-13900 140 13901-14000 141 14001-14100 142 14101-14200 143 14201-14300 144 14301-14400 145 14401-14485
  Copyright terms: Public domain < Previous  Next >