Theorem List for Intuitionistic Logic Explorer - 3301-3400 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
2.1.13.2 The union of two classes
|
|
Theorem | elun 3301 |
Expansion of membership in class union. Theorem 12 of [Suppes] p. 25.
(Contributed by NM, 7-Aug-1994.)
|
⊢ (𝐴 ∈ (𝐵 ∪ 𝐶) ↔ (𝐴 ∈ 𝐵 ∨ 𝐴 ∈ 𝐶)) |
|
Theorem | uneqri 3302* |
Inference from membership to union. (Contributed by NM, 5-Aug-1993.)
|
⊢ ((𝑥 ∈ 𝐴 ∨ 𝑥 ∈ 𝐵) ↔ 𝑥 ∈ 𝐶) ⇒ ⊢ (𝐴 ∪ 𝐵) = 𝐶 |
|
Theorem | unidm 3303 |
Idempotent law for union of classes. Theorem 23 of [Suppes] p. 27.
(Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∪ 𝐴) = 𝐴 |
|
Theorem | uncom 3304 |
Commutative law for union of classes. Exercise 6 of [TakeutiZaring]
p. 17. (Contributed by NM, 25-Jun-1998.) (Proof shortened by Andrew
Salmon, 26-Jun-2011.)
|
⊢ (𝐴 ∪ 𝐵) = (𝐵 ∪ 𝐴) |
|
Theorem | equncom 3305 |
If a class equals the union of two other classes, then it equals the union
of those two classes commuted. (Contributed by Alan Sare,
18-Feb-2012.)
|
⊢ (𝐴 = (𝐵 ∪ 𝐶) ↔ 𝐴 = (𝐶 ∪ 𝐵)) |
|
Theorem | equncomi 3306 |
Inference form of equncom 3305. (Contributed by Alan Sare,
18-Feb-2012.)
|
⊢ 𝐴 = (𝐵 ∪ 𝐶) ⇒ ⊢ 𝐴 = (𝐶 ∪ 𝐵) |
|
Theorem | uneq1 3307 |
Equality theorem for union of two classes. (Contributed by NM,
5-Aug-1993.)
|
⊢ (𝐴 = 𝐵 → (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐶)) |
|
Theorem | uneq2 3308 |
Equality theorem for the union of two classes. (Contributed by NM,
5-Aug-1993.)
|
⊢ (𝐴 = 𝐵 → (𝐶 ∪ 𝐴) = (𝐶 ∪ 𝐵)) |
|
Theorem | uneq12 3309 |
Equality theorem for union of two classes. (Contributed by NM,
29-Mar-1998.)
|
⊢ ((𝐴 = 𝐵 ∧ 𝐶 = 𝐷) → (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐷)) |
|
Theorem | uneq1i 3310 |
Inference adding union to the right in a class equality. (Contributed
by NM, 30-Aug-1993.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐶) |
|
Theorem | uneq2i 3311 |
Inference adding union to the left in a class equality. (Contributed by
NM, 30-Aug-1993.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐶 ∪ 𝐴) = (𝐶 ∪ 𝐵) |
|
Theorem | uneq12i 3312 |
Equality inference for union of two classes. (Contributed by NM,
12-Aug-2004.) (Proof shortened by Eric Schmidt, 26-Jan-2007.)
|
⊢ 𝐴 = 𝐵
& ⊢ 𝐶 = 𝐷 ⇒ ⊢ (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐷) |
|
Theorem | uneq1d 3313 |
Deduction adding union to the right in a class equality. (Contributed
by NM, 29-Mar-1998.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐶)) |
|
Theorem | uneq2d 3314 |
Deduction adding union to the left in a class equality. (Contributed by
NM, 29-Mar-1998.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐶 ∪ 𝐴) = (𝐶 ∪ 𝐵)) |
|
Theorem | uneq12d 3315 |
Equality deduction for union of two classes. (Contributed by NM,
29-Sep-2004.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐷)) |
|
Theorem | nfun 3316 |
Bound-variable hypothesis builder for the union of classes.
(Contributed by NM, 15-Sep-2003.) (Revised by Mario Carneiro,
14-Oct-2016.)
|
⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥(𝐴 ∪ 𝐵) |
|
Theorem | unass 3317 |
Associative law for union of classes. Exercise 8 of [TakeutiZaring]
p. 17. (Contributed by NM, 3-May-1994.) (Proof shortened by Andrew
Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ∪ 𝐵) ∪ 𝐶) = (𝐴 ∪ (𝐵 ∪ 𝐶)) |
|
Theorem | un12 3318 |
A rearrangement of union. (Contributed by NM, 12-Aug-2004.)
|
⊢ (𝐴 ∪ (𝐵 ∪ 𝐶)) = (𝐵 ∪ (𝐴 ∪ 𝐶)) |
|
Theorem | un23 3319 |
A rearrangement of union. (Contributed by NM, 12-Aug-2004.) (Proof
shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ∪ 𝐵) ∪ 𝐶) = ((𝐴 ∪ 𝐶) ∪ 𝐵) |
|
Theorem | un4 3320 |
A rearrangement of the union of 4 classes. (Contributed by NM,
12-Aug-2004.)
|
⊢ ((𝐴 ∪ 𝐵) ∪ (𝐶 ∪ 𝐷)) = ((𝐴 ∪ 𝐶) ∪ (𝐵 ∪ 𝐷)) |
|
Theorem | unundi 3321 |
Union distributes over itself. (Contributed by NM, 17-Aug-2004.)
|
⊢ (𝐴 ∪ (𝐵 ∪ 𝐶)) = ((𝐴 ∪ 𝐵) ∪ (𝐴 ∪ 𝐶)) |
|
Theorem | unundir 3322 |
Union distributes over itself. (Contributed by NM, 17-Aug-2004.)
|
⊢ ((𝐴 ∪ 𝐵) ∪ 𝐶) = ((𝐴 ∪ 𝐶) ∪ (𝐵 ∪ 𝐶)) |
|
Theorem | ssun1 3323 |
Subclass relationship for union of classes. Theorem 25 of [Suppes]
p. 27. (Contributed by NM, 5-Aug-1993.)
|
⊢ 𝐴 ⊆ (𝐴 ∪ 𝐵) |
|
Theorem | ssun2 3324 |
Subclass relationship for union of classes. (Contributed by NM,
30-Aug-1993.)
|
⊢ 𝐴 ⊆ (𝐵 ∪ 𝐴) |
|
Theorem | ssun3 3325 |
Subclass law for union of classes. (Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ⊆ 𝐵 → 𝐴 ⊆ (𝐵 ∪ 𝐶)) |
|
Theorem | ssun4 3326 |
Subclass law for union of classes. (Contributed by NM, 14-Aug-1994.)
|
⊢ (𝐴 ⊆ 𝐵 → 𝐴 ⊆ (𝐶 ∪ 𝐵)) |
|
Theorem | elun1 3327 |
Membership law for union of classes. (Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∈ 𝐵 → 𝐴 ∈ (𝐵 ∪ 𝐶)) |
|
Theorem | elun2 3328 |
Membership law for union of classes. (Contributed by NM, 30-Aug-1993.)
|
⊢ (𝐴 ∈ 𝐵 → 𝐴 ∈ (𝐶 ∪ 𝐵)) |
|
Theorem | unss1 3329 |
Subclass law for union of classes. (Contributed by NM, 14-Oct-1999.)
(Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐴 ∪ 𝐶) ⊆ (𝐵 ∪ 𝐶)) |
|
Theorem | ssequn1 3330 |
A relationship between subclass and union. Theorem 26 of [Suppes]
p. 27. (Contributed by NM, 30-Aug-1993.) (Proof shortened by Andrew
Salmon, 26-Jun-2011.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ (𝐴 ∪ 𝐵) = 𝐵) |
|
Theorem | unss2 3331 |
Subclass law for union of classes. Exercise 7 of [TakeutiZaring] p. 18.
(Contributed by NM, 14-Oct-1999.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐶 ∪ 𝐴) ⊆ (𝐶 ∪ 𝐵)) |
|
Theorem | unss12 3332 |
Subclass law for union of classes. (Contributed by NM, 2-Jun-2004.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ 𝐶 ⊆ 𝐷) → (𝐴 ∪ 𝐶) ⊆ (𝐵 ∪ 𝐷)) |
|
Theorem | ssequn2 3333 |
A relationship between subclass and union. (Contributed by NM,
13-Jun-1994.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ (𝐵 ∪ 𝐴) = 𝐵) |
|
Theorem | unss 3334 |
The union of two subclasses is a subclass. Theorem 27 of [Suppes] p. 27
and its converse. (Contributed by NM, 11-Jun-2004.)
|
⊢ ((𝐴 ⊆ 𝐶 ∧ 𝐵 ⊆ 𝐶) ↔ (𝐴 ∪ 𝐵) ⊆ 𝐶) |
|
Theorem | unssi 3335 |
An inference showing the union of two subclasses is a subclass.
(Contributed by Raph Levien, 10-Dec-2002.)
|
⊢ 𝐴 ⊆ 𝐶
& ⊢ 𝐵 ⊆ 𝐶 ⇒ ⊢ (𝐴 ∪ 𝐵) ⊆ 𝐶 |
|
Theorem | unssd 3336 |
A deduction showing the union of two subclasses is a subclass.
(Contributed by Jonathan Ben-Naim, 3-Jun-2011.)
|
⊢ (𝜑 → 𝐴 ⊆ 𝐶)
& ⊢ (𝜑 → 𝐵 ⊆ 𝐶) ⇒ ⊢ (𝜑 → (𝐴 ∪ 𝐵) ⊆ 𝐶) |
|
Theorem | unssad 3337 |
If (𝐴
∪ 𝐵) is
contained in 𝐶, so is 𝐴. One-way
deduction form of unss 3334. Partial converse of unssd 3336. (Contributed
by David Moews, 1-May-2017.)
|
⊢ (𝜑 → (𝐴 ∪ 𝐵) ⊆ 𝐶) ⇒ ⊢ (𝜑 → 𝐴 ⊆ 𝐶) |
|
Theorem | unssbd 3338 |
If (𝐴
∪ 𝐵) is
contained in 𝐶, so is 𝐵. One-way
deduction form of unss 3334. Partial converse of unssd 3336. (Contributed
by David Moews, 1-May-2017.)
|
⊢ (𝜑 → (𝐴 ∪ 𝐵) ⊆ 𝐶) ⇒ ⊢ (𝜑 → 𝐵 ⊆ 𝐶) |
|
Theorem | ssun 3339 |
A condition that implies inclusion in the union of two classes.
(Contributed by NM, 23-Nov-2003.)
|
⊢ ((𝐴 ⊆ 𝐵 ∨ 𝐴 ⊆ 𝐶) → 𝐴 ⊆ (𝐵 ∪ 𝐶)) |
|
Theorem | rexun 3340 |
Restricted existential quantification over union. (Contributed by Jeff
Madsen, 5-Jan-2011.)
|
⊢ (∃𝑥 ∈ (𝐴 ∪ 𝐵)𝜑 ↔ (∃𝑥 ∈ 𝐴 𝜑 ∨ ∃𝑥 ∈ 𝐵 𝜑)) |
|
Theorem | ralunb 3341 |
Restricted quantification over a union. (Contributed by Scott Fenton,
12-Apr-2011.) (Proof shortened by Andrew Salmon, 29-Jun-2011.)
|
⊢ (∀𝑥 ∈ (𝐴 ∪ 𝐵)𝜑 ↔ (∀𝑥 ∈ 𝐴 𝜑 ∧ ∀𝑥 ∈ 𝐵 𝜑)) |
|
Theorem | ralun 3342 |
Restricted quantification over union. (Contributed by Jeff Madsen,
2-Sep-2009.)
|
⊢ ((∀𝑥 ∈ 𝐴 𝜑 ∧ ∀𝑥 ∈ 𝐵 𝜑) → ∀𝑥 ∈ (𝐴 ∪ 𝐵)𝜑) |
|
2.1.13.3 The intersection of two
classes
|
|
Theorem | elin 3343 |
Expansion of membership in an intersection of two classes. Theorem 12
of [Suppes] p. 25. (Contributed by NM,
29-Apr-1994.)
|
⊢ (𝐴 ∈ (𝐵 ∩ 𝐶) ↔ (𝐴 ∈ 𝐵 ∧ 𝐴 ∈ 𝐶)) |
|
Theorem | elini 3344 |
Membership in an intersection of two classes. (Contributed by Glauco
Siliprandi, 17-Aug-2020.)
|
⊢ 𝐴 ∈ 𝐵
& ⊢ 𝐴 ∈ 𝐶 ⇒ ⊢ 𝐴 ∈ (𝐵 ∩ 𝐶) |
|
Theorem | elind 3345 |
Deduce membership in an intersection of two classes. (Contributed by
Jonathan Ben-Naim, 3-Jun-2011.)
|
⊢ (𝜑 → 𝑋 ∈ 𝐴)
& ⊢ (𝜑 → 𝑋 ∈ 𝐵) ⇒ ⊢ (𝜑 → 𝑋 ∈ (𝐴 ∩ 𝐵)) |
|
Theorem | elinel1 3346 |
Membership in an intersection implies membership in the first set.
(Contributed by Glauco Siliprandi, 11-Dec-2019.)
|
⊢ (𝐴 ∈ (𝐵 ∩ 𝐶) → 𝐴 ∈ 𝐵) |
|
Theorem | elinel2 3347 |
Membership in an intersection implies membership in the second set.
(Contributed by Glauco Siliprandi, 11-Dec-2019.)
|
⊢ (𝐴 ∈ (𝐵 ∩ 𝐶) → 𝐴 ∈ 𝐶) |
|
Theorem | elin2 3348 |
Membership in a class defined as an intersection. (Contributed by
Stefan O'Rear, 29-Mar-2015.)
|
⊢ 𝑋 = (𝐵 ∩ 𝐶) ⇒ ⊢ (𝐴 ∈ 𝑋 ↔ (𝐴 ∈ 𝐵 ∧ 𝐴 ∈ 𝐶)) |
|
Theorem | elin1d 3349 |
Elementhood in the first set of an intersection - deduction version.
(Contributed by Thierry Arnoux, 3-May-2020.)
|
⊢ (𝜑 → 𝑋 ∈ (𝐴 ∩ 𝐵)) ⇒ ⊢ (𝜑 → 𝑋 ∈ 𝐴) |
|
Theorem | elin2d 3350 |
Elementhood in the first set of an intersection - deduction version.
(Contributed by Thierry Arnoux, 3-May-2020.)
|
⊢ (𝜑 → 𝑋 ∈ (𝐴 ∩ 𝐵)) ⇒ ⊢ (𝜑 → 𝑋 ∈ 𝐵) |
|
Theorem | elin3 3351 |
Membership in a class defined as a ternary intersection. (Contributed
by Stefan O'Rear, 29-Mar-2015.)
|
⊢ 𝑋 = ((𝐵 ∩ 𝐶) ∩ 𝐷) ⇒ ⊢ (𝐴 ∈ 𝑋 ↔ (𝐴 ∈ 𝐵 ∧ 𝐴 ∈ 𝐶 ∧ 𝐴 ∈ 𝐷)) |
|
Theorem | incom 3352 |
Commutative law for intersection of classes. Exercise 7 of
[TakeutiZaring] p. 17.
(Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∩ 𝐵) = (𝐵 ∩ 𝐴) |
|
Theorem | ineqri 3353* |
Inference from membership to intersection. (Contributed by NM,
5-Aug-1993.)
|
⊢ ((𝑥 ∈ 𝐴 ∧ 𝑥 ∈ 𝐵) ↔ 𝑥 ∈ 𝐶) ⇒ ⊢ (𝐴 ∩ 𝐵) = 𝐶 |
|
Theorem | ineq1 3354 |
Equality theorem for intersection of two classes. (Contributed by NM,
14-Dec-1993.)
|
⊢ (𝐴 = 𝐵 → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐶)) |
|
Theorem | ineq2 3355 |
Equality theorem for intersection of two classes. (Contributed by NM,
26-Dec-1993.)
|
⊢ (𝐴 = 𝐵 → (𝐶 ∩ 𝐴) = (𝐶 ∩ 𝐵)) |
|
Theorem | ineq12 3356 |
Equality theorem for intersection of two classes. (Contributed by NM,
8-May-1994.)
|
⊢ ((𝐴 = 𝐵 ∧ 𝐶 = 𝐷) → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐷)) |
|
Theorem | ineq1i 3357 |
Equality inference for intersection of two classes. (Contributed by NM,
26-Dec-1993.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐶) |
|
Theorem | ineq2i 3358 |
Equality inference for intersection of two classes. (Contributed by NM,
26-Dec-1993.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐶 ∩ 𝐴) = (𝐶 ∩ 𝐵) |
|
Theorem | ineq12i 3359 |
Equality inference for intersection of two classes. (Contributed by
NM, 24-Jun-2004.) (Proof shortened by Eric Schmidt, 26-Jan-2007.)
|
⊢ 𝐴 = 𝐵
& ⊢ 𝐶 = 𝐷 ⇒ ⊢ (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐷) |
|
Theorem | ineq1d 3360 |
Equality deduction for intersection of two classes. (Contributed by NM,
10-Apr-1994.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐶)) |
|
Theorem | ineq2d 3361 |
Equality deduction for intersection of two classes. (Contributed by NM,
10-Apr-1994.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐶 ∩ 𝐴) = (𝐶 ∩ 𝐵)) |
|
Theorem | ineq12d 3362 |
Equality deduction for intersection of two classes. (Contributed by
NM, 24-Jun-2004.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐷)) |
|
Theorem | ineqan12d 3363 |
Equality deduction for intersection of two classes. (Contributed by
NM, 7-Feb-2007.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜓 → 𝐶 = 𝐷) ⇒ ⊢ ((𝜑 ∧ 𝜓) → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐷)) |
|
Theorem | dfss1 3364 |
A frequently-used variant of subclass definition df-ss 3167. (Contributed
by NM, 10-Jan-2015.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ (𝐵 ∩ 𝐴) = 𝐴) |
|
Theorem | dfss5 3365 |
Another definition of subclasshood. Similar to df-ss 3167, dfss 3168, and
dfss1 3364. (Contributed by David Moews, 1-May-2017.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ 𝐴 = (𝐵 ∩ 𝐴)) |
|
Theorem | nfin 3366 |
Bound-variable hypothesis builder for the intersection of classes.
(Contributed by NM, 15-Sep-2003.) (Revised by Mario Carneiro,
14-Oct-2016.)
|
⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥(𝐴 ∩ 𝐵) |
|
Theorem | csbing 3367 |
Distribute proper substitution through an intersection relation.
(Contributed by Alan Sare, 22-Jul-2012.)
|
⊢ (𝐴 ∈ 𝐵 → ⦋𝐴 / 𝑥⦌(𝐶 ∩ 𝐷) = (⦋𝐴 / 𝑥⦌𝐶 ∩ ⦋𝐴 / 𝑥⦌𝐷)) |
|
Theorem | rabbi2dva 3368* |
Deduction from a wff to a restricted class abstraction. (Contributed by
NM, 14-Jan-2014.)
|
⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝑥 ∈ 𝐵 ↔ 𝜓)) ⇒ ⊢ (𝜑 → (𝐴 ∩ 𝐵) = {𝑥 ∈ 𝐴 ∣ 𝜓}) |
|
Theorem | inidm 3369 |
Idempotent law for intersection of classes. Theorem 15 of [Suppes]
p. 26. (Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∩ 𝐴) = 𝐴 |
|
Theorem | inass 3370 |
Associative law for intersection of classes. Exercise 9 of
[TakeutiZaring] p. 17.
(Contributed by NM, 3-May-1994.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = (𝐴 ∩ (𝐵 ∩ 𝐶)) |
|
Theorem | in12 3371 |
A rearrangement of intersection. (Contributed by NM, 21-Apr-2001.)
|
⊢ (𝐴 ∩ (𝐵 ∩ 𝐶)) = (𝐵 ∩ (𝐴 ∩ 𝐶)) |
|
Theorem | in32 3372 |
A rearrangement of intersection. (Contributed by NM, 21-Apr-2001.)
(Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = ((𝐴 ∩ 𝐶) ∩ 𝐵) |
|
Theorem | in13 3373 |
A rearrangement of intersection. (Contributed by NM, 27-Aug-2012.)
|
⊢ (𝐴 ∩ (𝐵 ∩ 𝐶)) = (𝐶 ∩ (𝐵 ∩ 𝐴)) |
|
Theorem | in31 3374 |
A rearrangement of intersection. (Contributed by NM, 27-Aug-2012.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = ((𝐶 ∩ 𝐵) ∩ 𝐴) |
|
Theorem | inrot 3375 |
Rotate the intersection of 3 classes. (Contributed by NM,
27-Aug-2012.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = ((𝐶 ∩ 𝐴) ∩ 𝐵) |
|
Theorem | in4 3376 |
Rearrangement of intersection of 4 classes. (Contributed by NM,
21-Apr-2001.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ (𝐶 ∩ 𝐷)) = ((𝐴 ∩ 𝐶) ∩ (𝐵 ∩ 𝐷)) |
|
Theorem | inindi 3377 |
Intersection distributes over itself. (Contributed by NM, 6-May-1994.)
|
⊢ (𝐴 ∩ (𝐵 ∩ 𝐶)) = ((𝐴 ∩ 𝐵) ∩ (𝐴 ∩ 𝐶)) |
|
Theorem | inindir 3378 |
Intersection distributes over itself. (Contributed by NM,
17-Aug-2004.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = ((𝐴 ∩ 𝐶) ∩ (𝐵 ∩ 𝐶)) |
|
Theorem | sseqin2 3379 |
A relationship between subclass and intersection. Similar to Exercise 9
of [TakeutiZaring] p. 18.
(Contributed by NM, 17-May-1994.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ (𝐵 ∩ 𝐴) = 𝐴) |
|
Theorem | inss1 3380 |
The intersection of two classes is a subset of one of them. Part of
Exercise 12 of [TakeutiZaring] p.
18. (Contributed by NM,
27-Apr-1994.)
|
⊢ (𝐴 ∩ 𝐵) ⊆ 𝐴 |
|
Theorem | inss2 3381 |
The intersection of two classes is a subset of one of them. Part of
Exercise 12 of [TakeutiZaring] p.
18. (Contributed by NM,
27-Apr-1994.)
|
⊢ (𝐴 ∩ 𝐵) ⊆ 𝐵 |
|
Theorem | ssin 3382 |
Subclass of intersection. Theorem 2.8(vii) of [Monk1] p. 26.
(Contributed by NM, 15-Jun-2004.) (Proof shortened by Andrew Salmon,
26-Jun-2011.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ 𝐴 ⊆ 𝐶) ↔ 𝐴 ⊆ (𝐵 ∩ 𝐶)) |
|
Theorem | ssini 3383 |
An inference showing that a subclass of two classes is a subclass of
their intersection. (Contributed by NM, 24-Nov-2003.)
|
⊢ 𝐴 ⊆ 𝐵
& ⊢ 𝐴 ⊆ 𝐶 ⇒ ⊢ 𝐴 ⊆ (𝐵 ∩ 𝐶) |
|
Theorem | ssind 3384 |
A deduction showing that a subclass of two classes is a subclass of
their intersection. (Contributed by Jonathan Ben-Naim, 3-Jun-2011.)
|
⊢ (𝜑 → 𝐴 ⊆ 𝐵)
& ⊢ (𝜑 → 𝐴 ⊆ 𝐶) ⇒ ⊢ (𝜑 → 𝐴 ⊆ (𝐵 ∩ 𝐶)) |
|
Theorem | ssrin 3385 |
Add right intersection to subclass relation. (Contributed by NM,
16-Aug-1994.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐴 ∩ 𝐶) ⊆ (𝐵 ∩ 𝐶)) |
|
Theorem | sslin 3386 |
Add left intersection to subclass relation. (Contributed by NM,
19-Oct-1999.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐶 ∩ 𝐴) ⊆ (𝐶 ∩ 𝐵)) |
|
Theorem | ssrind 3387 |
Add right intersection to subclass relation. (Contributed by Glauco
Siliprandi, 2-Jan-2022.)
|
⊢ (𝜑 → 𝐴 ⊆ 𝐵) ⇒ ⊢ (𝜑 → (𝐴 ∩ 𝐶) ⊆ (𝐵 ∩ 𝐶)) |
|
Theorem | ss2in 3388 |
Intersection of subclasses. (Contributed by NM, 5-May-2000.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ 𝐶 ⊆ 𝐷) → (𝐴 ∩ 𝐶) ⊆ (𝐵 ∩ 𝐷)) |
|
Theorem | ssinss1 3389 |
Intersection preserves subclass relationship. (Contributed by NM,
14-Sep-1999.)
|
⊢ (𝐴 ⊆ 𝐶 → (𝐴 ∩ 𝐵) ⊆ 𝐶) |
|
Theorem | inss 3390 |
Inclusion of an intersection of two classes. (Contributed by NM,
30-Oct-2014.)
|
⊢ ((𝐴 ⊆ 𝐶 ∨ 𝐵 ⊆ 𝐶) → (𝐴 ∩ 𝐵) ⊆ 𝐶) |
|
2.1.13.4 Combinations of difference, union, and
intersection of two classes
|
|
Theorem | unabs 3391 |
Absorption law for union. (Contributed by NM, 16-Apr-2006.)
|
⊢ (𝐴 ∪ (𝐴 ∩ 𝐵)) = 𝐴 |
|
Theorem | inabs 3392 |
Absorption law for intersection. (Contributed by NM, 16-Apr-2006.)
|
⊢ (𝐴 ∩ (𝐴 ∪ 𝐵)) = 𝐴 |
|
Theorem | dfss4st 3393* |
Subclass defined in terms of class difference. (Contributed by NM,
22-Mar-1998.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (∀𝑥STAB 𝑥 ∈ 𝐴 → (𝐴 ⊆ 𝐵 ↔ (𝐵 ∖ (𝐵 ∖ 𝐴)) = 𝐴)) |
|
Theorem | ssddif 3394 |
Double complement and subset. Similar to ddifss 3398 but inside a class
𝐵 instead of the universal class V. In classical logic the
subset operation on the right hand side could be an equality (that is,
𝐴
⊆ 𝐵 ↔ (𝐵 ∖ (𝐵 ∖ 𝐴)) = 𝐴). (Contributed by Jim Kingdon,
24-Jul-2018.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ 𝐴 ⊆ (𝐵 ∖ (𝐵 ∖ 𝐴))) |
|
Theorem | unssdif 3395 |
Union of two classes and class difference. In classical logic this
would be an equality. (Contributed by Jim Kingdon, 24-Jul-2018.)
|
⊢ (𝐴 ∪ 𝐵) ⊆ (V ∖ ((V ∖ 𝐴) ∖ 𝐵)) |
|
Theorem | inssdif 3396 |
Intersection of two classes and class difference. In classical logic
this would be an equality. (Contributed by Jim Kingdon,
24-Jul-2018.)
|
⊢ (𝐴 ∩ 𝐵) ⊆ (𝐴 ∖ (V ∖ 𝐵)) |
|
Theorem | difin 3397 |
Difference with intersection. Theorem 33 of [Suppes] p. 29.
(Contributed by NM, 31-Mar-1998.) (Proof shortened by Andrew Salmon,
26-Jun-2011.)
|
⊢ (𝐴 ∖ (𝐴 ∩ 𝐵)) = (𝐴 ∖ 𝐵) |
|
Theorem | ddifss 3398 |
Double complement under universal class. In classical logic (or given an
additional hypothesis, as in ddifnel 3291), this is equality rather than
subset. (Contributed by Jim Kingdon, 24-Jul-2018.)
|
⊢ 𝐴 ⊆ (V ∖ (V ∖ 𝐴)) |
|
Theorem | unssin 3399 |
Union as a subset of class complement and intersection (De Morgan's
law). One direction of the definition of union in [Mendelson] p. 231.
This would be an equality, rather than subset, in classical logic.
(Contributed by Jim Kingdon, 25-Jul-2018.)
|
⊢ (𝐴 ∪ 𝐵) ⊆ (V ∖ ((V ∖ 𝐴) ∩ (V ∖ 𝐵))) |
|
Theorem | inssun 3400 |
Intersection in terms of class difference and union (De Morgan's law).
Similar to Exercise 4.10(n) of [Mendelson] p. 231. This would be an
equality, rather than subset, in classical logic. (Contributed by Jim
Kingdon, 25-Jul-2018.)
|
⊢ (𝐴 ∩ 𝐵) ⊆ (V ∖ ((V ∖ 𝐴) ∪ (V ∖ 𝐵))) |