Theorem List for Intuitionistic Logic Explorer - 3401-3500 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
Theorem | rabun2 3401 |
Abstraction restricted to a union. (Contributed by Stefan O'Rear,
5-Feb-2015.)
|
⊢ {𝑥 ∈ (𝐴 ∪ 𝐵) ∣ 𝜑} = ({𝑥 ∈ 𝐴 ∣ 𝜑} ∪ {𝑥 ∈ 𝐵 ∣ 𝜑}) |
|
2.1.13.6 Restricted uniqueness with difference,
union, and intersection
|
|
Theorem | reuss2 3402* |
Transfer uniqueness to a smaller subclass. (Contributed by NM,
20-Oct-2005.)
|
⊢ (((𝐴 ⊆ 𝐵 ∧ ∀𝑥 ∈ 𝐴 (𝜑 → 𝜓)) ∧ (∃𝑥 ∈ 𝐴 𝜑 ∧ ∃!𝑥 ∈ 𝐵 𝜓)) → ∃!𝑥 ∈ 𝐴 𝜑) |
|
Theorem | reuss 3403* |
Transfer uniqueness to a smaller subclass. (Contributed by NM,
21-Aug-1999.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ ∃𝑥 ∈ 𝐴 𝜑 ∧ ∃!𝑥 ∈ 𝐵 𝜑) → ∃!𝑥 ∈ 𝐴 𝜑) |
|
Theorem | reuun1 3404* |
Transfer uniqueness to a smaller class. (Contributed by NM,
21-Oct-2005.)
|
⊢ ((∃𝑥 ∈ 𝐴 𝜑 ∧ ∃!𝑥 ∈ (𝐴 ∪ 𝐵)(𝜑 ∨ 𝜓)) → ∃!𝑥 ∈ 𝐴 𝜑) |
|
Theorem | reuun2 3405* |
Transfer uniqueness to a smaller or larger class. (Contributed by NM,
21-Oct-2005.)
|
⊢ (¬ ∃𝑥 ∈ 𝐵 𝜑 → (∃!𝑥 ∈ (𝐴 ∪ 𝐵)𝜑 ↔ ∃!𝑥 ∈ 𝐴 𝜑)) |
|
Theorem | reupick 3406* |
Restricted uniqueness "picks" a member of a subclass. (Contributed
by
NM, 21-Aug-1999.)
|
⊢ (((𝐴 ⊆ 𝐵 ∧ (∃𝑥 ∈ 𝐴 𝜑 ∧ ∃!𝑥 ∈ 𝐵 𝜑)) ∧ 𝜑) → (𝑥 ∈ 𝐴 ↔ 𝑥 ∈ 𝐵)) |
|
Theorem | reupick3 3407* |
Restricted uniqueness "picks" a member of a subclass. (Contributed
by
Mario Carneiro, 19-Nov-2016.)
|
⊢ ((∃!𝑥 ∈ 𝐴 𝜑 ∧ ∃𝑥 ∈ 𝐴 (𝜑 ∧ 𝜓) ∧ 𝑥 ∈ 𝐴) → (𝜑 → 𝜓)) |
|
Theorem | reupick2 3408* |
Restricted uniqueness "picks" a member of a subclass. (Contributed
by
Mario Carneiro, 15-Dec-2013.) (Proof shortened by Mario Carneiro,
19-Nov-2016.)
|
⊢ (((∀𝑥 ∈ 𝐴 (𝜓 → 𝜑) ∧ ∃𝑥 ∈ 𝐴 𝜓 ∧ ∃!𝑥 ∈ 𝐴 𝜑) ∧ 𝑥 ∈ 𝐴) → (𝜑 ↔ 𝜓)) |
|
2.1.14 The empty set
|
|
Syntax | c0 3409 |
Extend class notation to include the empty set.
|
class ∅ |
|
Definition | df-nul 3410 |
Define the empty set. Special case of Exercise 4.10(o) of [Mendelson]
p. 231. For a more traditional definition, but requiring a dummy
variable, see dfnul2 3411. (Contributed by NM, 5-Aug-1993.)
|
⊢ ∅ = (V ∖ V) |
|
Theorem | dfnul2 3411 |
Alternate definition of the empty set. Definition 5.14 of [TakeutiZaring]
p. 20. (Contributed by NM, 26-Dec-1996.)
|
⊢ ∅ = {𝑥 ∣ ¬ 𝑥 = 𝑥} |
|
Theorem | dfnul3 3412 |
Alternate definition of the empty set. (Contributed by NM,
25-Mar-2004.)
|
⊢ ∅ = {𝑥 ∈ 𝐴 ∣ ¬ 𝑥 ∈ 𝐴} |
|
Theorem | noel 3413 |
The empty set has no elements. Theorem 6.14 of [Quine] p. 44.
(Contributed by NM, 5-Aug-1993.) (Proof shortened by Mario Carneiro,
1-Sep-2015.)
|
⊢ ¬ 𝐴 ∈ ∅ |
|
Theorem | n0i 3414 |
If a set has elements, it is not empty. A set with elements is also
inhabited, see elex2 2742. (Contributed by NM, 31-Dec-1993.)
|
⊢ (𝐵 ∈ 𝐴 → ¬ 𝐴 = ∅) |
|
Theorem | ne0i 3415 |
If a set has elements, it is not empty. A set with elements is also
inhabited, see elex2 2742. (Contributed by NM, 31-Dec-1993.)
|
⊢ (𝐵 ∈ 𝐴 → 𝐴 ≠ ∅) |
|
Theorem | ne0d 3416 |
Deduction form of ne0i 3415. If a class has elements, then it is
nonempty. (Contributed by Glauco Siliprandi, 23-Oct-2021.)
|
⊢ (𝜑 → 𝐵 ∈ 𝐴) ⇒ ⊢ (𝜑 → 𝐴 ≠ ∅) |
|
Theorem | n0ii 3417 |
If a class has elements, then it is not empty. Inference associated
with n0i 3414. (Contributed by BJ, 15-Jul-2021.)
|
⊢ 𝐴 ∈ 𝐵 ⇒ ⊢ ¬ 𝐵 = ∅ |
|
Theorem | ne0ii 3418 |
If a class has elements, then it is nonempty. Inference associated with
ne0i 3415. (Contributed by Glauco Siliprandi,
11-Dec-2019.)
|
⊢ 𝐴 ∈ 𝐵 ⇒ ⊢ 𝐵 ≠ ∅ |
|
Theorem | vn0 3419 |
The universal class is not equal to the empty set. (Contributed by NM,
11-Sep-2008.)
|
⊢ V ≠ ∅ |
|
Theorem | vn0m 3420 |
The universal class is inhabited. (Contributed by Jim Kingdon,
17-Dec-2018.)
|
⊢ ∃𝑥 𝑥 ∈ V |
|
Theorem | n0rf 3421 |
An inhabited class is nonempty. Following the Definition of [Bauer],
p. 483, we call a class 𝐴 nonempty if 𝐴 ≠ ∅ and
inhabited if
it has at least one element. In classical logic these two concepts are
equivalent, for example see Proposition 5.17(1) of [TakeutiZaring]
p. 20. This version of n0r 3422 requires only that 𝑥 not be free in,
rather than not occur in, 𝐴. (Contributed by Jim Kingdon,
31-Jul-2018.)
|
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ (∃𝑥 𝑥 ∈ 𝐴 → 𝐴 ≠ ∅) |
|
Theorem | n0r 3422* |
An inhabited class is nonempty. See n0rf 3421 for more discussion.
(Contributed by Jim Kingdon, 31-Jul-2018.)
|
⊢ (∃𝑥 𝑥 ∈ 𝐴 → 𝐴 ≠ ∅) |
|
Theorem | neq0r 3423* |
An inhabited class is nonempty. See n0rf 3421 for more discussion.
(Contributed by Jim Kingdon, 31-Jul-2018.)
|
⊢ (∃𝑥 𝑥 ∈ 𝐴 → ¬ 𝐴 = ∅) |
|
Theorem | reximdva0m 3424* |
Restricted existence deduced from inhabited class. (Contributed by Jim
Kingdon, 31-Jul-2018.)
|
⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝜓) ⇒ ⊢ ((𝜑 ∧ ∃𝑥 𝑥 ∈ 𝐴) → ∃𝑥 ∈ 𝐴 𝜓) |
|
Theorem | n0mmoeu 3425* |
A case of equivalence of "at most one" and "only one". If
a class is
inhabited, that class having at most one element is equivalent to it
having only one element. (Contributed by Jim Kingdon, 31-Jul-2018.)
|
⊢ (∃𝑥 𝑥 ∈ 𝐴 → (∃*𝑥 𝑥 ∈ 𝐴 ↔ ∃!𝑥 𝑥 ∈ 𝐴)) |
|
Theorem | rex0 3426 |
Vacuous existential quantification is false. (Contributed by NM,
15-Oct-2003.)
|
⊢ ¬ ∃𝑥 ∈ ∅ 𝜑 |
|
Theorem | eq0 3427* |
The empty set has no elements. Theorem 2 of [Suppes] p. 22.
(Contributed by NM, 29-Aug-1993.)
|
⊢ (𝐴 = ∅ ↔ ∀𝑥 ¬ 𝑥 ∈ 𝐴) |
|
Theorem | eqv 3428* |
The universe contains every set. (Contributed by NM, 11-Sep-2006.)
|
⊢ (𝐴 = V ↔ ∀𝑥 𝑥 ∈ 𝐴) |
|
Theorem | notm0 3429* |
A class is not inhabited if and only if it is empty. (Contributed by
Jim Kingdon, 1-Jul-2022.)
|
⊢ (¬ ∃𝑥 𝑥 ∈ 𝐴 ↔ 𝐴 = ∅) |
|
Theorem | nel0 3430* |
From the general negation of membership in 𝐴, infer that 𝐴 is
the empty set. (Contributed by BJ, 6-Oct-2018.)
|
⊢ ¬ 𝑥 ∈ 𝐴 ⇒ ⊢ 𝐴 = ∅ |
|
Theorem | 0el 3431* |
Membership of the empty set in another class. (Contributed by NM,
29-Jun-2004.)
|
⊢ (∅ ∈ 𝐴 ↔ ∃𝑥 ∈ 𝐴 ∀𝑦 ¬ 𝑦 ∈ 𝑥) |
|
Theorem | abvor0dc 3432* |
The class builder of a decidable proposition not containing the
abstraction variable is either the universal class or the empty set.
(Contributed by Jim Kingdon, 1-Aug-2018.)
|
⊢ (DECID 𝜑 → ({𝑥 ∣ 𝜑} = V ∨ {𝑥 ∣ 𝜑} = ∅)) |
|
Theorem | abn0r 3433 |
Nonempty class abstraction. (Contributed by Jim Kingdon, 1-Aug-2018.)
|
⊢ (∃𝑥𝜑 → {𝑥 ∣ 𝜑} ≠ ∅) |
|
Theorem | abn0m 3434* |
Inhabited class abstraction. (Contributed by Jim Kingdon,
8-Jul-2022.)
|
⊢ (∃𝑦 𝑦 ∈ {𝑥 ∣ 𝜑} ↔ ∃𝑥𝜑) |
|
Theorem | rabn0r 3435 |
Nonempty restricted class abstraction. (Contributed by Jim Kingdon,
1-Aug-2018.)
|
⊢ (∃𝑥 ∈ 𝐴 𝜑 → {𝑥 ∈ 𝐴 ∣ 𝜑} ≠ ∅) |
|
Theorem | rabn0m 3436* |
Inhabited restricted class abstraction. (Contributed by Jim Kingdon,
18-Sep-2018.)
|
⊢ (∃𝑦 𝑦 ∈ {𝑥 ∈ 𝐴 ∣ 𝜑} ↔ ∃𝑥 ∈ 𝐴 𝜑) |
|
Theorem | rab0 3437 |
Any restricted class abstraction restricted to the empty set is empty.
(Contributed by NM, 15-Oct-2003.) (Proof shortened by Andrew Salmon,
26-Jun-2011.)
|
⊢ {𝑥 ∈ ∅ ∣ 𝜑} = ∅ |
|
Theorem | rabeq0 3438 |
Condition for a restricted class abstraction to be empty. (Contributed
by Jeff Madsen, 7-Jun-2010.)
|
⊢ ({𝑥 ∈ 𝐴 ∣ 𝜑} = ∅ ↔ ∀𝑥 ∈ 𝐴 ¬ 𝜑) |
|
Theorem | abeq0 3439 |
Condition for a class abstraction to be empty. (Contributed by Jim
Kingdon, 12-Aug-2018.)
|
⊢ ({𝑥 ∣ 𝜑} = ∅ ↔ ∀𝑥 ¬ 𝜑) |
|
Theorem | rabxmdc 3440* |
Law of excluded middle given decidability, in terms of restricted class
abstractions. (Contributed by Jim Kingdon, 2-Aug-2018.)
|
⊢ (∀𝑥DECID 𝜑 → 𝐴 = ({𝑥 ∈ 𝐴 ∣ 𝜑} ∪ {𝑥 ∈ 𝐴 ∣ ¬ 𝜑})) |
|
Theorem | rabnc 3441* |
Law of noncontradiction, in terms of restricted class abstractions.
(Contributed by Jeff Madsen, 20-Jun-2011.)
|
⊢ ({𝑥 ∈ 𝐴 ∣ 𝜑} ∩ {𝑥 ∈ 𝐴 ∣ ¬ 𝜑}) = ∅ |
|
Theorem | un0 3442 |
The union of a class with the empty set is itself. Theorem 24 of
[Suppes] p. 27. (Contributed by NM,
5-Aug-1993.)
|
⊢ (𝐴 ∪ ∅) = 𝐴 |
|
Theorem | in0 3443 |
The intersection of a class with the empty set is the empty set.
Theorem 16 of [Suppes] p. 26.
(Contributed by NM, 5-Aug-1993.)
|
⊢ (𝐴 ∩ ∅) = ∅ |
|
Theorem | 0in 3444 |
The intersection of the empty set with a class is the empty set.
(Contributed by Glauco Siliprandi, 17-Aug-2020.)
|
⊢ (∅ ∩ 𝐴) = ∅ |
|
Theorem | inv1 3445 |
The intersection of a class with the universal class is itself. Exercise
4.10(k) of [Mendelson] p. 231.
(Contributed by NM, 17-May-1998.)
|
⊢ (𝐴 ∩ V) = 𝐴 |
|
Theorem | unv 3446 |
The union of a class with the universal class is the universal class.
Exercise 4.10(l) of [Mendelson] p. 231.
(Contributed by NM,
17-May-1998.)
|
⊢ (𝐴 ∪ V) = V |
|
Theorem | 0ss 3447 |
The null set is a subset of any class. Part of Exercise 1 of
[TakeutiZaring] p. 22.
(Contributed by NM, 5-Aug-1993.)
|
⊢ ∅ ⊆ 𝐴 |
|
Theorem | ss0b 3448 |
Any subset of the empty set is empty. Theorem 5 of [Suppes] p. 23 and its
converse. (Contributed by NM, 17-Sep-2003.)
|
⊢ (𝐴 ⊆ ∅ ↔ 𝐴 = ∅) |
|
Theorem | ss0 3449 |
Any subset of the empty set is empty. Theorem 5 of [Suppes] p. 23.
(Contributed by NM, 13-Aug-1994.)
|
⊢ (𝐴 ⊆ ∅ → 𝐴 = ∅) |
|
Theorem | sseq0 3450 |
A subclass of an empty class is empty. (Contributed by NM, 7-Mar-2007.)
(Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ 𝐵 = ∅) → 𝐴 = ∅) |
|
Theorem | ssn0 3451 |
A class with a nonempty subclass is nonempty. (Contributed by NM,
17-Feb-2007.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ 𝐴 ≠ ∅) → 𝐵 ≠ ∅) |
|
Theorem | abf 3452 |
A class builder with a false argument is empty. (Contributed by NM,
20-Jan-2012.)
|
⊢ ¬ 𝜑 ⇒ ⊢ {𝑥 ∣ 𝜑} = ∅ |
|
Theorem | eq0rdv 3453* |
Deduction for equality to the empty set. (Contributed by NM,
11-Jul-2014.)
|
⊢ (𝜑 → ¬ 𝑥 ∈ 𝐴) ⇒ ⊢ (𝜑 → 𝐴 = ∅) |
|
Theorem | csbprc 3454 |
The proper substitution of a proper class for a set into a class results
in the empty set. (Contributed by NM, 17-Aug-2018.)
|
⊢ (¬ 𝐴 ∈ V → ⦋𝐴 / 𝑥⦌𝐵 = ∅) |
|
Theorem | un00 3455 |
Two classes are empty iff their union is empty. (Contributed by NM,
11-Aug-2004.)
|
⊢ ((𝐴 = ∅ ∧ 𝐵 = ∅) ↔ (𝐴 ∪ 𝐵) = ∅) |
|
Theorem | vss 3456 |
Only the universal class has the universal class as a subclass.
(Contributed by NM, 17-Sep-2003.) (Proof shortened by Andrew Salmon,
26-Jun-2011.)
|
⊢ (V ⊆ 𝐴 ↔ 𝐴 = V) |
|
Theorem | disj 3457* |
Two ways of saying that two classes are disjoint (have no members in
common). (Contributed by NM, 17-Feb-2004.)
|
⊢ ((𝐴 ∩ 𝐵) = ∅ ↔ ∀𝑥 ∈ 𝐴 ¬ 𝑥 ∈ 𝐵) |
|
Theorem | disjr 3458* |
Two ways of saying that two classes are disjoint. (Contributed by Jeff
Madsen, 19-Jun-2011.)
|
⊢ ((𝐴 ∩ 𝐵) = ∅ ↔ ∀𝑥 ∈ 𝐵 ¬ 𝑥 ∈ 𝐴) |
|
Theorem | disj1 3459* |
Two ways of saying that two classes are disjoint (have no members in
common). (Contributed by NM, 19-Aug-1993.)
|
⊢ ((𝐴 ∩ 𝐵) = ∅ ↔ ∀𝑥(𝑥 ∈ 𝐴 → ¬ 𝑥 ∈ 𝐵)) |
|
Theorem | reldisj 3460 |
Two ways of saying that two classes are disjoint, using the complement
of 𝐵 relative to a universe 𝐶.
(Contributed by NM,
15-Feb-2007.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (𝐴 ⊆ 𝐶 → ((𝐴 ∩ 𝐵) = ∅ ↔ 𝐴 ⊆ (𝐶 ∖ 𝐵))) |
|
Theorem | disj3 3461 |
Two ways of saying that two classes are disjoint. (Contributed by NM,
19-May-1998.)
|
⊢ ((𝐴 ∩ 𝐵) = ∅ ↔ 𝐴 = (𝐴 ∖ 𝐵)) |
|
Theorem | disjne 3462 |
Members of disjoint sets are not equal. (Contributed by NM,
28-Mar-2007.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ (((𝐴 ∩ 𝐵) = ∅ ∧ 𝐶 ∈ 𝐴 ∧ 𝐷 ∈ 𝐵) → 𝐶 ≠ 𝐷) |
|
Theorem | disjel 3463 |
A set can't belong to both members of disjoint classes. (Contributed by
NM, 28-Feb-2015.)
|
⊢ (((𝐴 ∩ 𝐵) = ∅ ∧ 𝐶 ∈ 𝐴) → ¬ 𝐶 ∈ 𝐵) |
|
Theorem | disj2 3464 |
Two ways of saying that two classes are disjoint. (Contributed by NM,
17-May-1998.)
|
⊢ ((𝐴 ∩ 𝐵) = ∅ ↔ 𝐴 ⊆ (V ∖ 𝐵)) |
|
Theorem | ssdisj 3465 |
Intersection with a subclass of a disjoint class. (Contributed by FL,
24-Jan-2007.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ (𝐵 ∩ 𝐶) = ∅) → (𝐴 ∩ 𝐶) = ∅) |
|
Theorem | undisj1 3466 |
The union of disjoint classes is disjoint. (Contributed by NM,
26-Sep-2004.)
|
⊢ (((𝐴 ∩ 𝐶) = ∅ ∧ (𝐵 ∩ 𝐶) = ∅) ↔ ((𝐴 ∪ 𝐵) ∩ 𝐶) = ∅) |
|
Theorem | undisj2 3467 |
The union of disjoint classes is disjoint. (Contributed by NM,
13-Sep-2004.)
|
⊢ (((𝐴 ∩ 𝐵) = ∅ ∧ (𝐴 ∩ 𝐶) = ∅) ↔ (𝐴 ∩ (𝐵 ∪ 𝐶)) = ∅) |
|
Theorem | ssindif0im 3468 |
Subclass implies empty intersection with difference from the universal
class. (Contributed by NM, 17-Sep-2003.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐴 ∩ (V ∖ 𝐵)) = ∅) |
|
Theorem | inelcm 3469 |
The intersection of classes with a common member is nonempty.
(Contributed by NM, 7-Apr-1994.)
|
⊢ ((𝐴 ∈ 𝐵 ∧ 𝐴 ∈ 𝐶) → (𝐵 ∩ 𝐶) ≠ ∅) |
|
Theorem | minel 3470 |
A minimum element of a class has no elements in common with the class.
(Contributed by NM, 22-Jun-1994.)
|
⊢ ((𝐴 ∈ 𝐵 ∧ (𝐶 ∩ 𝐵) = ∅) → ¬ 𝐴 ∈ 𝐶) |
|
Theorem | undif4 3471 |
Distribute union over difference. (Contributed by NM, 17-May-1998.)
(Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ∩ 𝐶) = ∅ → (𝐴 ∪ (𝐵 ∖ 𝐶)) = ((𝐴 ∪ 𝐵) ∖ 𝐶)) |
|
Theorem | disjssun 3472 |
Subset relation for disjoint classes. (Contributed by NM, 25-Oct-2005.)
(Proof shortened by Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ∩ 𝐵) = ∅ → (𝐴 ⊆ (𝐵 ∪ 𝐶) ↔ 𝐴 ⊆ 𝐶)) |
|
Theorem | ssdif0im 3473 |
Subclass implies empty difference. One direction of Exercise 7 of
[TakeutiZaring] p. 22. In
classical logic this would be an equivalence.
(Contributed by Jim Kingdon, 2-Aug-2018.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐴 ∖ 𝐵) = ∅) |
|
Theorem | vdif0im 3474 |
Universal class equality in terms of empty difference. (Contributed by
Jim Kingdon, 3-Aug-2018.)
|
⊢ (𝐴 = V → (V ∖ 𝐴) = ∅) |
|
Theorem | difrab0eqim 3475* |
If the difference between the restricting class of a restricted class
abstraction and the restricted class abstraction is empty, the
restricting class is equal to this restricted class abstraction.
(Contributed by Jim Kingdon, 3-Aug-2018.)
|
⊢ (𝑉 = {𝑥 ∈ 𝑉 ∣ 𝜑} → (𝑉 ∖ {𝑥 ∈ 𝑉 ∣ 𝜑}) = ∅) |
|
Theorem | inssdif0im 3476 |
Intersection, subclass, and difference relationship. In classical logic
the converse would also hold. (Contributed by Jim Kingdon,
3-Aug-2018.)
|
⊢ ((𝐴 ∩ 𝐵) ⊆ 𝐶 → (𝐴 ∩ (𝐵 ∖ 𝐶)) = ∅) |
|
Theorem | difid 3477 |
The difference between a class and itself is the empty set. Proposition
5.15 of [TakeutiZaring] p. 20. Also
Theorem 32 of [Suppes] p. 28.
(Contributed by NM, 22-Apr-2004.)
|
⊢ (𝐴 ∖ 𝐴) = ∅ |
|
Theorem | difidALT 3478 |
The difference between a class and itself is the empty set. Proposition
5.15 of [TakeutiZaring] p. 20.
Also Theorem 32 of [Suppes] p. 28.
Alternate proof of difid 3477. (Contributed by David Abernethy,
17-Jun-2012.) (Proof modification is discouraged.)
(New usage is discouraged.)
|
⊢ (𝐴 ∖ 𝐴) = ∅ |
|
Theorem | dif0 3479 |
The difference between a class and the empty set. Part of Exercise 4.4 of
[Stoll] p. 16. (Contributed by NM,
17-Aug-2004.)
|
⊢ (𝐴 ∖ ∅) = 𝐴 |
|
Theorem | 0dif 3480 |
The difference between the empty set and a class. Part of Exercise 4.4 of
[Stoll] p. 16. (Contributed by NM,
17-Aug-2004.)
|
⊢ (∅ ∖ 𝐴) = ∅ |
|
Theorem | disjdif 3481 |
A class and its relative complement are disjoint. Theorem 38 of [Suppes]
p. 29. (Contributed by NM, 24-Mar-1998.)
|
⊢ (𝐴 ∩ (𝐵 ∖ 𝐴)) = ∅ |
|
Theorem | difin0 3482 |
The difference of a class from its intersection is empty. Theorem 37 of
[Suppes] p. 29. (Contributed by NM,
17-Aug-2004.) (Proof shortened by
Andrew Salmon, 26-Jun-2011.)
|
⊢ ((𝐴 ∩ 𝐵) ∖ 𝐵) = ∅ |
|
Theorem | undif1ss 3483 |
Absorption of difference by union. In classical logic, as Theorem 35 of
[Suppes] p. 29, this would be equality
rather than subset. (Contributed
by Jim Kingdon, 4-Aug-2018.)
|
⊢ ((𝐴 ∖ 𝐵) ∪ 𝐵) ⊆ (𝐴 ∪ 𝐵) |
|
Theorem | undif2ss 3484 |
Absorption of difference by union. In classical logic, as in Part of
proof of Corollary 6K of [Enderton] p.
144, this would be equality rather
than subset. (Contributed by Jim Kingdon, 4-Aug-2018.)
|
⊢ (𝐴 ∪ (𝐵 ∖ 𝐴)) ⊆ (𝐴 ∪ 𝐵) |
|
Theorem | undifabs 3485 |
Absorption of difference by union. (Contributed by NM, 18-Aug-2013.)
|
⊢ (𝐴 ∪ (𝐴 ∖ 𝐵)) = 𝐴 |
|
Theorem | inundifss 3486 |
The intersection and class difference of a class with another class are
contained in the original class. In classical logic we'd be able to make
a stronger statement: that everything in the original class is in the
intersection or the difference (that is, this theorem would be equality
rather than subset). (Contributed by Jim Kingdon, 4-Aug-2018.)
|
⊢ ((𝐴 ∩ 𝐵) ∪ (𝐴 ∖ 𝐵)) ⊆ 𝐴 |
|
Theorem | disjdif2 3487 |
The difference of a class and a class disjoint from it is the original
class. (Contributed by BJ, 21-Apr-2019.)
|
⊢ ((𝐴 ∩ 𝐵) = ∅ → (𝐴 ∖ 𝐵) = 𝐴) |
|
Theorem | difun2 3488 |
Absorption of union by difference. Theorem 36 of [Suppes] p. 29.
(Contributed by NM, 19-May-1998.)
|
⊢ ((𝐴 ∪ 𝐵) ∖ 𝐵) = (𝐴 ∖ 𝐵) |
|
Theorem | undifss 3489 |
Union of complementary parts into whole. (Contributed by Jim Kingdon,
4-Aug-2018.)
|
⊢ (𝐴 ⊆ 𝐵 ↔ (𝐴 ∪ (𝐵 ∖ 𝐴)) ⊆ 𝐵) |
|
Theorem | ssdifin0 3490 |
A subset of a difference does not intersect the subtrahend. (Contributed
by Jeff Hankins, 1-Sep-2013.) (Proof shortened by Mario Carneiro,
24-Aug-2015.)
|
⊢ (𝐴 ⊆ (𝐵 ∖ 𝐶) → (𝐴 ∩ 𝐶) = ∅) |
|
Theorem | ssdifeq0 3491 |
A class is a subclass of itself subtracted from another iff it is the
empty set. (Contributed by Steve Rodriguez, 20-Nov-2015.)
|
⊢ (𝐴 ⊆ (𝐵 ∖ 𝐴) ↔ 𝐴 = ∅) |
|
Theorem | ssundifim 3492 |
A consequence of inclusion in the union of two classes. In classical
logic this would be a biconditional. (Contributed by Jim Kingdon,
4-Aug-2018.)
|
⊢ (𝐴 ⊆ (𝐵 ∪ 𝐶) → (𝐴 ∖ 𝐵) ⊆ 𝐶) |
|
Theorem | difdifdirss 3493 |
Distributive law for class difference. In classical logic, as in Exercise
4.8 of [Stoll] p. 16, this would be equality
rather than subset.
(Contributed by Jim Kingdon, 4-Aug-2018.)
|
⊢ ((𝐴 ∖ 𝐵) ∖ 𝐶) ⊆ ((𝐴 ∖ 𝐶) ∖ (𝐵 ∖ 𝐶)) |
|
Theorem | uneqdifeqim 3494 |
Two ways that 𝐴 and 𝐵 can
"partition" 𝐶 (when 𝐴 and 𝐵
don't overlap and 𝐴 is a part of 𝐶). In classical logic,
the
second implication would be a biconditional. (Contributed by Jim Kingdon,
4-Aug-2018.)
|
⊢ ((𝐴 ⊆ 𝐶 ∧ (𝐴 ∩ 𝐵) = ∅) → ((𝐴 ∪ 𝐵) = 𝐶 → (𝐶 ∖ 𝐴) = 𝐵)) |
|
Theorem | r19.2m 3495* |
Theorem 19.2 of [Margaris] p. 89 with
restricted quantifiers (compare
19.2 1626). The restricted version is valid only when
the domain of
quantification is inhabited. (Contributed by Jim Kingdon, 5-Aug-2018.)
(Revised by Jim Kingdon, 7-Apr-2023.)
|
⊢ ((∃𝑦 𝑦 ∈ 𝐴 ∧ ∀𝑥 ∈ 𝐴 𝜑) → ∃𝑥 ∈ 𝐴 𝜑) |
|
Theorem | r19.2mOLD 3496* |
Theorem 19.2 of [Margaris] p. 89 with
restricted quantifiers (compare
19.2 1626). The restricted version is valid only when
the domain of
quantification is inhabited. (Contributed by Jim Kingdon, 5-Aug-2018.)
Obsolete version of r19.2m 3495 as of 7-Apr-2023.
(Proof modification is discouraged.) (New usage is discouraged.)
|
⊢ ((∃𝑥 𝑥 ∈ 𝐴 ∧ ∀𝑥 ∈ 𝐴 𝜑) → ∃𝑥 ∈ 𝐴 𝜑) |
|
Theorem | r19.3rm 3497* |
Restricted quantification of wff not containing quantified variable.
(Contributed by Jim Kingdon, 19-Dec-2018.)
|
⊢ Ⅎ𝑥𝜑 ⇒ ⊢ (∃𝑦 𝑦 ∈ 𝐴 → (𝜑 ↔ ∀𝑥 ∈ 𝐴 𝜑)) |
|
Theorem | r19.28m 3498* |
Restricted quantifier version of Theorem 19.28 of [Margaris] p. 90. It
is valid only when the domain of quantification is inhabited.
(Contributed by Jim Kingdon, 5-Aug-2018.)
|
⊢ Ⅎ𝑥𝜑 ⇒ ⊢ (∃𝑥 𝑥 ∈ 𝐴 → (∀𝑥 ∈ 𝐴 (𝜑 ∧ 𝜓) ↔ (𝜑 ∧ ∀𝑥 ∈ 𝐴 𝜓))) |
|
Theorem | r19.3rmv 3499* |
Restricted quantification of wff not containing quantified variable.
(Contributed by Jim Kingdon, 6-Aug-2018.)
|
⊢ (∃𝑦 𝑦 ∈ 𝐴 → (𝜑 ↔ ∀𝑥 ∈ 𝐴 𝜑)) |
|
Theorem | r19.9rmv 3500* |
Restricted quantification of wff not containing quantified variable.
(Contributed by Jim Kingdon, 5-Aug-2018.)
|
⊢ (∃𝑦 𝑦 ∈ 𝐴 → (𝜑 ↔ ∃𝑥 ∈ 𝐴 𝜑)) |