Theorem List for Intuitionistic Logic Explorer - 3101-3200 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
Theorem | difeq2d 3101 |
Deduction adding difference to the left in a class equality.
(Contributed by NM, 15-Nov-2002.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐶 ∖ 𝐴) = (𝐶 ∖ 𝐵)) |
|
Theorem | difeq12d 3102 |
Equality deduction for class difference. (Contributed by FL,
29-May-2014.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ∖ 𝐶) = (𝐵 ∖ 𝐷)) |
|
Theorem | difeqri 3103* |
Inference from membership to difference. (Contributed by NM,
17-May-1998.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝑥 ∈ 𝐴 ∧ ¬ 𝑥 ∈ 𝐵) ↔ 𝑥 ∈ 𝐶) ⇒ ⊢ (𝐴 ∖ 𝐵) = 𝐶 |
|
Theorem | nfdif 3104 |
Bound-variable hypothesis builder for class difference. (Contributed by
NM, 3-Dec-2003.) (Revised by Mario Carneiro, 13-Oct-2016.)
|
⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥(𝐴 ∖ 𝐵) |
|
Theorem | eldifi 3105 |
Implication of membership in a class difference. (Contributed by NM,
29-Apr-1994.)
|
⊢ (𝐴 ∈ (𝐵 ∖ 𝐶) → 𝐴 ∈ 𝐵) |
|
Theorem | eldifn 3106 |
Implication of membership in a class difference. (Contributed by NM,
3-May-1994.)
|
⊢ (𝐴 ∈ (𝐵 ∖ 𝐶) → ¬ 𝐴 ∈ 𝐶) |
|
Theorem | elndif 3107 |
A set does not belong to a class excluding it. (Contributed by NM,
27-Jun-1994.)
|
⊢ (𝐴 ∈ 𝐵 → ¬ 𝐴 ∈ (𝐶 ∖ 𝐵)) |
|
Theorem | difdif 3108 |
Double class difference. Exercise 11 of [TakeutiZaring] p. 22.
(Contributed by NM, 17-May-1998.)
|
⊢ (𝐴 ∖ (𝐵 ∖ 𝐴)) = 𝐴 |
|
Theorem | difss 3109 |
Subclass relationship for class difference. Exercise 14 of
[TakeutiZaring] p. 22.
(Contributed by NM, 29-Apr-1994.)
|
⊢ (𝐴 ∖ 𝐵) ⊆ 𝐴 |
|
Theorem | difssd 3110 |
A difference of two classes is contained in the minuend. Deduction form
of difss 3109. (Contributed by David Moews, 1-May-2017.)
|
⊢ (𝜑 → (𝐴 ∖ 𝐵) ⊆ 𝐴) |
|
Theorem | difss2 3111 |
If a class is contained in a difference, it is contained in the minuend.
(Contributed by David Moews, 1-May-2017.)
|
⊢ (𝐴 ⊆ (𝐵 ∖ 𝐶) → 𝐴 ⊆ 𝐵) |
|
Theorem | difss2d 3112 |
If a class is contained in a difference, it is contained in the minuend.
Deduction form of difss2 3111. (Contributed by David Moews,
1-May-2017.)
|
⊢ (𝜑 → 𝐴 ⊆ (𝐵 ∖ 𝐶)) ⇒ ⊢ (𝜑 → 𝐴 ⊆ 𝐵) |
|
Theorem | ssdifss 3113 |
Preservation of a subclass relationship by class difference. (Contributed
by NM, 15-Feb-2007.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐴 ∖ 𝐶) ⊆ 𝐵) |
|
Theorem | ddifnel 3114* |
Double complement under universal class. The hypothesis corresponds to
stability of membership in 𝐴, which is weaker than decidability
(see dcimpstab 786). Actually, the conclusion is a
characterization of
stability of membership in a class (see ddifstab 3115) . Exercise 4.10(s)
of [Mendelson] p. 231, but with an
additional hypothesis. For a version
without a hypothesis, but which only states that 𝐴 is a subset of
V ∖ (V ∖ 𝐴), see ddifss 3219. (Contributed by Jim Kingdon,
21-Jul-2018.)
|
⊢ (¬ 𝑥 ∈ (V ∖ 𝐴) → 𝑥 ∈ 𝐴) ⇒ ⊢ (V ∖ (V ∖ 𝐴)) = 𝐴 |
|
Theorem | ddifstab 3115* |
A class is equal to its double complement if and only if it is stable
(that is, membership in it is a stable property). (Contributed by BJ,
12-Dec-2021.)
|
⊢ ((V ∖ (V ∖ 𝐴)) = 𝐴 ↔ ∀𝑥STAB 𝑥 ∈ 𝐴) |
|
Theorem | ssconb 3116 |
Contraposition law for subsets. (Contributed by NM, 22-Mar-1998.)
|
⊢ ((𝐴 ⊆ 𝐶 ∧ 𝐵 ⊆ 𝐶) → (𝐴 ⊆ (𝐶 ∖ 𝐵) ↔ 𝐵 ⊆ (𝐶 ∖ 𝐴))) |
|
Theorem | sscon 3117 |
Contraposition law for subsets. Exercise 15 of [TakeutiZaring] p. 22.
(Contributed by NM, 22-Mar-1998.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐶 ∖ 𝐵) ⊆ (𝐶 ∖ 𝐴)) |
|
Theorem | ssdif 3118 |
Difference law for subsets. (Contributed by NM, 28-May-1998.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐴 ∖ 𝐶) ⊆ (𝐵 ∖ 𝐶)) |
|
Theorem | ssdifd 3119 |
If 𝐴 is contained in 𝐵, then
(𝐴 ∖
𝐶) is contained in
(𝐵
∖ 𝐶).
Deduction form of ssdif 3118. (Contributed by David
Moews, 1-May-2017.)
|
⊢ (𝜑 → 𝐴 ⊆ 𝐵) ⇒ ⊢ (𝜑 → (𝐴 ∖ 𝐶) ⊆ (𝐵 ∖ 𝐶)) |
|
Theorem | sscond 3120 |
If 𝐴 is contained in 𝐵, then
(𝐶 ∖
𝐵) is contained in
(𝐶
∖ 𝐴).
Deduction form of sscon 3117. (Contributed by David
Moews, 1-May-2017.)
|
⊢ (𝜑 → 𝐴 ⊆ 𝐵) ⇒ ⊢ (𝜑 → (𝐶 ∖ 𝐵) ⊆ (𝐶 ∖ 𝐴)) |
|
Theorem | ssdifssd 3121 |
If 𝐴 is contained in 𝐵, then
(𝐴 ∖
𝐶) is also contained
in
𝐵. Deduction form of ssdifss 3113. (Contributed by David Moews,
1-May-2017.)
|
⊢ (𝜑 → 𝐴 ⊆ 𝐵) ⇒ ⊢ (𝜑 → (𝐴 ∖ 𝐶) ⊆ 𝐵) |
|
Theorem | ssdif2d 3122 |
If 𝐴 is contained in 𝐵 and
𝐶
is contained in 𝐷, then
(𝐴
∖ 𝐷) is
contained in (𝐵 ∖ 𝐶). Deduction form.
(Contributed by David Moews, 1-May-2017.)
|
⊢ (𝜑 → 𝐴 ⊆ 𝐵)
& ⊢ (𝜑 → 𝐶 ⊆ 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ∖ 𝐷) ⊆ (𝐵 ∖ 𝐶)) |
|
Theorem | raldifb 3123 |
Restricted universal quantification on a class difference in terms of an
implication. (Contributed by Alexander van der Vekens, 3-Jan-2018.)
|
⊢ (∀𝑥 ∈ 𝐴 (𝑥 ∉ 𝐵 → 𝜑) ↔ ∀𝑥 ∈ (𝐴 ∖ 𝐵)𝜑) |
|
2.1.13.2 The union of two classes
|
|
Theorem | elun 3124 |
Expansion of membership in class union. Theorem 12 of [Suppes] p. 25.
(Contributed by NM, 7-Aug-1994.)
|
⊢ (𝐴 ∈ (𝐵 ∪ 𝐶) ↔ (𝐴 ∈ 𝐵 ∨ 𝐴 ∈ 𝐶)) |
|
Theorem | uneqri 3125* |
Inference from membership to union. (Contributed by NM, 5-Aug-1993.)
|
⊢ ((𝑥 ∈ 𝐴 ∨ 𝑥 ∈ 𝐵) ↔ 𝑥 ∈ 𝐶) ⇒ ⊢ (𝐴 ∪ 𝐵) = 𝐶 |
|
Theorem | unidm 3126 |
Idempotent law for union of classes. Theorem 23 of [Suppes] p. 27.
(Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∪ 𝐴) = 𝐴 |
|
Theorem | uncom 3127 |
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 3128 |
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 3129 |
Inference form of equncom 3128. (Contributed by Alan Sare,
18-Feb-2012.)
|
⊢ 𝐴 = (𝐵 ∪ 𝐶) ⇒ ⊢ 𝐴 = (𝐶 ∪ 𝐵) |
|
Theorem | uneq1 3130 |
Equality theorem for union of two classes. (Contributed by NM,
5-Aug-1993.)
|
⊢ (𝐴 = 𝐵 → (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐶)) |
|
Theorem | uneq2 3131 |
Equality theorem for the union of two classes. (Contributed by NM,
5-Aug-1993.)
|
⊢ (𝐴 = 𝐵 → (𝐶 ∪ 𝐴) = (𝐶 ∪ 𝐵)) |
|
Theorem | uneq12 3132 |
Equality theorem for union of two classes. (Contributed by NM,
29-Mar-1998.)
|
⊢ ((𝐴 = 𝐵 ∧ 𝐶 = 𝐷) → (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐷)) |
|
Theorem | uneq1i 3133 |
Inference adding union to the right in a class equality. (Contributed
by NM, 30-Aug-1993.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐶) |
|
Theorem | uneq2i 3134 |
Inference adding union to the left in a class equality. (Contributed by
NM, 30-Aug-1993.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐶 ∪ 𝐴) = (𝐶 ∪ 𝐵) |
|
Theorem | uneq12i 3135 |
Equality inference for union of two classes. (Contributed by NM,
12-Aug-2004.) (Proof shortened by Eric Schmidt, 26-Jan-2007.)
|
⊢ 𝐴 = 𝐵
& ⊢ 𝐶 = 𝐷 ⇒ ⊢ (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐷) |
|
Theorem | uneq1d 3136 |
Deduction adding union to the right in a class equality. (Contributed
by NM, 29-Mar-1998.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐶)) |
|
Theorem | uneq2d 3137 |
Deduction adding union to the left in a class equality. (Contributed by
NM, 29-Mar-1998.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐶 ∪ 𝐴) = (𝐶 ∪ 𝐵)) |
|
Theorem | uneq12d 3138 |
Equality deduction for union of two classes. (Contributed by NM,
29-Sep-2004.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ∪ 𝐶) = (𝐵 ∪ 𝐷)) |
|
Theorem | nfun 3139 |
Bound-variable hypothesis builder for the union of classes.
(Contributed by NM, 15-Sep-2003.) (Revised by Mario Carneiro,
14-Oct-2016.)
|
⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥(𝐴 ∪ 𝐵) |
|
Theorem | unass 3140 |
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 3141 |
A rearrangement of union. (Contributed by NM, 12-Aug-2004.)
|
⊢ (𝐴 ∪ (𝐵 ∪ 𝐶)) = (𝐵 ∪ (𝐴 ∪ 𝐶)) |
|
Theorem | un23 3142 |
A rearrangement of union. (Contributed by NM, 12-Aug-2004.) (Proof
shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ∪ 𝐵) ∪ 𝐶) = ((𝐴 ∪ 𝐶) ∪ 𝐵) |
|
Theorem | un4 3143 |
A rearrangement of the union of 4 classes. (Contributed by NM,
12-Aug-2004.)
|
⊢ ((𝐴 ∪ 𝐵) ∪ (𝐶 ∪ 𝐷)) = ((𝐴 ∪ 𝐶) ∪ (𝐵 ∪ 𝐷)) |
|
Theorem | unundi 3144 |
Union distributes over itself. (Contributed by NM, 17-Aug-2004.)
|
⊢ (𝐴 ∪ (𝐵 ∪ 𝐶)) = ((𝐴 ∪ 𝐵) ∪ (𝐴 ∪ 𝐶)) |
|
Theorem | unundir 3145 |
Union distributes over itself. (Contributed by NM, 17-Aug-2004.)
|
⊢ ((𝐴 ∪ 𝐵) ∪ 𝐶) = ((𝐴 ∪ 𝐶) ∪ (𝐵 ∪ 𝐶)) |
|
Theorem | ssun1 3146 |
Subclass relationship for union of classes. Theorem 25 of [Suppes]
p. 27. (Contributed by NM, 5-Aug-1993.)
|
⊢ 𝐴 ⊆ (𝐴 ∪ 𝐵) |
|
Theorem | ssun2 3147 |
Subclass relationship for union of classes. (Contributed by NM,
30-Aug-1993.)
|
⊢ 𝐴 ⊆ (𝐵 ∪ 𝐴) |
|
Theorem | ssun3 3148 |
Subclass law for union of classes. (Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ⊆ 𝐵 → 𝐴 ⊆ (𝐵 ∪ 𝐶)) |
|
Theorem | ssun4 3149 |
Subclass law for union of classes. (Contributed by NM, 14-Aug-1994.)
|
⊢ (𝐴 ⊆ 𝐵 → 𝐴 ⊆ (𝐶 ∪ 𝐵)) |
|
Theorem | elun1 3150 |
Membership law for union of classes. (Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∈ 𝐵 → 𝐴 ∈ (𝐵 ∪ 𝐶)) |
|
Theorem | elun2 3151 |
Membership law for union of classes. (Contributed by NM, 30-Aug-1993.)
|
⊢ (𝐴 ∈ 𝐵 → 𝐴 ∈ (𝐶 ∪ 𝐵)) |
|
Theorem | unss1 3152 |
Subclass law for union of classes. (Contributed by NM, 14-Oct-1999.)
(Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐴 ∪ 𝐶) ⊆ (𝐵 ∪ 𝐶)) |
|
Theorem | ssequn1 3153 |
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 3154 |
Subclass law for union of classes. Exercise 7 of [TakeutiZaring] p. 18.
(Contributed by NM, 14-Oct-1999.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐶 ∪ 𝐴) ⊆ (𝐶 ∪ 𝐵)) |
|
Theorem | unss12 3155 |
Subclass law for union of classes. (Contributed by NM, 2-Jun-2004.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ 𝐶 ⊆ 𝐷) → (𝐴 ∪ 𝐶) ⊆ (𝐵 ∪ 𝐷)) |
|
Theorem | ssequn2 3156 |
A relationship between subclass and union. (Contributed by NM,
13-Jun-1994.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ (𝐵 ∪ 𝐴) = 𝐵) |
|
Theorem | unss 3157 |
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 3158 |
An inference showing the union of two subclasses is a subclass.
(Contributed by Raph Levien, 10-Dec-2002.)
|
⊢ 𝐴 ⊆ 𝐶
& ⊢ 𝐵 ⊆ 𝐶 ⇒ ⊢ (𝐴 ∪ 𝐵) ⊆ 𝐶 |
|
Theorem | unssd 3159 |
A deduction showing the union of two subclasses is a subclass.
(Contributed by Jonathan Ben-Naim, 3-Jun-2011.)
|
⊢ (𝜑 → 𝐴 ⊆ 𝐶)
& ⊢ (𝜑 → 𝐵 ⊆ 𝐶) ⇒ ⊢ (𝜑 → (𝐴 ∪ 𝐵) ⊆ 𝐶) |
|
Theorem | unssad 3160 |
If (𝐴
∪ 𝐵) is
contained in 𝐶, so is 𝐴. One-way
deduction form of unss 3157. Partial converse of unssd 3159. (Contributed
by David Moews, 1-May-2017.)
|
⊢ (𝜑 → (𝐴 ∪ 𝐵) ⊆ 𝐶) ⇒ ⊢ (𝜑 → 𝐴 ⊆ 𝐶) |
|
Theorem | unssbd 3161 |
If (𝐴
∪ 𝐵) is
contained in 𝐶, so is 𝐵. One-way
deduction form of unss 3157. Partial converse of unssd 3159. (Contributed
by David Moews, 1-May-2017.)
|
⊢ (𝜑 → (𝐴 ∪ 𝐵) ⊆ 𝐶) ⇒ ⊢ (𝜑 → 𝐵 ⊆ 𝐶) |
|
Theorem | ssun 3162 |
A condition that implies inclusion in the union of two classes.
(Contributed by NM, 23-Nov-2003.)
|
⊢ ((𝐴 ⊆ 𝐵 ∨ 𝐴 ⊆ 𝐶) → 𝐴 ⊆ (𝐵 ∪ 𝐶)) |
|
Theorem | rexun 3163 |
Restricted existential quantification over union. (Contributed by Jeff
Madsen, 5-Jan-2011.)
|
⊢ (∃𝑥 ∈ (𝐴 ∪ 𝐵)𝜑 ↔ (∃𝑥 ∈ 𝐴 𝜑 ∨ ∃𝑥 ∈ 𝐵 𝜑)) |
|
Theorem | ralunb 3164 |
Restricted quantification over a union. (Contributed by Scott Fenton,
12-Apr-2011.) (Proof shortened by Andrew Salmon, 29-Jun-2011.)
|
⊢ (∀𝑥 ∈ (𝐴 ∪ 𝐵)𝜑 ↔ (∀𝑥 ∈ 𝐴 𝜑 ∧ ∀𝑥 ∈ 𝐵 𝜑)) |
|
Theorem | ralun 3165 |
Restricted quantification over union. (Contributed by Jeff Madsen,
2-Sep-2009.)
|
⊢ ((∀𝑥 ∈ 𝐴 𝜑 ∧ ∀𝑥 ∈ 𝐵 𝜑) → ∀𝑥 ∈ (𝐴 ∪ 𝐵)𝜑) |
|
2.1.13.3 The intersection of two
classes
|
|
Theorem | elin 3166 |
Expansion of membership in an intersection of two classes. Theorem 12
of [Suppes] p. 25. (Contributed by NM,
29-Apr-1994.)
|
⊢ (𝐴 ∈ (𝐵 ∩ 𝐶) ↔ (𝐴 ∈ 𝐵 ∧ 𝐴 ∈ 𝐶)) |
|
Theorem | elini 3167 |
Membership in an intersection of two classes. (Contributed by Glauco
Siliprandi, 17-Aug-2020.)
|
⊢ 𝐴 ∈ 𝐵
& ⊢ 𝐴 ∈ 𝐶 ⇒ ⊢ 𝐴 ∈ (𝐵 ∩ 𝐶) |
|
Theorem | elind 3168 |
Deduce membership in an intersection of two classes. (Contributed by
Jonathan Ben-Naim, 3-Jun-2011.)
|
⊢ (𝜑 → 𝑋 ∈ 𝐴)
& ⊢ (𝜑 → 𝑋 ∈ 𝐵) ⇒ ⊢ (𝜑 → 𝑋 ∈ (𝐴 ∩ 𝐵)) |
|
Theorem | elinel1 3169 |
Membership in an intersection implies membership in the first set.
(Contributed by Glauco Siliprandi, 11-Dec-2019.)
|
⊢ (𝐴 ∈ (𝐵 ∩ 𝐶) → 𝐴 ∈ 𝐵) |
|
Theorem | elinel2 3170 |
Membership in an intersection implies membership in the second set.
(Contributed by Glauco Siliprandi, 11-Dec-2019.)
|
⊢ (𝐴 ∈ (𝐵 ∩ 𝐶) → 𝐴 ∈ 𝐶) |
|
Theorem | elin2 3171 |
Membership in a class defined as an intersection. (Contributed by
Stefan O'Rear, 29-Mar-2015.)
|
⊢ 𝑋 = (𝐵 ∩ 𝐶) ⇒ ⊢ (𝐴 ∈ 𝑋 ↔ (𝐴 ∈ 𝐵 ∧ 𝐴 ∈ 𝐶)) |
|
Theorem | elin1d 3172 |
Elementhood in the first set of an intersection - deduction version.
(Contributed by Thierry Arnoux, 3-May-2020.)
|
⊢ (𝜑 → 𝑋 ∈ (𝐴 ∩ 𝐵)) ⇒ ⊢ (𝜑 → 𝑋 ∈ 𝐴) |
|
Theorem | elin2d 3173 |
Elementhood in the first set of an intersection - deduction version.
(Contributed by Thierry Arnoux, 3-May-2020.)
|
⊢ (𝜑 → 𝑋 ∈ (𝐴 ∩ 𝐵)) ⇒ ⊢ (𝜑 → 𝑋 ∈ 𝐵) |
|
Theorem | elin3 3174 |
Membership in a class defined as a ternary intersection. (Contributed
by Stefan O'Rear, 29-Mar-2015.)
|
⊢ 𝑋 = ((𝐵 ∩ 𝐶) ∩ 𝐷) ⇒ ⊢ (𝐴 ∈ 𝑋 ↔ (𝐴 ∈ 𝐵 ∧ 𝐴 ∈ 𝐶 ∧ 𝐴 ∈ 𝐷)) |
|
Theorem | incom 3175 |
Commutative law for intersection of classes. Exercise 7 of
[TakeutiZaring] p. 17.
(Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∩ 𝐵) = (𝐵 ∩ 𝐴) |
|
Theorem | ineqri 3176* |
Inference from membership to intersection. (Contributed by NM,
5-Aug-1993.)
|
⊢ ((𝑥 ∈ 𝐴 ∧ 𝑥 ∈ 𝐵) ↔ 𝑥 ∈ 𝐶) ⇒ ⊢ (𝐴 ∩ 𝐵) = 𝐶 |
|
Theorem | ineq1 3177 |
Equality theorem for intersection of two classes. (Contributed by NM,
14-Dec-1993.)
|
⊢ (𝐴 = 𝐵 → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐶)) |
|
Theorem | ineq2 3178 |
Equality theorem for intersection of two classes. (Contributed by NM,
26-Dec-1993.)
|
⊢ (𝐴 = 𝐵 → (𝐶 ∩ 𝐴) = (𝐶 ∩ 𝐵)) |
|
Theorem | ineq12 3179 |
Equality theorem for intersection of two classes. (Contributed by NM,
8-May-1994.)
|
⊢ ((𝐴 = 𝐵 ∧ 𝐶 = 𝐷) → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐷)) |
|
Theorem | ineq1i 3180 |
Equality inference for intersection of two classes. (Contributed by NM,
26-Dec-1993.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐶) |
|
Theorem | ineq2i 3181 |
Equality inference for intersection of two classes. (Contributed by NM,
26-Dec-1993.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐶 ∩ 𝐴) = (𝐶 ∩ 𝐵) |
|
Theorem | ineq12i 3182 |
Equality inference for intersection of two classes. (Contributed by
NM, 24-Jun-2004.) (Proof shortened by Eric Schmidt, 26-Jan-2007.)
|
⊢ 𝐴 = 𝐵
& ⊢ 𝐶 = 𝐷 ⇒ ⊢ (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐷) |
|
Theorem | ineq1d 3183 |
Equality deduction for intersection of two classes. (Contributed by NM,
10-Apr-1994.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐶)) |
|
Theorem | ineq2d 3184 |
Equality deduction for intersection of two classes. (Contributed by NM,
10-Apr-1994.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐶 ∩ 𝐴) = (𝐶 ∩ 𝐵)) |
|
Theorem | ineq12d 3185 |
Equality deduction for intersection of two classes. (Contributed by
NM, 24-Jun-2004.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐷)) |
|
Theorem | ineqan12d 3186 |
Equality deduction for intersection of two classes. (Contributed by
NM, 7-Feb-2007.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜓 → 𝐶 = 𝐷) ⇒ ⊢ ((𝜑 ∧ 𝜓) → (𝐴 ∩ 𝐶) = (𝐵 ∩ 𝐷)) |
|
Theorem | dfss1 3187 |
A frequently-used variant of subclass definition df-ss 2996. (Contributed
by NM, 10-Jan-2015.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ (𝐵 ∩ 𝐴) = 𝐴) |
|
Theorem | dfss5 3188 |
Another definition of subclasshood. Similar to df-ss 2996, dfss 2997, and
dfss1 3187. (Contributed by David Moews, 1-May-2017.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ 𝐴 = (𝐵 ∩ 𝐴)) |
|
Theorem | nfin 3189 |
Bound-variable hypothesis builder for the intersection of classes.
(Contributed by NM, 15-Sep-2003.) (Revised by Mario Carneiro,
14-Oct-2016.)
|
⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥(𝐴 ∩ 𝐵) |
|
Theorem | csbing 3190 |
Distribute proper substitution through an intersection relation.
(Contributed by Alan Sare, 22-Jul-2012.)
|
⊢ (𝐴 ∈ 𝐵 → ⦋𝐴 / 𝑥⦌(𝐶 ∩ 𝐷) = (⦋𝐴 / 𝑥⦌𝐶 ∩ ⦋𝐴 / 𝑥⦌𝐷)) |
|
Theorem | rabbi2dva 3191* |
Deduction from a wff to a restricted class abstraction. (Contributed by
NM, 14-Jan-2014.)
|
⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝑥 ∈ 𝐵 ↔ 𝜓)) ⇒ ⊢ (𝜑 → (𝐴 ∩ 𝐵) = {𝑥 ∈ 𝐴 ∣ 𝜓}) |
|
Theorem | inidm 3192 |
Idempotent law for intersection of classes. Theorem 15 of [Suppes]
p. 26. (Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∩ 𝐴) = 𝐴 |
|
Theorem | inass 3193 |
Associative law for intersection of classes. Exercise 9 of
[TakeutiZaring] p. 17.
(Contributed by NM, 3-May-1994.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = (𝐴 ∩ (𝐵 ∩ 𝐶)) |
|
Theorem | in12 3194 |
A rearrangement of intersection. (Contributed by NM, 21-Apr-2001.)
|
⊢ (𝐴 ∩ (𝐵 ∩ 𝐶)) = (𝐵 ∩ (𝐴 ∩ 𝐶)) |
|
Theorem | in32 3195 |
A rearrangement of intersection. (Contributed by NM, 21-Apr-2001.)
(Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = ((𝐴 ∩ 𝐶) ∩ 𝐵) |
|
Theorem | in13 3196 |
A rearrangement of intersection. (Contributed by NM, 27-Aug-2012.)
|
⊢ (𝐴 ∩ (𝐵 ∩ 𝐶)) = (𝐶 ∩ (𝐵 ∩ 𝐴)) |
|
Theorem | in31 3197 |
A rearrangement of intersection. (Contributed by NM, 27-Aug-2012.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = ((𝐶 ∩ 𝐵) ∩ 𝐴) |
|
Theorem | inrot 3198 |
Rotate the intersection of 3 classes. (Contributed by NM,
27-Aug-2012.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ 𝐶) = ((𝐶 ∩ 𝐴) ∩ 𝐵) |
|
Theorem | in4 3199 |
Rearrangement of intersection of 4 classes. (Contributed by NM,
21-Apr-2001.)
|
⊢ ((𝐴 ∩ 𝐵) ∩ (𝐶 ∩ 𝐷)) = ((𝐴 ∩ 𝐶) ∩ (𝐵 ∩ 𝐷)) |
|
Theorem | inindi 3200 |
Intersection distributes over itself. (Contributed by NM, 6-May-1994.)
|
⊢ (𝐴 ∩ (𝐵 ∩ 𝐶)) = ((𝐴 ∩ 𝐵) ∩ (𝐴 ∩ 𝐶)) |