| Metamath
Proof Explorer Theorem List (p. 370 of 497) | < 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-30845) |
(30846-32368) |
(32369-49617) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | bj-gabeqd 36901 | Equality of generalized class abstractions. Deduction form. (Contributed by BJ, 4-Oct-2024.) |
| ⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → {𝐴 ∣ 𝑥 ∣ 𝜓} = {𝐵 ∣ 𝑥 ∣ 𝜒}) | ||
| Theorem | bj-gabeqis 36902* | Equality of generalized class abstractions, with implicit substitution. (Contributed by BJ, 4-Oct-2024.) |
| ⊢ (𝑥 = 𝑦 → 𝐴 = 𝐵) & ⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ {𝐴 ∣ 𝑥 ∣ 𝜑} = {𝐵 ∣ 𝑦 ∣ 𝜓} | ||
| Theorem | bj-elgab 36903 | Elements of a generalized class abstraction. (Contributed by BJ, 4-Oct-2024.) |
| ⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → Ⅎ𝑥𝐴) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → (∃𝑥(𝐴 = 𝐵 ∧ 𝜓) ↔ 𝜒)) ⇒ ⊢ (𝜑 → (𝐴 ∈ {𝐵 ∣ 𝑥 ∣ 𝜓} ↔ 𝜒)) | ||
| Theorem | bj-gabima 36904 |
Generalized class abstraction as a direct image.
TODO: improve the support lemmas elimag 6051 and fvelima 6943 to nonfreeness hypothesis (and for the latter, biconditional). (Contributed by BJ, 4-Oct-2024.) |
| ⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → Ⅎ𝑥𝐹) & ⊢ (𝜑 → Fun 𝐹) & ⊢ (𝜑 → {𝑥 ∣ 𝜓} ⊆ dom 𝐹) ⇒ ⊢ (𝜑 → {(𝐹‘𝑥) ∣ 𝑥 ∣ 𝜓} = (𝐹 “ {𝑥 ∣ 𝜓})) | ||
In this subsection, we define restricted nonfreeness (or relative nonfreeness). | ||
| Syntax | wrnf 36905 | Syntax for restricted nonfreeness. |
| wff Ⅎ𝑥 ∈ 𝐴𝜑 | ||
| Definition | df-bj-rnf 36906 | Definition of restricted nonfreeness. Informally, the proposition Ⅎ𝑥 ∈ 𝐴𝜑 means that 𝜑(𝑥) does not vary on 𝐴. (Contributed by BJ, 19-Mar-2021.) |
| ⊢ (Ⅎ𝑥 ∈ 𝐴𝜑 ↔ (∃𝑥 ∈ 𝐴 𝜑 → ∀𝑥 ∈ 𝐴 𝜑)) | ||
A few results around Russell's paradox. For clarity, we prove separately a FOL statement (now in the main part as ru0 2127) and then two versions (bj-ru1 36907 and bj-ru 36908). Special attention is put on minimizing axiom depencencies. | ||
| Theorem | bj-ru1 36907* | A version of Russell's paradox ru 3763 not mentioning the universal class. (see also bj-ru 36908). (Contributed by BJ, 12-Oct-2019.) Remove usage of ax-10 2141, ax-11 2157, ax-12 2177 by using eqabbw 2808 following BTernaryTau's similar revision of ru 3763. (Revised by BJ, 28-Jun-2025.) (Proof modification is discouraged.) |
| ⊢ ¬ ∃𝑦 𝑦 = {𝑥 ∣ ¬ 𝑥 ∈ 𝑥} | ||
| Theorem | bj-ru 36908 | Remove dependency on ax-13 2376 (and df-v 3461) from Russell's paradox ru 3763 expressed with primitive symbols and with a class variable 𝑉. Note the more economical use of elissetv 2815 instead of isset 3473 to avoid use of df-v 3461. (Contributed by BJ, 12-Oct-2019.) (Proof modification is discouraged.) |
| ⊢ ¬ {𝑥 ∣ ¬ 𝑥 ∈ 𝑥} ∈ 𝑉 | ||
| Theorem | currysetlem 36909* | Lemma for currysetlem 36909, where it is used with (𝑥 ∈ 𝑥 → 𝜑) substituted for 𝜓. (Contributed by BJ, 23-Sep-2023.) This proof is intuitionistically valid. (Proof modification is discouraged.) |
| ⊢ ({𝑥 ∣ 𝜓} ∈ 𝑉 → ({𝑥 ∣ 𝜓} ∈ {𝑥 ∣ (𝑥 ∈ 𝑥 → 𝜑)} ↔ ({𝑥 ∣ 𝜓} ∈ {𝑥 ∣ 𝜓} → 𝜑))) | ||
| Theorem | curryset 36910* | Curry's paradox in set theory. This can be seen as a generalization of Russell's paradox, which corresponds to the case where 𝜑 is ⊥. See alternate exposal of basically the same proof currysetALT 36914. (Contributed by BJ, 23-Sep-2023.) This proof is intuitionistically valid. (Proof modification is discouraged.) |
| ⊢ ¬ {𝑥 ∣ (𝑥 ∈ 𝑥 → 𝜑)} ∈ 𝑉 | ||
| Theorem | currysetlem1 36911* | Lemma for currysetALT 36914. (Contributed by BJ, 23-Sep-2023.) This proof is intuitionistically valid. (Proof modification is discouraged.) |
| ⊢ 𝑋 = {𝑥 ∣ (𝑥 ∈ 𝑥 → 𝜑)} ⇒ ⊢ (𝑋 ∈ 𝑉 → (𝑋 ∈ 𝑋 ↔ (𝑋 ∈ 𝑋 → 𝜑))) | ||
| Theorem | currysetlem2 36912* | Lemma for currysetALT 36914. (Contributed by BJ, 23-Sep-2023.) This proof is intuitionistically valid. (Proof modification is discouraged.) |
| ⊢ 𝑋 = {𝑥 ∣ (𝑥 ∈ 𝑥 → 𝜑)} ⇒ ⊢ (𝑋 ∈ 𝑉 → (𝑋 ∈ 𝑋 → 𝜑)) | ||
| Theorem | currysetlem3 36913* | Lemma for currysetALT 36914. (Contributed by BJ, 23-Sep-2023.) This proof is intuitionistically valid. (Proof modification is discouraged.) |
| ⊢ 𝑋 = {𝑥 ∣ (𝑥 ∈ 𝑥 → 𝜑)} ⇒ ⊢ ¬ 𝑋 ∈ 𝑉 | ||
| Theorem | currysetALT 36914* | Alternate proof of curryset 36910, or more precisely alternate exposal of the same proof. (Contributed by BJ, 23-Sep-2023.) This proof is intuitionistically valid. (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ ¬ {𝑥 ∣ (𝑥 ∈ 𝑥 → 𝜑)} ∈ 𝑉 | ||
A few utility theorems on disjointness of classes. | ||
| Theorem | bj-n0i 36915* | Inference associated with n0 4328. Shortens 2ndcdisj 23392 (2888>2878), notzfaus 5333 (264>253). (Contributed by BJ, 22-Apr-2019.) |
| ⊢ 𝐴 ≠ ∅ ⇒ ⊢ ∃𝑥 𝑥 ∈ 𝐴 | ||
| Theorem | bj-disjsn01 36916 | Disjointness of the singletons containing 0 and 1. This is a consequence of disjcsn 9616 but the present proof does not use regularity. (Contributed by BJ, 4-Apr-2019.) (Proof modification is discouraged.) |
| ⊢ ({∅} ∩ {1o}) = ∅ | ||
| Theorem | bj-0nel1 36917 | The empty set does not belong to {1o}. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ ∅ ∉ {1o} | ||
| Theorem | bj-1nel0 36918 | 1o does not belong to {∅}. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ 1o ∉ {∅} | ||
A few utility theorems on direct products. | ||
| Theorem | bj-xpimasn 36919 | The image of a singleton, general case. [Change and relabel xpimasn 6174 accordingly, maybe to xpima2sn.] (Contributed by BJ, 6-Apr-2019.) |
| ⊢ ((𝐴 × 𝐵) “ {𝑋}) = if(𝑋 ∈ 𝐴, 𝐵, ∅) | ||
| Theorem | bj-xpima1sn 36920 | The image of a singleton by a direct product, empty case. [Change and relabel xpimasn 6174 accordingly, maybe to xpima2sn.] (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (¬ 𝑋 ∈ 𝐴 → ((𝐴 × 𝐵) “ {𝑋}) = ∅) | ||
| Theorem | bj-xpima1snALT 36921 | Alternate proof of bj-xpima1sn 36920. (Contributed by BJ, 6-Apr-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ (¬ 𝑋 ∈ 𝐴 → ((𝐴 × 𝐵) “ {𝑋}) = ∅) | ||
| Theorem | bj-xpima2sn 36922 | The image of a singleton by a direct product, nonempty case. [To replace xpimasn 6174.] (Contributed by BJ, 6-Apr-2019.) (Proof modification is discouraged.) |
| ⊢ (𝑋 ∈ 𝐴 → ((𝐴 × 𝐵) “ {𝑋}) = 𝐵) | ||
| Theorem | bj-xpnzex 36923 | If the first factor of a product is nonempty, and the product is a set, then the second factor is a set. UPDATE: this is actually the curried (exported) form of xpexcnv 7914 (up to commutation in the product). (Contributed by BJ, 6-Oct-2018.) (Proof modification is discouraged.) |
| ⊢ (𝐴 ≠ ∅ → ((𝐴 × 𝐵) ∈ 𝑉 → 𝐵 ∈ V)) | ||
| Theorem | bj-xpexg2 36924 | Curried (exported) form of xpexg 7742. (Contributed by BJ, 2-Apr-2019.) |
| ⊢ (𝐴 ∈ 𝑉 → (𝐵 ∈ 𝑊 → (𝐴 × 𝐵) ∈ V)) | ||
| Theorem | bj-xpnzexb 36925 | If the first factor of a product is a nonempty set, then the product is a set if and only if the second factor is a set. (Contributed by BJ, 2-Apr-2019.) |
| ⊢ (𝐴 ∈ (𝑉 ∖ {∅}) → (𝐵 ∈ V ↔ (𝐴 × 𝐵) ∈ V)) | ||
| Theorem | bj-cleq 36926* | Substitution property for certain classes. (Contributed by BJ, 2-Apr-2019.) |
| ⊢ (𝐴 = 𝐵 → {𝑥 ∣ {𝑥} ∈ (𝐴 “ 𝐶)} = {𝑥 ∣ {𝑥} ∈ (𝐵 “ 𝐶)}) | ||
This subsection introduces the "singletonization" and the "tagging" of a class. The singletonization of a class is the class of singletons of elements of that class. It is useful since all nonsingletons are disjoint from it, so one can easily adjoin to it disjoint elements, which is what the tagging does: it adjoins the empty set. This can be used for instance to define the one-point compactification of a topological space. It will be used in the next section to define tuples which work for proper classes. | ||
| Theorem | bj-snsetex 36927* | The class of sets "whose singletons" belong to a set is a set. Nice application of ax-rep 5249. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ 𝑉 → {𝑥 ∣ {𝑥} ∈ 𝐴} ∈ V) | ||
| Theorem | bj-clexab 36928* | Sethood of certain classes. (Contributed by BJ, 2-Apr-2019.) |
| ⊢ (𝐴 ∈ 𝑉 → {𝑥 ∣ {𝑥} ∈ (𝐴 “ 𝐵)} ∈ V) | ||
| Syntax | bj-csngl 36929 | Syntax for singletonization. (Contributed by BJ, 6-Oct-2018.) |
| class sngl 𝐴 | ||
| Definition | df-bj-sngl 36930* | Definition of "singletonization". The class sngl 𝐴 is isomorphic to 𝐴 and since it contains only singletons, it can be easily be adjoined disjoint elements, which can be useful in various constructions. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ sngl 𝐴 = {𝑥 ∣ ∃𝑦 ∈ 𝐴 𝑥 = {𝑦}} | ||
| Theorem | bj-sngleq 36931 | Substitution property for sngl. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 = 𝐵 → sngl 𝐴 = sngl 𝐵) | ||
| Theorem | bj-elsngl 36932* | Characterization of the elements of the singletonization of a class. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ sngl 𝐵 ↔ ∃𝑥 ∈ 𝐵 𝐴 = {𝑥}) | ||
| Theorem | bj-snglc 36933 | Characterization of the elements of 𝐴 in terms of elements of its singletonization. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ 𝐵 ↔ {𝐴} ∈ sngl 𝐵) | ||
| Theorem | bj-snglss 36934 | The singletonization of a class is included in its powerclass. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ sngl 𝐴 ⊆ 𝒫 𝐴 | ||
| Theorem | bj-0nelsngl 36935 | The empty set is not a member of a singletonization (neither is any nonsingleton, in particular any von Neuman ordinal except possibly df-1o 8478). (Contributed by BJ, 6-Oct-2018.) |
| ⊢ ∅ ∉ sngl 𝐴 | ||
| Theorem | bj-snglinv 36936* | Inverse of singletonization. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ 𝐴 = {𝑥 ∣ {𝑥} ∈ sngl 𝐴} | ||
| Theorem | bj-snglex 36937 | A class is a set if and only if its singletonization is a set. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ V ↔ sngl 𝐴 ∈ V) | ||
| Syntax | bj-ctag 36938 | Syntax for the tagged copy of a class. (Contributed by BJ, 6-Oct-2018.) |
| class tag 𝐴 | ||
| Definition | df-bj-tag 36939 | Definition of the tagged copy of a class, that is, the adjunction to (an isomorph of) 𝐴 of a disjoint element (here, the empty set). Remark: this could be used for the one-point compactification of a topological space. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ tag 𝐴 = (sngl 𝐴 ∪ {∅}) | ||
| Theorem | bj-tageq 36940 | Substitution property for tag. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 = 𝐵 → tag 𝐴 = tag 𝐵) | ||
| Theorem | bj-eltag 36941* | Characterization of the elements of the tagging of a class. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ tag 𝐵 ↔ (∃𝑥 ∈ 𝐵 𝐴 = {𝑥} ∨ 𝐴 = ∅)) | ||
| Theorem | bj-0eltag 36942 | The empty set belongs to the tagging of a class. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ ∅ ∈ tag 𝐴 | ||
| Theorem | bj-tagn0 36943 | The tagging of a class is nonempty. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ tag 𝐴 ≠ ∅ | ||
| Theorem | bj-tagss 36944 | The tagging of a class is included in its powerclass. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ tag 𝐴 ⊆ 𝒫 𝐴 | ||
| Theorem | bj-snglsstag 36945 | The singletonization is included in the tagging. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ sngl 𝐴 ⊆ tag 𝐴 | ||
| Theorem | bj-sngltagi 36946 | The singletonization is included in the tagging. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ sngl 𝐵 → 𝐴 ∈ tag 𝐵) | ||
| Theorem | bj-sngltag 36947 | The singletonization and the tagging of a set contain the same singletons. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ 𝑉 → ({𝐴} ∈ sngl 𝐵 ↔ {𝐴} ∈ tag 𝐵)) | ||
| Theorem | bj-tagci 36948 | Characterization of the elements of 𝐵 in terms of elements of its tagged version. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ 𝐵 → {𝐴} ∈ tag 𝐵) | ||
| Theorem | bj-tagcg 36949 | Characterization of the elements of 𝐵 in terms of elements of its tagged version. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ 𝑉 → (𝐴 ∈ 𝐵 ↔ {𝐴} ∈ tag 𝐵)) | ||
| Theorem | bj-taginv 36950* | Inverse of tagging. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ 𝐴 = {𝑥 ∣ {𝑥} ∈ tag 𝐴} | ||
| Theorem | bj-tagex 36951 | A class is a set if and only if its tagging is a set. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ V ↔ tag 𝐴 ∈ V) | ||
| Theorem | bj-xtageq 36952 | The products of a given class and the tagging of either of two equal classes are equal. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (𝐴 = 𝐵 → (𝐶 × tag 𝐴) = (𝐶 × tag 𝐵)) | ||
| Theorem | bj-xtagex 36953 | The product of a set and the tagging of a set is a set. (Contributed by BJ, 2-Apr-2019.) |
| ⊢ (𝐴 ∈ 𝑉 → (𝐵 ∈ 𝑊 → (𝐴 × tag 𝐵) ∈ V)) | ||
This subsection gives a definition of an ordered pair, or couple (2-tuple), that "works" for proper classes, as evidenced by Theorems bj-2uplth 36985 and bj-2uplex 36986, and more importantly, bj-pr21val 36977 and bj-pr22val 36983. In particular, one can define well-behaved tuples of classes. Classes in ZF(C) are only virtual, and in particular they cannot be quantified over. Theorem bj-2uplex 36986 has advantages: in view of df-br 5120, several sethood antecedents could be removed from existing theorems. For instance, relsnopg 5782 (resp. relsnop 5784) would hold without antecedents (resp. hypotheses) thanks to relsnb 5781). Also, the antecedent Rel 𝑅 could be removed from brrelex12 5706 and related theorems brrelex*, and, as a consequence, of multiple later theorems. Similarly, df-struct 17164 could be simplified by removing the exception currently made for the empty set. The projections are denoted by pr1 and pr2 and the couple with projections (or coordinates) 𝐴 and 𝐵 is denoted by ⦅𝐴, 𝐵⦆. Note that this definition uses the Kuratowski definition (df-op 4608) as a preliminary definition, and then "redefines" a couple. It could also use the "short" version of the Kuratowski pair (see opthreg 9630) without needing the axiom of regularity; it could even bypass this definition by "inlining" it. This definition is due to Anthony Morse and is expounded (with idiosyncratic notation) in Anthony P. Morse, A Theory of Sets, Academic Press, 1965 (second edition 1986). Note that this extends in a natural way to tuples. A variation of this definition is justified in opthprc 5718, but here we use "tagged versions" of the factors (see df-bj-tag 36939) so that an m-tuple can equal an n-tuple only when m = n (and the projections are the same). A comparison of the different definitions of tuples (strangely not mentioning Morse's), is given in Dominic McCarty and Dana Scott, Reconsidering ordered pairs, Bull. Symbolic Logic, Volume 14, Issue 3 (Sept. 2008), 379--397. where a recursive definition of tuples is given that avoids the two-step definition of tuples and that can be adapted to various set theories. Finally, another survey is Akihiro Kanamori, The empty set, the singleton, and the ordered pair, Bull. Symbolic Logic, Volume 9, Number 3 (Sept. 2003), 273--298. (available at http://math.bu.edu/people/aki/8.pdf 36939) | ||
| Syntax | bj-cproj 36954 | Syntax for the class projection. (Contributed by BJ, 6-Apr-2019.) |
| class (𝐴 Proj 𝐵) | ||
| Definition | df-bj-proj 36955* | Definition of the class projection corresponding to tagged tuples. The expression (𝐴 Proj 𝐵) denotes the projection on the A^th component. (Contributed by BJ, 6-Apr-2019.) (New usage is discouraged.) |
| ⊢ (𝐴 Proj 𝐵) = {𝑥 ∣ {𝑥} ∈ (𝐵 “ {𝐴})} | ||
| Theorem | bj-projeq 36956 | Substitution property for Proj. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (𝐴 = 𝐶 → (𝐵 = 𝐷 → (𝐴 Proj 𝐵) = (𝐶 Proj 𝐷))) | ||
| Theorem | bj-projeq2 36957 | Substitution property for Proj. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (𝐵 = 𝐶 → (𝐴 Proj 𝐵) = (𝐴 Proj 𝐶)) | ||
| Theorem | bj-projun 36958 | The class projection on a given component preserves unions. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (𝐴 Proj (𝐵 ∪ 𝐶)) = ((𝐴 Proj 𝐵) ∪ (𝐴 Proj 𝐶)) | ||
| Theorem | bj-projex 36959 | Sethood of the class projection. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (𝐵 ∈ 𝑉 → (𝐴 Proj 𝐵) ∈ V) | ||
| Theorem | bj-projval 36960 | Value of the class projection. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (𝐴 ∈ 𝑉 → (𝐴 Proj ({𝐵} × tag 𝐶)) = if(𝐵 = 𝐴, 𝐶, ∅)) | ||
| Syntax | bj-c1upl 36961 | Syntax for Morse monuple. (Contributed by BJ, 6-Apr-2019.) |
| class ⦅𝐴⦆ | ||
| Definition | df-bj-1upl 36962 | Definition of the Morse monuple (1-tuple). This is not useful per se, but is used as a step towards the definition of couples (2-tuples, or ordered pairs). The reason for "tagging" the set is so that an m-tuple and an n-tuple be equal only when m = n. Note that with this definition, the 0-tuple is the empty set. New usage is discouraged because the precise definition is generally unimportant compared to the characteristic properties bj-2upleq 36976, bj-2uplth 36985, bj-2uplex 36986, and the properties of the projections (see df-bj-pr1 36965 and df-bj-pr2 36979). (Contributed by BJ, 6-Apr-2019.) (New usage is discouraged.) |
| ⊢ ⦅𝐴⦆ = ({∅} × tag 𝐴) | ||
| Theorem | bj-1upleq 36963 | Substitution property for ⦅ − ⦆. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (𝐴 = 𝐵 → ⦅𝐴⦆ = ⦅𝐵⦆) | ||
| Syntax | bj-cpr1 36964 | Syntax for the first class tuple projection. (Contributed by BJ, 6-Apr-2019.) |
| class pr1 𝐴 | ||
| Definition | df-bj-pr1 36965 | Definition of the first projection of a class tuple. New usage is discouraged because the precise definition is generally unimportant compared to the characteristic properties bj-pr1eq 36966, bj-pr11val 36969, bj-pr21val 36977, bj-pr1ex 36970. (Contributed by BJ, 6-Apr-2019.) (New usage is discouraged.) |
| ⊢ pr1 𝐴 = (∅ Proj 𝐴) | ||
| Theorem | bj-pr1eq 36966 | Substitution property for pr1. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (𝐴 = 𝐵 → pr1 𝐴 = pr1 𝐵) | ||
| Theorem | bj-pr1un 36967 | The first projection preserves unions. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ pr1 (𝐴 ∪ 𝐵) = (pr1 𝐴 ∪ pr1 𝐵) | ||
| Theorem | bj-pr1val 36968 | Value of the first projection. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ pr1 ({𝐴} × tag 𝐵) = if(𝐴 = ∅, 𝐵, ∅) | ||
| Theorem | bj-pr11val 36969 | Value of the first projection of a monuple. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ pr1 ⦅𝐴⦆ = 𝐴 | ||
| Theorem | bj-pr1ex 36970 | Sethood of the first projection. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ 𝑉 → pr1 𝐴 ∈ V) | ||
| Theorem | bj-1uplth 36971 | The characteristic property of monuples. Note that this holds without sethood hypotheses. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (⦅𝐴⦆ = ⦅𝐵⦆ ↔ 𝐴 = 𝐵) | ||
| Theorem | bj-1uplex 36972 | A monuple is a set if and only if its coordinates are sets. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ (⦅𝐴⦆ ∈ V ↔ 𝐴 ∈ V) | ||
| Theorem | bj-1upln0 36973 | A monuple is nonempty. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ ⦅𝐴⦆ ≠ ∅ | ||
| Syntax | bj-c2uple 36974 | Syntax for Morse couple. (Contributed by BJ, 6-Oct-2018.) |
| class ⦅𝐴, 𝐵⦆ | ||
| Definition | df-bj-2upl 36975 | Definition of the Morse couple. See df-bj-1upl 36962. New usage is discouraged because the precise definition is generally unimportant compared to the characteristic properties bj-2upleq 36976, bj-2uplth 36985, bj-2uplex 36986, and the properties of the projections (see df-bj-pr1 36965 and df-bj-pr2 36979). (Contributed by BJ, 6-Oct-2018.) (New usage is discouraged.) |
| ⊢ ⦅𝐴, 𝐵⦆ = (⦅𝐴⦆ ∪ ({1o} × tag 𝐵)) | ||
| Theorem | bj-2upleq 36976 | Substitution property for ⦅ − , − ⦆. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 = 𝐵 → (𝐶 = 𝐷 → ⦅𝐴, 𝐶⦆ = ⦅𝐵, 𝐷⦆)) | ||
| Theorem | bj-pr21val 36977 | Value of the first projection of a couple. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ pr1 ⦅𝐴, 𝐵⦆ = 𝐴 | ||
| Syntax | bj-cpr2 36978 | Syntax for the second class tuple projection. (Contributed by BJ, 6-Oct-2018.) |
| class pr2 𝐴 | ||
| Definition | df-bj-pr2 36979 | Definition of the second projection of a class tuple. New usage is discouraged because the precise definition is generally unimportant compared to the characteristic properties bj-pr2eq 36980, bj-pr22val 36983, bj-pr2ex 36984. (Contributed by BJ, 6-Oct-2018.) (New usage is discouraged.) |
| ⊢ pr2 𝐴 = (1o Proj 𝐴) | ||
| Theorem | bj-pr2eq 36980 | Substitution property for pr2. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 = 𝐵 → pr2 𝐴 = pr2 𝐵) | ||
| Theorem | bj-pr2un 36981 | The second projection preserves unions. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ pr2 (𝐴 ∪ 𝐵) = (pr2 𝐴 ∪ pr2 𝐵) | ||
| Theorem | bj-pr2val 36982 | Value of the second projection. (Contributed by BJ, 6-Apr-2019.) |
| ⊢ pr2 ({𝐴} × tag 𝐵) = if(𝐴 = 1o, 𝐵, ∅) | ||
| Theorem | bj-pr22val 36983 | Value of the second projection of a couple. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ pr2 ⦅𝐴, 𝐵⦆ = 𝐵 | ||
| Theorem | bj-pr2ex 36984 | Sethood of the second projection. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (𝐴 ∈ 𝑉 → pr2 𝐴 ∈ V) | ||
| Theorem | bj-2uplth 36985 | The characteristic property of couples. Note that this holds without sethood hypotheses (compare opth 5451). (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (⦅𝐴, 𝐵⦆ = ⦅𝐶, 𝐷⦆ ↔ (𝐴 = 𝐶 ∧ 𝐵 = 𝐷)) | ||
| Theorem | bj-2uplex 36986 | A couple is a set if and only if its coordinates are sets. For the advantages offered by the reverse closure property, see the section head comment. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (⦅𝐴, 𝐵⦆ ∈ V ↔ (𝐴 ∈ V ∧ 𝐵 ∈ V)) | ||
| Theorem | bj-2upln0 36987 | A couple is nonempty. (Contributed by BJ, 21-Apr-2019.) |
| ⊢ ⦅𝐴, 𝐵⦆ ≠ ∅ | ||
| Theorem | bj-2upln1upl 36988 | A couple is never equal to a monuple. It is in order to have this "non-clashing" result that tagging was used. Without tagging, we would have ⦅𝐴, ∅⦆ = ⦅𝐴⦆. Note that in the context of Morse tuples, it is natural to define the 0-tuple as the empty set. Therefore, the present theorem together with bj-1upln0 36973 and bj-2upln0 36987 tell us that an m-tuple may equal an n-tuple only when m = n, at least for m, n <= 2, but this result would extend as soon as we define n-tuples for higher values of n. (Contributed by BJ, 21-Apr-2019.) |
| ⊢ ⦅𝐴, 𝐵⦆ ≠ ⦅𝐶⦆ | ||
Some elementary set-theoretic operations "relative to a universe" (by which is merely meant some given class considered as a universe). | ||
| Theorem | bj-rcleqf 36989 | Relative version of cleqf 2927. (Contributed by BJ, 27-Dec-2023.) |
| ⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐵 & ⊢ Ⅎ𝑥𝑉 ⇒ ⊢ ((𝑉 ∩ 𝐴) = (𝑉 ∩ 𝐵) ↔ ∀𝑥 ∈ 𝑉 (𝑥 ∈ 𝐴 ↔ 𝑥 ∈ 𝐵)) | ||
| Theorem | bj-rcleq 36990* | Relative version of dfcleq 2728. (Contributed by BJ, 27-Dec-2023.) |
| ⊢ ((𝑉 ∩ 𝐴) = (𝑉 ∩ 𝐵) ↔ ∀𝑥 ∈ 𝑉 (𝑥 ∈ 𝐴 ↔ 𝑥 ∈ 𝐵)) | ||
| Theorem | bj-reabeq 36991* | Relative form of eqabb 2874. (Contributed by BJ, 27-Dec-2023.) |
| ⊢ ((𝑉 ∩ 𝐴) = {𝑥 ∈ 𝑉 ∣ 𝜑} ↔ ∀𝑥 ∈ 𝑉 (𝑥 ∈ 𝐴 ↔ 𝜑)) | ||
| Theorem | bj-disj2r 36992 | Relative version of ssdifin0 4461, allowing a biconditional, and of disj2 4433. (Contributed by BJ, 11-Nov-2021.) This proof does not rely, even indirectly, on ssdifin0 4461 nor disj2 4433. (Proof modification is discouraged.) |
| ⊢ ((𝐴 ∩ 𝑉) ⊆ (𝑉 ∖ 𝐵) ↔ ((𝐴 ∩ 𝐵) ∩ 𝑉) = ∅) | ||
| Theorem | bj-sscon 36993 | Contraposition law for relative subclasses. Relative and generalized version of ssconb 4117, which it can shorten, as well as conss2 44415. (Contributed by BJ, 11-Nov-2021.) This proof does not rely, even indirectly, on ssconb 4117 nor conss2 44415. (Proof modification is discouraged.) |
| ⊢ ((𝐴 ∩ 𝑉) ⊆ (𝑉 ∖ 𝐵) ↔ (𝐵 ∩ 𝑉) ⊆ (𝑉 ∖ 𝐴)) | ||
In this section, we introduce the axiom of singleton ax-bj-sn 36997 and the axiom of binary union ax-bj-bun 37001. Both axioms are implied by the standard axioms of unordered pair ax-pr 5402 and of union ax-un 7727 (see snex 5406 and unex 7736). Conversely, the axiom of unordered pair ax-pr 5402 is implied by the axioms of singleton and of binary union, as proved in bj-prexg 37003 and bj-prex 37004. The axioms of union ax-un 7727 and of powerset ax-pow 5335 are independent of these axioms: consider respectively the class of pseudo-hereditarily sets of cardinality less than a given singular strong limit cardinal, see Greg Oman, On the axiom of union, Arch. Math. Logic (2010) 49:283--289 (that model does have finite unions), and the class of well-founded hereditarily countable sets (or hereditarily less than a given uncountable regular cardinal). See also https://mathoverflow.net/questions/81815 5335 and https://mathoverflow.net/questions/48365 5335. A proof by finite induction shows that the existence of finite unions is equivalent to the existence of binary unions and of nullary unions (the latter being the axiom of the empty set ax-nul 5276). The axiom of binary union is useful in theories without the axioms of union ax-un 7727 and of powerset ax-pow 5335. For instance, the class of well-founded sets hereditarily of cardinality at most 𝑛 ∈ ℕ0 with ordinary membership relation is a model of { ax-ext 2707, ax-rep 5249, ax-sep 5266, ax-nul 5276, ax-reg 9604 } and the axioms of existence of unordered 𝑚-tuples for all 𝑚 ≤ 𝑛, and in most cases one would like to rule out such models, hence the need for extra axioms, typically variants of powersets or unions. The axiom of adjunction ax-bj-adj 37006 is more widely used, and is an axiom of General Set Theory. We prove how to retrieve it from binary union and singleton in bj-adjfrombun 37010 and conversely how to prove from adjunction singleton (bj-snfromadj 37008) and unordered pair (bj-prfromadj 37009). | ||
| Theorem | bj-abex 36994* | Two ways of stating that the extension of a formula is a set. (Contributed by BJ, 18-Jan-2025.) (Proof modification is discouraged.) |
| ⊢ ({𝑥 ∣ 𝜑} ∈ V ↔ ∃𝑦∀𝑥(𝑥 ∈ 𝑦 ↔ 𝜑)) | ||
| Theorem | bj-clex 36995* | Two ways of stating that a class is a set. (Contributed by BJ, 18-Jan-2025.) (Proof modification is discouraged.) |
| ⊢ (𝑥 ∈ 𝐴 ↔ 𝜑) ⇒ ⊢ (𝐴 ∈ V ↔ ∃𝑦∀𝑥(𝑥 ∈ 𝑦 ↔ 𝜑)) | ||
| Theorem | bj-axsn 36996* | Two ways of stating the axiom of singleton (which is the universal closure of either side, see ax-bj-sn 36997). (Contributed by BJ, 12-Jan-2025.) (Proof modification is discouraged.) |
| ⊢ ({𝑥} ∈ V ↔ ∃𝑦∀𝑧(𝑧 ∈ 𝑦 ↔ 𝑧 = 𝑥)) | ||
| Axiom | ax-bj-sn 36997* | Axiom of singleton. (Contributed by BJ, 12-Jan-2025.) |
| ⊢ ∀𝑥∃𝑦∀𝑧(𝑧 ∈ 𝑦 ↔ 𝑧 = 𝑥) | ||
| Theorem | bj-snexg 36998 | A singleton built on a set is a set. Contrary to bj-snex 36999, this proof is intuitionistically valid and does not require ax-nul 5276. (Contributed by NM, 7-Aug-1994.) Extract it from snex 5406 and prove it from ax-bj-sn 36997. (Revised by BJ, 12-Jan-2025.) (Proof modification is discouraged.) |
| ⊢ (𝐴 ∈ 𝑉 → {𝐴} ∈ V) | ||
| Theorem | bj-snex 36999 | A singleton is a set. See also snex 5406, snexALT 5353. (Contributed by NM, 7-Aug-1994.) Prove it from ax-bj-sn 36997. (Revised by BJ, 12-Jan-2025.) (Proof modification is discouraged.) |
| ⊢ {𝐴} ∈ V | ||
| Theorem | bj-axbun 37000* | Two ways of stating the axiom of binary union (which is the universal closure of either side, see ax-bj-bun 37001). (Contributed by BJ, 12-Jan-2025.) (Proof modification is discouraged.) |
| ⊢ ((𝑥 ∪ 𝑦) ∈ V ↔ ∃𝑧∀𝑡(𝑡 ∈ 𝑧 ↔ (𝑡 ∈ 𝑥 ∨ 𝑡 ∈ 𝑦))) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |