Theorem List for Intuitionistic Logic Explorer - 3801-3900 *Has distinct variable
group(s)
| Type | Label | Description |
| Statement |
| |
| Theorem | prel12 3801 |
Equality of two unordered pairs. (Contributed by NM, 17-Oct-1996.)
|
| ⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V & ⊢ 𝐶 ∈ V & ⊢ 𝐷 ∈
V ⇒ ⊢ (¬ 𝐴 = 𝐵 → ({𝐴, 𝐵} = {𝐶, 𝐷} ↔ (𝐴 ∈ {𝐶, 𝐷} ∧ 𝐵 ∈ {𝐶, 𝐷}))) |
| |
| Theorem | opthpr 3802 |
A way to represent ordered pairs using unordered pairs with distinct
members. (Contributed by NM, 27-Mar-2007.)
|
| ⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V & ⊢ 𝐶 ∈ V & ⊢ 𝐷 ∈
V ⇒ ⊢ (𝐴 ≠ 𝐷 → ({𝐴, 𝐵} = {𝐶, 𝐷} ↔ (𝐴 = 𝐶 ∧ 𝐵 = 𝐷))) |
| |
| Theorem | preq12bg 3803 |
Closed form of preq12b 3800. (Contributed by Scott Fenton,
28-Mar-2014.)
|
| ⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) ∧ (𝐶 ∈ 𝑋 ∧ 𝐷 ∈ 𝑌)) → ({𝐴, 𝐵} = {𝐶, 𝐷} ↔ ((𝐴 = 𝐶 ∧ 𝐵 = 𝐷) ∨ (𝐴 = 𝐷 ∧ 𝐵 = 𝐶)))) |
| |
| Theorem | prneimg 3804 |
Two pairs are not equal if at least one element of the first pair is not
contained in the second pair. (Contributed by Alexander van der Vekens,
13-Aug-2017.)
|
| ⊢ (((𝐴 ∈ 𝑈 ∧ 𝐵 ∈ 𝑉) ∧ (𝐶 ∈ 𝑋 ∧ 𝐷 ∈ 𝑌)) → (((𝐴 ≠ 𝐶 ∧ 𝐴 ≠ 𝐷) ∨ (𝐵 ≠ 𝐶 ∧ 𝐵 ≠ 𝐷)) → {𝐴, 𝐵} ≠ {𝐶, 𝐷})) |
| |
| Theorem | preqsn 3805 |
Equivalence for a pair equal to a singleton. (Contributed by NM,
3-Jun-2008.)
|
| ⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V & ⊢ 𝐶 ∈
V ⇒ ⊢ ({𝐴, 𝐵} = {𝐶} ↔ (𝐴 = 𝐵 ∧ 𝐵 = 𝐶)) |
| |
| Theorem | dfopg 3806 |
Value of the ordered pair when the arguments are sets. (Contributed by
Mario Carneiro, 26-Apr-2015.)
|
| ⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → 〈𝐴, 𝐵〉 = {{𝐴}, {𝐴, 𝐵}}) |
| |
| Theorem | dfop 3807 |
Value of an ordered pair when the arguments are sets, with the
conclusion corresponding to Kuratowski's original definition.
(Contributed by NM, 25-Jun-1998.)
|
| ⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ 〈𝐴, 𝐵〉 = {{𝐴}, {𝐴, 𝐵}} |
| |
| Theorem | opeq1 3808 |
Equality theorem for ordered pairs. (Contributed by NM, 25-Jun-1998.)
(Revised by Mario Carneiro, 26-Apr-2015.)
|
| ⊢ (𝐴 = 𝐵 → 〈𝐴, 𝐶〉 = 〈𝐵, 𝐶〉) |
| |
| Theorem | opeq2 3809 |
Equality theorem for ordered pairs. (Contributed by NM, 25-Jun-1998.)
(Revised by Mario Carneiro, 26-Apr-2015.)
|
| ⊢ (𝐴 = 𝐵 → 〈𝐶, 𝐴〉 = 〈𝐶, 𝐵〉) |
| |
| Theorem | opeq12 3810 |
Equality theorem for ordered pairs. (Contributed by NM, 28-May-1995.)
|
| ⊢ ((𝐴 = 𝐶 ∧ 𝐵 = 𝐷) → 〈𝐴, 𝐵〉 = 〈𝐶, 𝐷〉) |
| |
| Theorem | opeq1i 3811 |
Equality inference for ordered pairs. (Contributed by NM,
16-Dec-2006.)
|
| ⊢ 𝐴 = 𝐵 ⇒ ⊢ 〈𝐴, 𝐶〉 = 〈𝐵, 𝐶〉 |
| |
| Theorem | opeq2i 3812 |
Equality inference for ordered pairs. (Contributed by NM,
16-Dec-2006.)
|
| ⊢ 𝐴 = 𝐵 ⇒ ⊢ 〈𝐶, 𝐴〉 = 〈𝐶, 𝐵〉 |
| |
| Theorem | opeq12i 3813 |
Equality inference for ordered pairs. (Contributed by NM,
16-Dec-2006.) (Proof shortened by Eric Schmidt, 4-Apr-2007.)
|
| ⊢ 𝐴 = 𝐵
& ⊢ 𝐶 = 𝐷 ⇒ ⊢ 〈𝐴, 𝐶〉 = 〈𝐵, 𝐷〉 |
| |
| Theorem | opeq1d 3814 |
Equality deduction for ordered pairs. (Contributed by NM,
16-Dec-2006.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → 〈𝐴, 𝐶〉 = 〈𝐵, 𝐶〉) |
| |
| Theorem | opeq2d 3815 |
Equality deduction for ordered pairs. (Contributed by NM,
16-Dec-2006.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → 〈𝐶, 𝐴〉 = 〈𝐶, 𝐵〉) |
| |
| Theorem | opeq12d 3816 |
Equality deduction for ordered pairs. (Contributed by NM, 16-Dec-2006.)
(Proof shortened by Andrew Salmon, 29-Jun-2011.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → 〈𝐴, 𝐶〉 = 〈𝐵, 𝐷〉) |
| |
| Theorem | oteq1 3817 |
Equality theorem for ordered triples. (Contributed by NM, 3-Apr-2015.)
|
| ⊢ (𝐴 = 𝐵 → 〈𝐴, 𝐶, 𝐷〉 = 〈𝐵, 𝐶, 𝐷〉) |
| |
| Theorem | oteq2 3818 |
Equality theorem for ordered triples. (Contributed by NM, 3-Apr-2015.)
|
| ⊢ (𝐴 = 𝐵 → 〈𝐶, 𝐴, 𝐷〉 = 〈𝐶, 𝐵, 𝐷〉) |
| |
| Theorem | oteq3 3819 |
Equality theorem for ordered triples. (Contributed by NM, 3-Apr-2015.)
|
| ⊢ (𝐴 = 𝐵 → 〈𝐶, 𝐷, 𝐴〉 = 〈𝐶, 𝐷, 𝐵〉) |
| |
| Theorem | oteq1d 3820 |
Equality deduction for ordered triples. (Contributed by Mario Carneiro,
11-Jan-2017.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → 〈𝐴, 𝐶, 𝐷〉 = 〈𝐵, 𝐶, 𝐷〉) |
| |
| Theorem | oteq2d 3821 |
Equality deduction for ordered triples. (Contributed by Mario Carneiro,
11-Jan-2017.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → 〈𝐶, 𝐴, 𝐷〉 = 〈𝐶, 𝐵, 𝐷〉) |
| |
| Theorem | oteq3d 3822 |
Equality deduction for ordered triples. (Contributed by Mario Carneiro,
11-Jan-2017.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → 〈𝐶, 𝐷, 𝐴〉 = 〈𝐶, 𝐷, 𝐵〉) |
| |
| Theorem | oteq123d 3823 |
Equality deduction for ordered triples. (Contributed by Mario Carneiro,
11-Jan-2017.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷)
& ⊢ (𝜑 → 𝐸 = 𝐹) ⇒ ⊢ (𝜑 → 〈𝐴, 𝐶, 𝐸〉 = 〈𝐵, 𝐷, 𝐹〉) |
| |
| Theorem | nfop 3824 |
Bound-variable hypothesis builder for ordered pairs. (Contributed by
NM, 14-Nov-1995.)
|
| ⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥〈𝐴, 𝐵〉 |
| |
| Theorem | nfopd 3825 |
Deduction version of bound-variable hypothesis builder nfop 3824.
This
shows how the deduction version of a not-free theorem such as nfop 3824
can
be created from the corresponding not-free inference theorem.
(Contributed by NM, 4-Feb-2008.)
|
| ⊢ (𝜑 → Ⅎ𝑥𝐴)
& ⊢ (𝜑 → Ⅎ𝑥𝐵) ⇒ ⊢ (𝜑 → Ⅎ𝑥〈𝐴, 𝐵〉) |
| |
| Theorem | opid 3826 |
The ordered pair 〈𝐴, 𝐴〉 in Kuratowski's
representation.
(Contributed by FL, 28-Dec-2011.)
|
| ⊢ 𝐴 ∈ V ⇒ ⊢ 〈𝐴, 𝐴〉 = {{𝐴}} |
| |
| Theorem | ralunsn 3827* |
Restricted quantification over the union of a set and a singleton, using
implicit substitution. (Contributed by Paul Chapman, 17-Nov-2012.)
(Revised by Mario Carneiro, 23-Apr-2015.)
|
| ⊢ (𝑥 = 𝐵 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (𝐵 ∈ 𝐶 → (∀𝑥 ∈ (𝐴 ∪ {𝐵})𝜑 ↔ (∀𝑥 ∈ 𝐴 𝜑 ∧ 𝜓))) |
| |
| Theorem | 2ralunsn 3828* |
Double restricted quantification over the union of a set and a
singleton, using implicit substitution. (Contributed by Paul Chapman,
17-Nov-2012.)
|
| ⊢ (𝑥 = 𝐵 → (𝜑 ↔ 𝜒)) & ⊢ (𝑦 = 𝐵 → (𝜑 ↔ 𝜓)) & ⊢ (𝑥 = 𝐵 → (𝜓 ↔ 𝜃)) ⇒ ⊢ (𝐵 ∈ 𝐶 → (∀𝑥 ∈ (𝐴 ∪ {𝐵})∀𝑦 ∈ (𝐴 ∪ {𝐵})𝜑 ↔ ((∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 𝜑 ∧ ∀𝑥 ∈ 𝐴 𝜓) ∧ (∀𝑦 ∈ 𝐴 𝜒 ∧ 𝜃)))) |
| |
| Theorem | opprc 3829 |
Expansion of an ordered pair when either member is a proper class.
(Contributed by Mario Carneiro, 26-Apr-2015.)
|
| ⊢ (¬ (𝐴 ∈ V ∧ 𝐵 ∈ V) → 〈𝐴, 𝐵〉 = ∅) |
| |
| Theorem | opprc1 3830 |
Expansion of an ordered pair when the first member is a proper class. See
also opprc 3829. (Contributed by NM, 10-Apr-2004.) (Revised
by Mario
Carneiro, 26-Apr-2015.)
|
| ⊢ (¬ 𝐴 ∈ V → 〈𝐴, 𝐵〉 = ∅) |
| |
| Theorem | opprc2 3831 |
Expansion of an ordered pair when the second member is a proper class.
See also opprc 3829. (Contributed by NM, 15-Nov-1994.) (Revised
by Mario
Carneiro, 26-Apr-2015.)
|
| ⊢ (¬ 𝐵 ∈ V → 〈𝐴, 𝐵〉 = ∅) |
| |
| Theorem | oprcl 3832 |
If an ordered pair has an element, then its arguments are sets.
(Contributed by Mario Carneiro, 26-Apr-2015.)
|
| ⊢ (𝐶 ∈ 〈𝐴, 𝐵〉 → (𝐴 ∈ V ∧ 𝐵 ∈ V)) |
| |
| Theorem | pwsnss 3833 |
The power set of a singleton. (Contributed by Jim Kingdon,
12-Aug-2018.)
|
| ⊢ {∅, {𝐴}} ⊆ 𝒫 {𝐴} |
| |
| Theorem | pwpw0ss 3834 |
Compute the power set of the power set of the empty set. (See pw0 3769
for
the power set of the empty set.) Theorem 90 of [Suppes] p. 48 (but with
subset in place of equality). (Contributed by Jim Kingdon,
12-Aug-2018.)
|
| ⊢ {∅, {∅}} ⊆ 𝒫
{∅} |
| |
| Theorem | pwprss 3835 |
The power set of an unordered pair. (Contributed by Jim Kingdon,
13-Aug-2018.)
|
| ⊢ ({∅, {𝐴}} ∪ {{𝐵}, {𝐴, 𝐵}}) ⊆ 𝒫 {𝐴, 𝐵} |
| |
| Theorem | pwtpss 3836 |
The power set of an unordered triple. (Contributed by Jim Kingdon,
13-Aug-2018.)
|
| ⊢ (({∅, {𝐴}} ∪ {{𝐵}, {𝐴, 𝐵}}) ∪ ({{𝐶}, {𝐴, 𝐶}} ∪ {{𝐵, 𝐶}, {𝐴, 𝐵, 𝐶}})) ⊆ 𝒫 {𝐴, 𝐵, 𝐶} |
| |
| Theorem | pwpwpw0ss 3837 |
Compute the power set of the power set of the power set of the empty set.
(See also pw0 3769 and pwpw0ss 3834.) (Contributed by Jim Kingdon,
13-Aug-2018.)
|
| ⊢ ({∅, {∅}} ∪ {{{∅}},
{∅, {∅}}}) ⊆ 𝒫 {∅, {∅}} |
| |
| Theorem | pwv 3838 |
The power class of the universe is the universe. Exercise 4.12(d) of
[Mendelson] p. 235. (Contributed by NM,
14-Sep-2003.)
|
| ⊢ 𝒫 V = V |
| |
| 2.1.18 The union of a class
|
| |
| Syntax | cuni 3839 |
Extend class notation to include the union of a class. Read: "union (of)
𝐴".
|
| class ∪ 𝐴 |
| |
| Definition | df-uni 3840* |
Define the union of a class i.e. the collection of all members of the
members of the class. Definition 5.5 of [TakeutiZaring] p. 16. For
example, ∪ {{1, 3}, {1, 8}}
= {1, 3, 8}. This is
similar to the union of two classes df-un 3161. (Contributed by NM,
23-Aug-1993.)
|
| ⊢ ∪ 𝐴 = {𝑥 ∣ ∃𝑦(𝑥 ∈ 𝑦 ∧ 𝑦 ∈ 𝐴)} |
| |
| Theorem | dfuni2 3841* |
Alternate definition of class union. (Contributed by NM,
28-Jun-1998.)
|
| ⊢ ∪ 𝐴 = {𝑥 ∣ ∃𝑦 ∈ 𝐴 𝑥 ∈ 𝑦} |
| |
| Theorem | eluni 3842* |
Membership in class union. (Contributed by NM, 22-May-1994.)
|
| ⊢ (𝐴 ∈ ∪ 𝐵 ↔ ∃𝑥(𝐴 ∈ 𝑥 ∧ 𝑥 ∈ 𝐵)) |
| |
| Theorem | eluni2 3843* |
Membership in class union. Restricted quantifier version. (Contributed
by NM, 31-Aug-1999.)
|
| ⊢ (𝐴 ∈ ∪ 𝐵 ↔ ∃𝑥 ∈ 𝐵 𝐴 ∈ 𝑥) |
| |
| Theorem | elunii 3844 |
Membership in class union. (Contributed by NM, 24-Mar-1995.)
|
| ⊢ ((𝐴 ∈ 𝐵 ∧ 𝐵 ∈ 𝐶) → 𝐴 ∈ ∪ 𝐶) |
| |
| Theorem | nfuni 3845 |
Bound-variable hypothesis builder for union. (Contributed by NM,
30-Dec-1996.) (Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
| ⊢ Ⅎ𝑥𝐴 ⇒ ⊢ Ⅎ𝑥∪
𝐴 |
| |
| Theorem | nfunid 3846 |
Deduction version of nfuni 3845. (Contributed by NM, 18-Feb-2013.)
|
| ⊢ (𝜑 → Ⅎ𝑥𝐴) ⇒ ⊢ (𝜑 → Ⅎ𝑥∪ 𝐴) |
| |
| Theorem | csbunig 3847 |
Distribute proper substitution through the union of a class.
(Contributed by Alan Sare, 10-Nov-2012.)
|
| ⊢ (𝐴 ∈ 𝑉 → ⦋𝐴 / 𝑥⦌∪
𝐵 = ∪ ⦋𝐴 / 𝑥⦌𝐵) |
| |
| Theorem | unieq 3848 |
Equality theorem for class union. Exercise 15 of [TakeutiZaring] p. 18.
(Contributed by NM, 10-Aug-1993.) (Proof shortened by Andrew Salmon,
29-Jun-2011.)
|
| ⊢ (𝐴 = 𝐵 → ∪ 𝐴 = ∪
𝐵) |
| |
| Theorem | unieqi 3849 |
Inference of equality of two class unions. (Contributed by NM,
30-Aug-1993.)
|
| ⊢ 𝐴 = 𝐵 ⇒ ⊢ ∪
𝐴 = ∪ 𝐵 |
| |
| Theorem | unieqd 3850 |
Deduction of equality of two class unions. (Contributed by NM,
21-Apr-1995.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → ∪ 𝐴 = ∪
𝐵) |
| |
| Theorem | eluniab 3851* |
Membership in union of a class abstraction. (Contributed by NM,
11-Aug-1994.) (Revised by Mario Carneiro, 14-Nov-2016.)
|
| ⊢ (𝐴 ∈ ∪ {𝑥 ∣ 𝜑} ↔ ∃𝑥(𝐴 ∈ 𝑥 ∧ 𝜑)) |
| |
| Theorem | elunirab 3852* |
Membership in union of a class abstraction. (Contributed by NM,
4-Oct-2006.)
|
| ⊢ (𝐴 ∈ ∪ {𝑥 ∈ 𝐵 ∣ 𝜑} ↔ ∃𝑥 ∈ 𝐵 (𝐴 ∈ 𝑥 ∧ 𝜑)) |
| |
| Theorem | unipr 3853 |
The union of a pair is the union of its members. Proposition 5.7 of
[TakeutiZaring] p. 16.
(Contributed by NM, 23-Aug-1993.)
|
| ⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ ∪
{𝐴, 𝐵} = (𝐴 ∪ 𝐵) |
| |
| Theorem | uniprg 3854 |
The union of a pair is the union of its members. Proposition 5.7 of
[TakeutiZaring] p. 16.
(Contributed by NM, 25-Aug-2006.)
|
| ⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → ∪
{𝐴, 𝐵} = (𝐴 ∪ 𝐵)) |
| |
| Theorem | unisn 3855 |
A set equals the union of its singleton. Theorem 8.2 of [Quine] p. 53.
(Contributed by NM, 30-Aug-1993.)
|
| ⊢ 𝐴 ∈ V ⇒ ⊢ ∪
{𝐴} = 𝐴 |
| |
| Theorem | unisng 3856 |
A set equals the union of its singleton. Theorem 8.2 of [Quine] p. 53.
(Contributed by NM, 13-Aug-2002.)
|
| ⊢ (𝐴 ∈ 𝑉 → ∪ {𝐴} = 𝐴) |
| |
| Theorem | dfnfc2 3857* |
An alternate statement of the effective freeness of a class 𝐴, when
it is a set. (Contributed by Mario Carneiro, 14-Oct-2016.)
|
| ⊢ (∀𝑥 𝐴 ∈ 𝑉 → (Ⅎ𝑥𝐴 ↔ ∀𝑦Ⅎ𝑥 𝑦 = 𝐴)) |
| |
| Theorem | uniun 3858 |
The class union of the union of two classes. Theorem 8.3 of [Quine]
p. 53. (Contributed by NM, 20-Aug-1993.)
|
| ⊢ ∪ (𝐴 ∪ 𝐵) = (∪ 𝐴 ∪ ∪ 𝐵) |
| |
| Theorem | uniin 3859 |
The class union of the intersection of two classes. Exercise 4.12(n) of
[Mendelson] p. 235. (Contributed by
NM, 4-Dec-2003.) (Proof shortened
by Andrew Salmon, 29-Jun-2011.)
|
| ⊢ ∪ (𝐴 ∩ 𝐵) ⊆ (∪
𝐴 ∩ ∪ 𝐵) |
| |
| Theorem | uniss 3860 |
Subclass relationship for class union. Theorem 61 of [Suppes] p. 39.
(Contributed by NM, 22-Mar-1998.) (Proof shortened by Andrew Salmon,
29-Jun-2011.)
|
| ⊢ (𝐴 ⊆ 𝐵 → ∪ 𝐴 ⊆ ∪ 𝐵) |
| |
| Theorem | ssuni 3861 |
Subclass relationship for class union. (Contributed by NM,
24-May-1994.) (Proof shortened by Andrew Salmon, 29-Jun-2011.)
|
| ⊢ ((𝐴 ⊆ 𝐵 ∧ 𝐵 ∈ 𝐶) → 𝐴 ⊆ ∪ 𝐶) |
| |
| Theorem | unissi 3862 |
Subclass relationship for subclass union. Inference form of uniss 3860.
(Contributed by David Moews, 1-May-2017.)
|
| ⊢ 𝐴 ⊆ 𝐵 ⇒ ⊢ ∪
𝐴 ⊆ ∪ 𝐵 |
| |
| Theorem | unissd 3863 |
Subclass relationship for subclass union. Deduction form of uniss 3860.
(Contributed by David Moews, 1-May-2017.)
|
| ⊢ (𝜑 → 𝐴 ⊆ 𝐵) ⇒ ⊢ (𝜑 → ∪ 𝐴 ⊆ ∪ 𝐵) |
| |
| Theorem | uni0b 3864 |
The union of a set is empty iff the set is included in the singleton of
the empty set. (Contributed by NM, 12-Sep-2004.)
|
| ⊢ (∪ 𝐴 = ∅ ↔ 𝐴 ⊆
{∅}) |
| |
| Theorem | uni0c 3865* |
The union of a set is empty iff all of its members are empty.
(Contributed by NM, 16-Aug-2006.)
|
| ⊢ (∪ 𝐴 = ∅ ↔ ∀𝑥 ∈ 𝐴 𝑥 = ∅) |
| |
| Theorem | uni0 3866 |
The union of the empty set is the empty set. Theorem 8.7 of [Quine]
p. 54. (Reproved without relying on ax-nul by Eric Schmidt.)
(Contributed by NM, 16-Sep-1993.) (Revised by Eric Schmidt,
4-Apr-2007.)
|
| ⊢ ∪ ∅ =
∅ |
| |
| Theorem | elssuni 3867 |
An element of a class is a subclass of its union. Theorem 8.6 of [Quine]
p. 54. Also the basis for Proposition 7.20 of [TakeutiZaring] p. 40.
(Contributed by NM, 6-Jun-1994.)
|
| ⊢ (𝐴 ∈ 𝐵 → 𝐴 ⊆ ∪ 𝐵) |
| |
| Theorem | unissel 3868 |
Condition turning a subclass relationship for union into an equality.
(Contributed by NM, 18-Jul-2006.)
|
| ⊢ ((∪ 𝐴 ⊆ 𝐵 ∧ 𝐵 ∈ 𝐴) → ∪ 𝐴 = 𝐵) |
| |
| Theorem | unissb 3869* |
Relationship involving membership, subset, and union. Exercise 5 of
[Enderton] p. 26 and its converse.
(Contributed by NM, 20-Sep-2003.)
|
| ⊢ (∪ 𝐴 ⊆ 𝐵 ↔ ∀𝑥 ∈ 𝐴 𝑥 ⊆ 𝐵) |
| |
| Theorem | uniss2 3870* |
A subclass condition on the members of two classes that implies a
subclass relation on their unions. Proposition 8.6 of [TakeutiZaring]
p. 59. (Contributed by NM, 22-Mar-2004.)
|
| ⊢ (∀𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝑥 ⊆ 𝑦 → ∪ 𝐴 ⊆ ∪ 𝐵) |
| |
| Theorem | unidif 3871* |
If the difference 𝐴 ∖ 𝐵 contains the largest members of
𝐴,
then
the union of the difference is the union of 𝐴. (Contributed by NM,
22-Mar-2004.)
|
| ⊢ (∀𝑥 ∈ 𝐴 ∃𝑦 ∈ (𝐴 ∖ 𝐵)𝑥 ⊆ 𝑦 → ∪ (𝐴 ∖ 𝐵) = ∪ 𝐴) |
| |
| Theorem | ssunieq 3872* |
Relationship implying union. (Contributed by NM, 10-Nov-1999.)
|
| ⊢ ((𝐴 ∈ 𝐵 ∧ ∀𝑥 ∈ 𝐵 𝑥 ⊆ 𝐴) → 𝐴 = ∪ 𝐵) |
| |
| Theorem | unimax 3873* |
Any member of a class is the largest of those members that it includes.
(Contributed by NM, 13-Aug-2002.)
|
| ⊢ (𝐴 ∈ 𝐵 → ∪ {𝑥 ∈ 𝐵 ∣ 𝑥 ⊆ 𝐴} = 𝐴) |
| |
| 2.1.19 The intersection of a class
|
| |
| Syntax | cint 3874 |
Extend class notation to include the intersection of a class. Read:
"intersection (of) 𝐴".
|
| class ∩ 𝐴 |
| |
| Definition | df-int 3875* |
Define the intersection of a class. Definition 7.35 of [TakeutiZaring]
p. 44. For example, ∩ {{1,
3}, {1, 8}} = {1}.
Compare this with the intersection of two classes, df-in 3163.
(Contributed by NM, 18-Aug-1993.)
|
| ⊢ ∩ 𝐴 = {𝑥 ∣ ∀𝑦(𝑦 ∈ 𝐴 → 𝑥 ∈ 𝑦)} |
| |
| Theorem | dfint2 3876* |
Alternate definition of class intersection. (Contributed by NM,
28-Jun-1998.)
|
| ⊢ ∩ 𝐴 = {𝑥 ∣ ∀𝑦 ∈ 𝐴 𝑥 ∈ 𝑦} |
| |
| Theorem | inteq 3877 |
Equality law for intersection. (Contributed by NM, 13-Sep-1999.)
|
| ⊢ (𝐴 = 𝐵 → ∩ 𝐴 = ∩
𝐵) |
| |
| Theorem | inteqi 3878 |
Equality inference for class intersection. (Contributed by NM,
2-Sep-2003.)
|
| ⊢ 𝐴 = 𝐵 ⇒ ⊢ ∩
𝐴 = ∩ 𝐵 |
| |
| Theorem | inteqd 3879 |
Equality deduction for class intersection. (Contributed by NM,
2-Sep-2003.)
|
| ⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → ∩ 𝐴 = ∩
𝐵) |
| |
| Theorem | elint 3880* |
Membership in class intersection. (Contributed by NM, 21-May-1994.)
|
| ⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ ∩ 𝐵 ↔ ∀𝑥(𝑥 ∈ 𝐵 → 𝐴 ∈ 𝑥)) |
| |
| Theorem | elint2 3881* |
Membership in class intersection. (Contributed by NM, 14-Oct-1999.)
|
| ⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ ∩ 𝐵 ↔ ∀𝑥 ∈ 𝐵 𝐴 ∈ 𝑥) |
| |
| Theorem | elintg 3882* |
Membership in class intersection, with the sethood requirement expressed
as an antecedent. (Contributed by NM, 20-Nov-2003.)
|
| ⊢ (𝐴 ∈ 𝑉 → (𝐴 ∈ ∩ 𝐵 ↔ ∀𝑥 ∈ 𝐵 𝐴 ∈ 𝑥)) |
| |
| Theorem | elinti 3883 |
Membership in class intersection. (Contributed by NM, 14-Oct-1999.)
(Proof shortened by Andrew Salmon, 9-Jul-2011.)
|
| ⊢ (𝐴 ∈ ∩ 𝐵 → (𝐶 ∈ 𝐵 → 𝐴 ∈ 𝐶)) |
| |
| Theorem | nfint 3884 |
Bound-variable hypothesis builder for intersection. (Contributed by NM,
2-Feb-1997.) (Proof shortened by Andrew Salmon, 12-Aug-2011.)
|
| ⊢ Ⅎ𝑥𝐴 ⇒ ⊢ Ⅎ𝑥∩
𝐴 |
| |
| Theorem | elintab 3885* |
Membership in the intersection of a class abstraction. (Contributed by
NM, 30-Aug-1993.)
|
| ⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ ∩ {𝑥 ∣ 𝜑} ↔ ∀𝑥(𝜑 → 𝐴 ∈ 𝑥)) |
| |
| Theorem | elintrab 3886* |
Membership in the intersection of a class abstraction. (Contributed by
NM, 17-Oct-1999.)
|
| ⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ ∩ {𝑥 ∈ 𝐵 ∣ 𝜑} ↔ ∀𝑥 ∈ 𝐵 (𝜑 → 𝐴 ∈ 𝑥)) |
| |
| Theorem | elintrabg 3887* |
Membership in the intersection of a class abstraction. (Contributed by
NM, 17-Feb-2007.)
|
| ⊢ (𝐴 ∈ 𝑉 → (𝐴 ∈ ∩ {𝑥 ∈ 𝐵 ∣ 𝜑} ↔ ∀𝑥 ∈ 𝐵 (𝜑 → 𝐴 ∈ 𝑥))) |
| |
| Theorem | int0 3888 |
The intersection of the empty set is the universal class. Exercise 2 of
[TakeutiZaring] p. 44.
(Contributed by NM, 18-Aug-1993.)
|
| ⊢ ∩ ∅ =
V |
| |
| Theorem | intss1 3889 |
An element of a class includes the intersection of the class. Exercise
4 of [TakeutiZaring] p. 44 (with
correction), generalized to classes.
(Contributed by NM, 18-Nov-1995.)
|
| ⊢ (𝐴 ∈ 𝐵 → ∩ 𝐵 ⊆ 𝐴) |
| |
| Theorem | ssint 3890* |
Subclass of a class intersection. Theorem 5.11(viii) of [Monk1] p. 52
and its converse. (Contributed by NM, 14-Oct-1999.)
|
| ⊢ (𝐴 ⊆ ∩ 𝐵 ↔ ∀𝑥 ∈ 𝐵 𝐴 ⊆ 𝑥) |
| |
| Theorem | ssintab 3891* |
Subclass of the intersection of a class abstraction. (Contributed by
NM, 31-Jul-2006.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
|
| ⊢ (𝐴 ⊆ ∩
{𝑥 ∣ 𝜑} ↔ ∀𝑥(𝜑 → 𝐴 ⊆ 𝑥)) |
| |
| Theorem | ssintub 3892* |
Subclass of the least upper bound. (Contributed by NM, 8-Aug-2000.)
|
| ⊢ 𝐴 ⊆ ∩
{𝑥 ∈ 𝐵 ∣ 𝐴 ⊆ 𝑥} |
| |
| Theorem | ssmin 3893* |
Subclass of the minimum value of class of supersets. (Contributed by
NM, 10-Aug-2006.)
|
| ⊢ 𝐴 ⊆ ∩
{𝑥 ∣ (𝐴 ⊆ 𝑥 ∧ 𝜑)} |
| |
| Theorem | intmin 3894* |
Any member of a class is the smallest of those members that include it.
(Contributed by NM, 13-Aug-2002.) (Proof shortened by Andrew Salmon,
9-Jul-2011.)
|
| ⊢ (𝐴 ∈ 𝐵 → ∩ {𝑥 ∈ 𝐵 ∣ 𝐴 ⊆ 𝑥} = 𝐴) |
| |
| Theorem | intss 3895 |
Intersection of subclasses. (Contributed by NM, 14-Oct-1999.)
|
| ⊢ (𝐴 ⊆ 𝐵 → ∩ 𝐵 ⊆ ∩ 𝐴) |
| |
| Theorem | intssunim 3896* |
The intersection of an inhabited set is a subclass of its union.
(Contributed by NM, 29-Jul-2006.)
|
| ⊢ (∃𝑥 𝑥 ∈ 𝐴 → ∩ 𝐴 ⊆ ∪ 𝐴) |
| |
| Theorem | ssintrab 3897* |
Subclass of the intersection of a restricted class builder.
(Contributed by NM, 30-Jan-2015.)
|
| ⊢ (𝐴 ⊆ ∩
{𝑥 ∈ 𝐵 ∣ 𝜑} ↔ ∀𝑥 ∈ 𝐵 (𝜑 → 𝐴 ⊆ 𝑥)) |
| |
| Theorem | intssuni2m 3898* |
Subclass relationship for intersection and union. (Contributed by Jim
Kingdon, 14-Aug-2018.)
|
| ⊢ ((𝐴 ⊆ 𝐵 ∧ ∃𝑥 𝑥 ∈ 𝐴) → ∩ 𝐴 ⊆ ∪ 𝐵) |
| |
| Theorem | intminss 3899* |
Under subset ordering, the intersection of a restricted class
abstraction is less than or equal to any of its members. (Contributed
by NM, 7-Sep-2013.)
|
| ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜓)) ⇒ ⊢ ((𝐴 ∈ 𝐵 ∧ 𝜓) → ∩
{𝑥 ∈ 𝐵 ∣ 𝜑} ⊆ 𝐴) |
| |
| Theorem | intmin2 3900* |
Any set is the smallest of all sets that include it. (Contributed by
NM, 20-Sep-2003.)
|
| ⊢ 𝐴 ∈ V ⇒ ⊢ ∩
{𝑥 ∣ 𝐴 ⊆ 𝑥} = 𝐴 |