Theorem List for Intuitionistic Logic Explorer - 3801-3900 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
Theorem | unissel 3801 |
Condition turning a subclass relationship for union into an equality.
(Contributed by NM, 18-Jul-2006.)
|
⊢ ((∪ 𝐴 ⊆ 𝐵 ∧ 𝐵 ∈ 𝐴) → ∪ 𝐴 = 𝐵) |
|
Theorem | unissb 3802* |
Relationship involving membership, subset, and union. Exercise 5 of
[Enderton] p. 26 and its converse.
(Contributed by NM, 20-Sep-2003.)
|
⊢ (∪ 𝐴 ⊆ 𝐵 ↔ ∀𝑥 ∈ 𝐴 𝑥 ⊆ 𝐵) |
|
Theorem | uniss2 3803* |
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 3804* |
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 3805* |
Relationship implying union. (Contributed by NM, 10-Nov-1999.)
|
⊢ ((𝐴 ∈ 𝐵 ∧ ∀𝑥 ∈ 𝐵 𝑥 ⊆ 𝐴) → 𝐴 = ∪ 𝐵) |
|
Theorem | unimax 3806* |
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 3807 |
Extend class notation to include the intersection of a class. Read:
"intersection (of) 𝐴".
|
class ∩ 𝐴 |
|
Definition | df-int 3808* |
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 3108.
(Contributed by NM, 18-Aug-1993.)
|
⊢ ∩ 𝐴 = {𝑥 ∣ ∀𝑦(𝑦 ∈ 𝐴 → 𝑥 ∈ 𝑦)} |
|
Theorem | dfint2 3809* |
Alternate definition of class intersection. (Contributed by NM,
28-Jun-1998.)
|
⊢ ∩ 𝐴 = {𝑥 ∣ ∀𝑦 ∈ 𝐴 𝑥 ∈ 𝑦} |
|
Theorem | inteq 3810 |
Equality law for intersection. (Contributed by NM, 13-Sep-1999.)
|
⊢ (𝐴 = 𝐵 → ∩ 𝐴 = ∩
𝐵) |
|
Theorem | inteqi 3811 |
Equality inference for class intersection. (Contributed by NM,
2-Sep-2003.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ ∩
𝐴 = ∩ 𝐵 |
|
Theorem | inteqd 3812 |
Equality deduction for class intersection. (Contributed by NM,
2-Sep-2003.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → ∩ 𝐴 = ∩
𝐵) |
|
Theorem | elint 3813* |
Membership in class intersection. (Contributed by NM, 21-May-1994.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ ∩ 𝐵 ↔ ∀𝑥(𝑥 ∈ 𝐵 → 𝐴 ∈ 𝑥)) |
|
Theorem | elint2 3814* |
Membership in class intersection. (Contributed by NM, 14-Oct-1999.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ ∩ 𝐵 ↔ ∀𝑥 ∈ 𝐵 𝐴 ∈ 𝑥) |
|
Theorem | elintg 3815* |
Membership in class intersection, with the sethood requirement expressed
as an antecedent. (Contributed by NM, 20-Nov-2003.)
|
⊢ (𝐴 ∈ 𝑉 → (𝐴 ∈ ∩ 𝐵 ↔ ∀𝑥 ∈ 𝐵 𝐴 ∈ 𝑥)) |
|
Theorem | elinti 3816 |
Membership in class intersection. (Contributed by NM, 14-Oct-1999.)
(Proof shortened by Andrew Salmon, 9-Jul-2011.)
|
⊢ (𝐴 ∈ ∩ 𝐵 → (𝐶 ∈ 𝐵 → 𝐴 ∈ 𝐶)) |
|
Theorem | nfint 3817 |
Bound-variable hypothesis builder for intersection. (Contributed by NM,
2-Feb-1997.) (Proof shortened by Andrew Salmon, 12-Aug-2011.)
|
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ Ⅎ𝑥∩
𝐴 |
|
Theorem | elintab 3818* |
Membership in the intersection of a class abstraction. (Contributed by
NM, 30-Aug-1993.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ ∩ {𝑥 ∣ 𝜑} ↔ ∀𝑥(𝜑 → 𝐴 ∈ 𝑥)) |
|
Theorem | elintrab 3819* |
Membership in the intersection of a class abstraction. (Contributed by
NM, 17-Oct-1999.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ ∩ {𝑥 ∈ 𝐵 ∣ 𝜑} ↔ ∀𝑥 ∈ 𝐵 (𝜑 → 𝐴 ∈ 𝑥)) |
|
Theorem | elintrabg 3820* |
Membership in the intersection of a class abstraction. (Contributed by
NM, 17-Feb-2007.)
|
⊢ (𝐴 ∈ 𝑉 → (𝐴 ∈ ∩ {𝑥 ∈ 𝐵 ∣ 𝜑} ↔ ∀𝑥 ∈ 𝐵 (𝜑 → 𝐴 ∈ 𝑥))) |
|
Theorem | int0 3821 |
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 3822 |
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 3823* |
Subclass of a class intersection. Theorem 5.11(viii) of [Monk1] p. 52
and its converse. (Contributed by NM, 14-Oct-1999.)
|
⊢ (𝐴 ⊆ ∩ 𝐵 ↔ ∀𝑥 ∈ 𝐵 𝐴 ⊆ 𝑥) |
|
Theorem | ssintab 3824* |
Subclass of the intersection of a class abstraction. (Contributed by
NM, 31-Jul-2006.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
|
⊢ (𝐴 ⊆ ∩
{𝑥 ∣ 𝜑} ↔ ∀𝑥(𝜑 → 𝐴 ⊆ 𝑥)) |
|
Theorem | ssintub 3825* |
Subclass of the least upper bound. (Contributed by NM, 8-Aug-2000.)
|
⊢ 𝐴 ⊆ ∩
{𝑥 ∈ 𝐵 ∣ 𝐴 ⊆ 𝑥} |
|
Theorem | ssmin 3826* |
Subclass of the minimum value of class of supersets. (Contributed by
NM, 10-Aug-2006.)
|
⊢ 𝐴 ⊆ ∩
{𝑥 ∣ (𝐴 ⊆ 𝑥 ∧ 𝜑)} |
|
Theorem | intmin 3827* |
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 3828 |
Intersection of subclasses. (Contributed by NM, 14-Oct-1999.)
|
⊢ (𝐴 ⊆ 𝐵 → ∩ 𝐵 ⊆ ∩ 𝐴) |
|
Theorem | intssunim 3829* |
The intersection of an inhabited set is a subclass of its union.
(Contributed by NM, 29-Jul-2006.)
|
⊢ (∃𝑥 𝑥 ∈ 𝐴 → ∩ 𝐴 ⊆ ∪ 𝐴) |
|
Theorem | ssintrab 3830* |
Subclass of the intersection of a restricted class builder.
(Contributed by NM, 30-Jan-2015.)
|
⊢ (𝐴 ⊆ ∩
{𝑥 ∈ 𝐵 ∣ 𝜑} ↔ ∀𝑥 ∈ 𝐵 (𝜑 → 𝐴 ⊆ 𝑥)) |
|
Theorem | intssuni2m 3831* |
Subclass relationship for intersection and union. (Contributed by Jim
Kingdon, 14-Aug-2018.)
|
⊢ ((𝐴 ⊆ 𝐵 ∧ ∃𝑥 𝑥 ∈ 𝐴) → ∩ 𝐴 ⊆ ∪ 𝐵) |
|
Theorem | intminss 3832* |
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 3833* |
Any set is the smallest of all sets that include it. (Contributed by
NM, 20-Sep-2003.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ ∩
{𝑥 ∣ 𝐴 ⊆ 𝑥} = 𝐴 |
|
Theorem | intmin3 3834* |
Under subset ordering, the intersection of a class abstraction is less
than or equal to any of its members. (Contributed by NM,
3-Jul-2005.)
|
⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜓)) & ⊢ 𝜓 ⇒ ⊢ (𝐴 ∈ 𝑉 → ∩ {𝑥 ∣ 𝜑} ⊆ 𝐴) |
|
Theorem | intmin4 3835* |
Elimination of a conjunct in a class intersection. (Contributed by NM,
31-Jul-2006.)
|
⊢ (𝐴 ⊆ ∩
{𝑥 ∣ 𝜑} → ∩
{𝑥 ∣ (𝐴 ⊆ 𝑥 ∧ 𝜑)} = ∩ {𝑥 ∣ 𝜑}) |
|
Theorem | intab 3836* |
The intersection of a special case of a class abstraction. 𝑦 may be
free in 𝜑 and 𝐴, which can be thought of
a 𝜑(𝑦) and
𝐴(𝑦). (Contributed by NM, 28-Jul-2006.)
(Proof shortened by
Mario Carneiro, 14-Nov-2016.)
|
⊢ 𝐴 ∈ V & ⊢ {𝑥 ∣ ∃𝑦(𝜑 ∧ 𝑥 = 𝐴)} ∈ V ⇒ ⊢ ∩
{𝑥 ∣ ∀𝑦(𝜑 → 𝐴 ∈ 𝑥)} = {𝑥 ∣ ∃𝑦(𝜑 ∧ 𝑥 = 𝐴)} |
|
Theorem | int0el 3837 |
The intersection of a class containing the empty set is empty.
(Contributed by NM, 24-Apr-2004.)
|
⊢ (∅ ∈ 𝐴 → ∩ 𝐴 = ∅) |
|
Theorem | intun 3838 |
The class intersection of the union of two classes. Theorem 78 of
[Suppes] p. 42. (Contributed by NM,
22-Sep-2002.)
|
⊢ ∩ (𝐴 ∪ 𝐵) = (∩ 𝐴 ∩ ∩ 𝐵) |
|
Theorem | intpr 3839 |
The intersection of a pair is the intersection of its members. Theorem
71 of [Suppes] p. 42. (Contributed by
NM, 14-Oct-1999.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ ∩
{𝐴, 𝐵} = (𝐴 ∩ 𝐵) |
|
Theorem | intprg 3840 |
The intersection of a pair is the intersection of its members. Closed
form of intpr 3839. Theorem 71 of [Suppes] p. 42. (Contributed by FL,
27-Apr-2008.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → ∩
{𝐴, 𝐵} = (𝐴 ∩ 𝐵)) |
|
Theorem | intsng 3841 |
Intersection of a singleton. (Contributed by Stefan O'Rear,
22-Feb-2015.)
|
⊢ (𝐴 ∈ 𝑉 → ∩ {𝐴} = 𝐴) |
|
Theorem | intsn 3842 |
The intersection of a singleton is its member. Theorem 70 of [Suppes]
p. 41. (Contributed by NM, 29-Sep-2002.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ ∩
{𝐴} = 𝐴 |
|
Theorem | uniintsnr 3843* |
The union and intersection of a singleton are equal. See also eusn 3633.
(Contributed by Jim Kingdon, 14-Aug-2018.)
|
⊢ (∃𝑥 𝐴 = {𝑥} → ∪ 𝐴 = ∩
𝐴) |
|
Theorem | uniintabim 3844 |
The union and the intersection of a class abstraction are equal if there
is a unique satisfying value of 𝜑(𝑥). (Contributed by Jim
Kingdon, 14-Aug-2018.)
|
⊢ (∃!𝑥𝜑 → ∪ {𝑥 ∣ 𝜑} = ∩ {𝑥 ∣ 𝜑}) |
|
Theorem | intunsn 3845 |
Theorem joining a singleton to an intersection. (Contributed by NM,
29-Sep-2002.)
|
⊢ 𝐵 ∈ V ⇒ ⊢ ∩
(𝐴 ∪ {𝐵}) = (∩ 𝐴
∩ 𝐵) |
|
Theorem | rint0 3846 |
Relative intersection of an empty set. (Contributed by Stefan O'Rear,
3-Apr-2015.)
|
⊢ (𝑋 = ∅ → (𝐴 ∩ ∩ 𝑋) = 𝐴) |
|
Theorem | elrint 3847* |
Membership in a restricted intersection. (Contributed by Stefan O'Rear,
3-Apr-2015.)
|
⊢ (𝑋 ∈ (𝐴 ∩ ∩ 𝐵) ↔ (𝑋 ∈ 𝐴 ∧ ∀𝑦 ∈ 𝐵 𝑋 ∈ 𝑦)) |
|
Theorem | elrint2 3848* |
Membership in a restricted intersection. (Contributed by Stefan O'Rear,
3-Apr-2015.)
|
⊢ (𝑋 ∈ 𝐴 → (𝑋 ∈ (𝐴 ∩ ∩ 𝐵) ↔ ∀𝑦 ∈ 𝐵 𝑋 ∈ 𝑦)) |
|
2.1.20 Indexed union and
intersection
|
|
Syntax | ciun 3849 |
Extend class notation to include indexed union. Note: Historically
(prior to 21-Oct-2005), set.mm used the notation ∪ 𝑥
∈ 𝐴𝐵, with
the same union symbol as cuni 3772. While that syntax was unambiguous, it
did not allow for LALR parsing of the syntax constructions in set.mm. The
new syntax uses as distinguished symbol ∪ instead of ∪ and does
allow LALR parsing. Thanks to Peter Backes for suggesting this change.
|
class ∪ 𝑥 ∈ 𝐴 𝐵 |
|
Syntax | ciin 3850 |
Extend class notation to include indexed intersection. Note:
Historically (prior to 21-Oct-2005), set.mm used the notation
∩ 𝑥 ∈ 𝐴𝐵, with the same intersection symbol
as cint 3807. Although
that syntax was unambiguous, it did not allow for LALR parsing of the
syntax constructions in set.mm. The new syntax uses a distinguished
symbol ∩ instead
of ∩ and does allow LALR
parsing. Thanks to
Peter Backes for suggesting this change.
|
class ∩ 𝑥 ∈ 𝐴 𝐵 |
|
Definition | df-iun 3851* |
Define indexed union. Definition indexed union in [Stoll] p. 45. In
most applications, 𝐴 is independent of 𝑥
(although this is not
required by the definition), and 𝐵 depends on 𝑥 i.e. can be read
informally as 𝐵(𝑥). We call 𝑥 the index, 𝐴 the
index
set, and 𝐵 the indexed set. In most books,
𝑥 ∈
𝐴 is written as
a subscript or underneath a union symbol ∪. We use a special
union symbol ∪
to make it easier to distinguish from plain class
union. In many theorems, you will see that 𝑥 and 𝐴 are in
the
same disjoint variable group (meaning 𝐴 cannot depend on 𝑥) and
that 𝐵 and 𝑥 do not share a disjoint
variable group (meaning
that can be thought of as 𝐵(𝑥) i.e. can be substituted with a
class expression containing 𝑥). An alternate definition tying
indexed union to ordinary union is dfiun2 3883. Theorem uniiun 3902 provides
a definition of ordinary union in terms of indexed union. (Contributed
by NM, 27-Jun-1998.)
|
⊢ ∪ 𝑥 ∈ 𝐴 𝐵 = {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 ∈ 𝐵} |
|
Definition | df-iin 3852* |
Define indexed intersection. Definition of [Stoll] p. 45. See the
remarks for its sibling operation of indexed union df-iun 3851. An
alternate definition tying indexed intersection to ordinary intersection
is dfiin2 3884. Theorem intiin 3903 provides a definition of ordinary
intersection in terms of indexed intersection. (Contributed by NM,
27-Jun-1998.)
|
⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = {𝑦 ∣ ∀𝑥 ∈ 𝐴 𝑦 ∈ 𝐵} |
|
Theorem | eliun 3853* |
Membership in indexed union. (Contributed by NM, 3-Sep-2003.)
|
⊢ (𝐴 ∈ ∪
𝑥 ∈ 𝐵 𝐶 ↔ ∃𝑥 ∈ 𝐵 𝐴 ∈ 𝐶) |
|
Theorem | eliin 3854* |
Membership in indexed intersection. (Contributed by NM, 3-Sep-2003.)
|
⊢ (𝐴 ∈ 𝑉 → (𝐴 ∈ ∩
𝑥 ∈ 𝐵 𝐶 ↔ ∀𝑥 ∈ 𝐵 𝐴 ∈ 𝐶)) |
|
Theorem | iuncom 3855* |
Commutation of indexed unions. (Contributed by NM, 18-Dec-2008.)
|
⊢ ∪ 𝑥 ∈ 𝐴 ∪ 𝑦 ∈ 𝐵 𝐶 = ∪
𝑦 ∈ 𝐵 ∪ 𝑥 ∈ 𝐴 𝐶 |
|
Theorem | iuncom4 3856 |
Commutation of union with indexed union. (Contributed by Mario
Carneiro, 18-Jan-2014.)
|
⊢ ∪ 𝑥 ∈ 𝐴 ∪ 𝐵 = ∪
∪ 𝑥 ∈ 𝐴 𝐵 |
|
Theorem | iunconstm 3857* |
Indexed union of a constant class, i.e. where 𝐵 does not depend on
𝑥. (Contributed by Jim Kingdon,
15-Aug-2018.)
|
⊢ (∃𝑥 𝑥 ∈ 𝐴 → ∪
𝑥 ∈ 𝐴 𝐵 = 𝐵) |
|
Theorem | iinconstm 3858* |
Indexed intersection of a constant class, i.e. where 𝐵 does not
depend on 𝑥. (Contributed by Jim Kingdon,
19-Dec-2018.)
|
⊢ (∃𝑦 𝑦 ∈ 𝐴 → ∩
𝑥 ∈ 𝐴 𝐵 = 𝐵) |
|
Theorem | iuniin 3859* |
Law combining indexed union with indexed intersection. Eq. 14 in
[KuratowskiMostowski] p.
109. This theorem also appears as the last
example at http://en.wikipedia.org/wiki/Union%5F%28set%5Ftheory%29.
(Contributed by NM, 17-Aug-2004.) (Proof shortened by Andrew Salmon,
25-Jul-2011.)
|
⊢ ∪ 𝑥 ∈ 𝐴 ∩ 𝑦 ∈ 𝐵 𝐶 ⊆ ∩ 𝑦 ∈ 𝐵 ∪ 𝑥 ∈ 𝐴 𝐶 |
|
Theorem | iunss1 3860* |
Subclass theorem for indexed union. (Contributed by NM, 10-Dec-2004.)
(Proof shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ (𝐴 ⊆ 𝐵 → ∪
𝑥 ∈ 𝐴 𝐶 ⊆ ∪ 𝑥 ∈ 𝐵 𝐶) |
|
Theorem | iinss1 3861* |
Subclass theorem for indexed union. (Contributed by NM,
24-Jan-2012.)
|
⊢ (𝐴 ⊆ 𝐵 → ∩
𝑥 ∈ 𝐵 𝐶 ⊆ ∩ 𝑥 ∈ 𝐴 𝐶) |
|
Theorem | iuneq1 3862* |
Equality theorem for indexed union. (Contributed by NM,
27-Jun-1998.)
|
⊢ (𝐴 = 𝐵 → ∪
𝑥 ∈ 𝐴 𝐶 = ∪
𝑥 ∈ 𝐵 𝐶) |
|
Theorem | iineq1 3863* |
Equality theorem for restricted existential quantifier. (Contributed by
NM, 27-Jun-1998.)
|
⊢ (𝐴 = 𝐵 → ∩
𝑥 ∈ 𝐴 𝐶 = ∩
𝑥 ∈ 𝐵 𝐶) |
|
Theorem | ss2iun 3864 |
Subclass theorem for indexed union. (Contributed by NM, 26-Nov-2003.)
(Proof shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ (∀𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶 → ∪
𝑥 ∈ 𝐴 𝐵 ⊆ ∪ 𝑥 ∈ 𝐴 𝐶) |
|
Theorem | iuneq2 3865 |
Equality theorem for indexed union. (Contributed by NM,
22-Oct-2003.)
|
⊢ (∀𝑥 ∈ 𝐴 𝐵 = 𝐶 → ∪
𝑥 ∈ 𝐴 𝐵 = ∪
𝑥 ∈ 𝐴 𝐶) |
|
Theorem | iineq2 3866 |
Equality theorem for indexed intersection. (Contributed by NM,
22-Oct-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ (∀𝑥 ∈ 𝐴 𝐵 = 𝐶 → ∩
𝑥 ∈ 𝐴 𝐵 = ∩
𝑥 ∈ 𝐴 𝐶) |
|
Theorem | iuneq2i 3867 |
Equality inference for indexed union. (Contributed by NM,
22-Oct-2003.)
|
⊢ (𝑥 ∈ 𝐴 → 𝐵 = 𝐶) ⇒ ⊢ ∪ 𝑥 ∈ 𝐴 𝐵 = ∪
𝑥 ∈ 𝐴 𝐶 |
|
Theorem | iineq2i 3868 |
Equality inference for indexed intersection. (Contributed by NM,
22-Oct-2003.)
|
⊢ (𝑥 ∈ 𝐴 → 𝐵 = 𝐶) ⇒ ⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = ∩
𝑥 ∈ 𝐴 𝐶 |
|
Theorem | iineq2d 3869 |
Equality deduction for indexed intersection. (Contributed by NM,
7-Dec-2011.)
|
⊢ Ⅎ𝑥𝜑
& ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → ∩
𝑥 ∈ 𝐴 𝐵 = ∩
𝑥 ∈ 𝐴 𝐶) |
|
Theorem | iuneq2dv 3870* |
Equality deduction for indexed union. (Contributed by NM,
3-Aug-2004.)
|
⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → ∪
𝑥 ∈ 𝐴 𝐵 = ∪
𝑥 ∈ 𝐴 𝐶) |
|
Theorem | iineq2dv 3871* |
Equality deduction for indexed intersection. (Contributed by NM,
3-Aug-2004.)
|
⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → ∩
𝑥 ∈ 𝐴 𝐵 = ∩
𝑥 ∈ 𝐴 𝐶) |
|
Theorem | iuneq1d 3872* |
Equality theorem for indexed union, deduction version. (Contributed by
Drahflow, 22-Oct-2015.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → ∪
𝑥 ∈ 𝐴 𝐶 = ∪
𝑥 ∈ 𝐵 𝐶) |
|
Theorem | iuneq12d 3873* |
Equality deduction for indexed union, deduction version. (Contributed
by Drahflow, 22-Oct-2015.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → ∪
𝑥 ∈ 𝐴 𝐶 = ∪
𝑥 ∈ 𝐵 𝐷) |
|
Theorem | iuneq2d 3874* |
Equality deduction for indexed union. (Contributed by Drahflow,
22-Oct-2015.)
|
⊢ (𝜑 → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → ∪
𝑥 ∈ 𝐴 𝐵 = ∪
𝑥 ∈ 𝐴 𝐶) |
|
Theorem | nfiunxy 3875* |
Bound-variable hypothesis builder for indexed union. (Contributed by
Mario Carneiro, 25-Jan-2014.)
|
⊢ Ⅎ𝑦𝐴
& ⊢ Ⅎ𝑦𝐵 ⇒ ⊢ Ⅎ𝑦∪ 𝑥 ∈ 𝐴 𝐵 |
|
Theorem | nfiinxy 3876* |
Bound-variable hypothesis builder for indexed intersection.
(Contributed by Mario Carneiro, 25-Jan-2014.)
|
⊢ Ⅎ𝑦𝐴
& ⊢ Ⅎ𝑦𝐵 ⇒ ⊢ Ⅎ𝑦∩ 𝑥 ∈ 𝐴 𝐵 |
|
Theorem | nfiunya 3877* |
Bound-variable hypothesis builder for indexed union. (Contributed by
Mario Carneiro, 25-Jan-2014.)
|
⊢ Ⅎ𝑦𝐴
& ⊢ Ⅎ𝑦𝐵 ⇒ ⊢ Ⅎ𝑦∪ 𝑥 ∈ 𝐴 𝐵 |
|
Theorem | nfiinya 3878* |
Bound-variable hypothesis builder for indexed intersection.
(Contributed by Mario Carneiro, 25-Jan-2014.)
|
⊢ Ⅎ𝑦𝐴
& ⊢ Ⅎ𝑦𝐵 ⇒ ⊢ Ⅎ𝑦∩ 𝑥 ∈ 𝐴 𝐵 |
|
Theorem | nfiu1 3879 |
Bound-variable hypothesis builder for indexed union. (Contributed by
NM, 12-Oct-2003.)
|
⊢ Ⅎ𝑥∪ 𝑥 ∈ 𝐴 𝐵 |
|
Theorem | nfii1 3880 |
Bound-variable hypothesis builder for indexed intersection.
(Contributed by NM, 15-Oct-2003.)
|
⊢ Ⅎ𝑥∩ 𝑥 ∈ 𝐴 𝐵 |
|
Theorem | dfiun2g 3881* |
Alternate definition of indexed union when 𝐵 is a set. Definition
15(a) of [Suppes] p. 44. (Contributed by
NM, 23-Mar-2006.) (Proof
shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ (∀𝑥 ∈ 𝐴 𝐵 ∈ 𝐶 → ∪
𝑥 ∈ 𝐴 𝐵 = ∪ {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵}) |
|
Theorem | dfiin2g 3882* |
Alternate definition of indexed intersection when 𝐵 is a set.
(Contributed by Jeff Hankins, 27-Aug-2009.)
|
⊢ (∀𝑥 ∈ 𝐴 𝐵 ∈ 𝐶 → ∩
𝑥 ∈ 𝐴 𝐵 = ∩ {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵}) |
|
Theorem | dfiun2 3883* |
Alternate definition of indexed union when 𝐵 is a set. Definition
15(a) of [Suppes] p. 44. (Contributed by
NM, 27-Jun-1998.) (Revised by
David Abernethy, 19-Jun-2012.)
|
⊢ 𝐵 ∈ V ⇒ ⊢ ∪ 𝑥 ∈ 𝐴 𝐵 = ∪ {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵} |
|
Theorem | dfiin2 3884* |
Alternate definition of indexed intersection when 𝐵 is a set.
Definition 15(b) of [Suppes] p. 44.
(Contributed by NM, 28-Jun-1998.)
(Proof shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ 𝐵 ∈ V ⇒ ⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵} |
|
Theorem | dfiunv2 3885* |
Define double indexed union. (Contributed by FL, 6-Nov-2013.)
|
⊢ ∪ 𝑥 ∈ 𝐴 ∪ 𝑦 ∈ 𝐵 𝐶 = {𝑧 ∣ ∃𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝑧 ∈ 𝐶} |
|
Theorem | cbviun 3886* |
Rule used to change the bound variables in an indexed union, with the
substitution specified implicitly by the hypothesis. (Contributed by
NM, 26-Mar-2006.) (Revised by Andrew Salmon, 25-Jul-2011.)
|
⊢ Ⅎ𝑦𝐵
& ⊢ Ⅎ𝑥𝐶
& ⊢ (𝑥 = 𝑦 → 𝐵 = 𝐶) ⇒ ⊢ ∪ 𝑥 ∈ 𝐴 𝐵 = ∪
𝑦 ∈ 𝐴 𝐶 |
|
Theorem | cbviin 3887* |
Change bound variables in an indexed intersection. (Contributed by Jeff
Hankins, 26-Aug-2009.) (Revised by Mario Carneiro, 14-Oct-2016.)
|
⊢ Ⅎ𝑦𝐵
& ⊢ Ⅎ𝑥𝐶
& ⊢ (𝑥 = 𝑦 → 𝐵 = 𝐶) ⇒ ⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = ∩
𝑦 ∈ 𝐴 𝐶 |
|
Theorem | cbviunv 3888* |
Rule used to change the bound variables in an indexed union, with the
substitution specified implicitly by the hypothesis. (Contributed by
NM, 15-Sep-2003.)
|
⊢ (𝑥 = 𝑦 → 𝐵 = 𝐶) ⇒ ⊢ ∪ 𝑥 ∈ 𝐴 𝐵 = ∪
𝑦 ∈ 𝐴 𝐶 |
|
Theorem | cbviinv 3889* |
Change bound variables in an indexed intersection. (Contributed by Jeff
Hankins, 26-Aug-2009.)
|
⊢ (𝑥 = 𝑦 → 𝐵 = 𝐶) ⇒ ⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = ∩
𝑦 ∈ 𝐴 𝐶 |
|
Theorem | iunss 3890* |
Subset theorem for an indexed union. (Contributed by NM, 13-Sep-2003.)
(Proof shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ (∪ 𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶 ↔ ∀𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶) |
|
Theorem | ssiun 3891* |
Subset implication for an indexed union. (Contributed by NM,
3-Sep-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ (∃𝑥 ∈ 𝐴 𝐶 ⊆ 𝐵 → 𝐶 ⊆ ∪ 𝑥 ∈ 𝐴 𝐵) |
|
Theorem | ssiun2 3892 |
Identity law for subset of an indexed union. (Contributed by NM,
12-Oct-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ (𝑥 ∈ 𝐴 → 𝐵 ⊆ ∪ 𝑥 ∈ 𝐴 𝐵) |
|
Theorem | ssiun2s 3893* |
Subset relationship for an indexed union. (Contributed by NM,
26-Oct-2003.)
|
⊢ (𝑥 = 𝐶 → 𝐵 = 𝐷) ⇒ ⊢ (𝐶 ∈ 𝐴 → 𝐷 ⊆ ∪ 𝑥 ∈ 𝐴 𝐵) |
|
Theorem | iunss2 3894* |
A subclass condition on the members of two indexed classes 𝐶(𝑥)
and 𝐷(𝑦) that implies a subclass relation on
their indexed
unions. Generalization of Proposition 8.6 of [TakeutiZaring] p. 59.
Compare uniss2 3803. (Contributed by NM, 9-Dec-2004.)
|
⊢ (∀𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝐶 ⊆ 𝐷 → ∪
𝑥 ∈ 𝐴 𝐶 ⊆ ∪ 𝑦 ∈ 𝐵 𝐷) |
|
Theorem | iunab 3895* |
The indexed union of a class abstraction. (Contributed by NM,
27-Dec-2004.)
|
⊢ ∪ 𝑥 ∈ 𝐴 {𝑦 ∣ 𝜑} = {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝜑} |
|
Theorem | iunrab 3896* |
The indexed union of a restricted class abstraction. (Contributed by
NM, 3-Jan-2004.) (Proof shortened by Mario Carneiro, 14-Nov-2016.)
|
⊢ ∪ 𝑥 ∈ 𝐴 {𝑦 ∈ 𝐵 ∣ 𝜑} = {𝑦 ∈ 𝐵 ∣ ∃𝑥 ∈ 𝐴 𝜑} |
|
Theorem | iunxdif2 3897* |
Indexed union with a class difference as its index. (Contributed by NM,
10-Dec-2004.)
|
⊢ (𝑥 = 𝑦 → 𝐶 = 𝐷) ⇒ ⊢ (∀𝑥 ∈ 𝐴 ∃𝑦 ∈ (𝐴 ∖ 𝐵)𝐶 ⊆ 𝐷 → ∪
𝑦 ∈ (𝐴 ∖ 𝐵)𝐷 = ∪
𝑥 ∈ 𝐴 𝐶) |
|
Theorem | ssiinf 3898 |
Subset theorem for an indexed intersection. (Contributed by FL,
15-Oct-2012.) (Proof shortened by Mario Carneiro, 14-Oct-2016.)
|
⊢ Ⅎ𝑥𝐶 ⇒ ⊢ (𝐶 ⊆ ∩ 𝑥 ∈ 𝐴 𝐵 ↔ ∀𝑥 ∈ 𝐴 𝐶 ⊆ 𝐵) |
|
Theorem | ssiin 3899* |
Subset theorem for an indexed intersection. (Contributed by NM,
15-Oct-2003.)
|
⊢ (𝐶 ⊆ ∩ 𝑥 ∈ 𝐴 𝐵 ↔ ∀𝑥 ∈ 𝐴 𝐶 ⊆ 𝐵) |
|
Theorem | iinss 3900* |
Subset implication for an indexed intersection. (Contributed by NM,
15-Oct-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.)
|
⊢ (∃𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶 → ∩
𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶) |