![]() |
Metamath
Proof Explorer Theorem List (p. 46 of 426) | < Previous Next > |
Bad symbols? Try the
GIF version. |
||
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Color key: | ![]() (1-27775) |
![]() (27776-29300) |
![]() (29301-42551) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | unissint 4501 | If the union of a class is included in its intersection, the class is either the empty set or a singleton (uniintsn 4514). (Contributed by NM, 30-Oct-2010.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (∪ 𝐴 ⊆ ∩ 𝐴 ↔ (𝐴 = ∅ ∨ ∪ 𝐴 = ∩ 𝐴)) | ||
Theorem | intssuni2 4502 | Subclass relationship for intersection and union. (Contributed by NM, 29-Jul-2006.) |
⊢ ((𝐴 ⊆ 𝐵 ∧ 𝐴 ≠ ∅) → ∩ 𝐴 ⊆ ∪ 𝐵) | ||
Theorem | intminss 4503* | 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 4504* | Any set is the smallest of all sets that include it. (Contributed by NM, 20-Sep-2003.) |
⊢ 𝐴 ∈ V ⇒ ⊢ ∩ {𝑥 ∣ 𝐴 ⊆ 𝑥} = 𝐴 | ||
Theorem | intmin3 4505* | 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 4506* | Elimination of a conjunct in a class intersection. (Contributed by NM, 31-Jul-2006.) |
⊢ (𝐴 ⊆ ∩ {𝑥 ∣ 𝜑} → ∩ {𝑥 ∣ (𝐴 ⊆ 𝑥 ∧ 𝜑)} = ∩ {𝑥 ∣ 𝜑}) | ||
Theorem | intab 4507* | The intersection of a special case of a class abstraction. 𝑦 may be free in 𝜑 and 𝐴, which can be thought of a 𝜑(𝑦) and 𝐴(𝑦). Typically, abrexex2 7148 or abexssex 7149 can be used to satisfy the second hypothesis. (Contributed by NM, 28-Jul-2006.) (Proof shortened by Mario Carneiro, 14-Nov-2016.) |
⊢ 𝐴 ∈ V & ⊢ {𝑥 ∣ ∃𝑦(𝜑 ∧ 𝑥 = 𝐴)} ∈ V ⇒ ⊢ ∩ {𝑥 ∣ ∀𝑦(𝜑 → 𝐴 ∈ 𝑥)} = {𝑥 ∣ ∃𝑦(𝜑 ∧ 𝑥 = 𝐴)} | ||
Theorem | int0el 4508 | The intersection of a class containing the empty set is empty. (Contributed by NM, 24-Apr-2004.) |
⊢ (∅ ∈ 𝐴 → ∩ 𝐴 = ∅) | ||
Theorem | intun 4509 | The class intersection of the union of two classes. Theorem 78 of [Suppes] p. 42. (Contributed by NM, 22-Sep-2002.) |
⊢ ∩ (𝐴 ∪ 𝐵) = (∩ 𝐴 ∩ ∩ 𝐵) | ||
Theorem | intpr 4510 | 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 4511 | The intersection of a pair is the intersection of its members. Closed form of intpr 4510. Theorem 71 of [Suppes] p. 42. (Contributed by FL, 27-Apr-2008.) |
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → ∩ {𝐴, 𝐵} = (𝐴 ∩ 𝐵)) | ||
Theorem | intsng 4512 | Intersection of a singleton. (Contributed by Stefan O'Rear, 22-Feb-2015.) |
⊢ (𝐴 ∈ 𝑉 → ∩ {𝐴} = 𝐴) | ||
Theorem | intsn 4513 | The intersection of a singleton is its member. Theorem 70 of [Suppes] p. 41. (Contributed by NM, 29-Sep-2002.) |
⊢ 𝐴 ∈ V ⇒ ⊢ ∩ {𝐴} = 𝐴 | ||
Theorem | uniintsn 4514* | Two ways to express "𝐴 is a singleton." See also en1 8023, en1b 8024, card1 8794, and eusn 4265. (Contributed by NM, 2-Aug-2010.) |
⊢ (∪ 𝐴 = ∩ 𝐴 ↔ ∃𝑥 𝐴 = {𝑥}) | ||
Theorem | uniintab 4515 | The union and the intersection of a class abstraction are equal exactly when there is a unique satisfying value of 𝜑(𝑥). (Contributed by Mario Carneiro, 24-Dec-2016.) |
⊢ (∃!𝑥𝜑 ↔ ∪ {𝑥 ∣ 𝜑} = ∩ {𝑥 ∣ 𝜑}) | ||
Theorem | intunsn 4516 | Theorem joining a singleton to an intersection. (Contributed by NM, 29-Sep-2002.) |
⊢ 𝐵 ∈ V ⇒ ⊢ ∩ (𝐴 ∪ {𝐵}) = (∩ 𝐴 ∩ 𝐵) | ||
Theorem | rint0 4517 | Relative intersection of an empty set. (Contributed by Stefan O'Rear, 3-Apr-2015.) |
⊢ (𝑋 = ∅ → (𝐴 ∩ ∩ 𝑋) = 𝐴) | ||
Theorem | elrint 4518* | Membership in a restricted intersection. (Contributed by Stefan O'Rear, 3-Apr-2015.) |
⊢ (𝑋 ∈ (𝐴 ∩ ∩ 𝐵) ↔ (𝑋 ∈ 𝐴 ∧ ∀𝑦 ∈ 𝐵 𝑋 ∈ 𝑦)) | ||
Theorem | elrint2 4519* | Membership in a restricted intersection. (Contributed by Stefan O'Rear, 3-Apr-2015.) |
⊢ (𝑋 ∈ 𝐴 → (𝑋 ∈ (𝐴 ∩ ∩ 𝐵) ↔ ∀𝑦 ∈ 𝐵 𝑋 ∈ 𝑦)) | ||
Syntax | ciun 4520 | 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 4436. While 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 ∪ 𝑥 ∈ 𝐴 𝐵 | ||
Syntax | ciin 4521 | 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 4475. 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 4522* | 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 distinct variable group (meaning 𝐴 cannot depend on 𝑥) and that 𝐵 and 𝑥 do not share a distinct 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 4554. Theorem uniiun 4573 provides a definition of ordinary union in terms of indexed union. Theorems fniunfv 6505 and funiunfv 6506 are useful when 𝐵 is a function. (Contributed by NM, 27-Jun-1998.) |
⊢ ∪ 𝑥 ∈ 𝐴 𝐵 = {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 ∈ 𝐵} | ||
Definition | df-iin 4523* | Define indexed intersection. Definition of [Stoll] p. 45. See the remarks for its sibling operation of indexed union df-iun 4522. An alternate definition tying indexed intersection to ordinary intersection is dfiin2 4555. Theorem intiin 4574 provides a definition of ordinary intersection in terms of indexed intersection. (Contributed by NM, 27-Jun-1998.) |
⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = {𝑦 ∣ ∀𝑥 ∈ 𝐴 𝑦 ∈ 𝐵} | ||
Theorem | eliun 4524* | Membership in indexed union. (Contributed by NM, 3-Sep-2003.) |
⊢ (𝐴 ∈ ∪ 𝑥 ∈ 𝐵 𝐶 ↔ ∃𝑥 ∈ 𝐵 𝐴 ∈ 𝐶) | ||
Theorem | eliin 4525* | Membership in indexed intersection. (Contributed by NM, 3-Sep-2003.) |
⊢ (𝐴 ∈ 𝑉 → (𝐴 ∈ ∩ 𝑥 ∈ 𝐵 𝐶 ↔ ∀𝑥 ∈ 𝐵 𝐴 ∈ 𝐶)) | ||
Theorem | eliuni 4526* | Membership in an indexed union, one way. (Contributed by JJ, 27-Jul-2021.) |
⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶) ⇒ ⊢ ((𝐴 ∈ 𝐷 ∧ 𝐸 ∈ 𝐶) → 𝐸 ∈ ∪ 𝑥 ∈ 𝐷 𝐵) | ||
Theorem | iuncom 4527* | Commutation of indexed unions. (Contributed by NM, 18-Dec-2008.) |
⊢ ∪ 𝑥 ∈ 𝐴 ∪ 𝑦 ∈ 𝐵 𝐶 = ∪ 𝑦 ∈ 𝐵 ∪ 𝑥 ∈ 𝐴 𝐶 | ||
Theorem | iuncom4 4528 | Commutation of union with indexed union. (Contributed by Mario Carneiro, 18-Jan-2014.) |
⊢ ∪ 𝑥 ∈ 𝐴 ∪ 𝐵 = ∪ ∪ 𝑥 ∈ 𝐴 𝐵 | ||
Theorem | iunconst 4529* | Indexed union of a constant class, i.e. where 𝐵 does not depend on 𝑥. (Contributed by NM, 5-Sep-2004.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (𝐴 ≠ ∅ → ∪ 𝑥 ∈ 𝐴 𝐵 = 𝐵) | ||
Theorem | iinconst 4530* | Indexed intersection of a constant class, i.e. where 𝐵 does not depend on 𝑥. (Contributed by Mario Carneiro, 6-Feb-2015.) |
⊢ (𝐴 ≠ ∅ → ∩ 𝑥 ∈ 𝐴 𝐵 = 𝐵) | ||
Theorem | iuniin 4531* | 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 4532* | Subclass theorem for indexed union. (Contributed by NM, 10-Dec-2004.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (𝐴 ⊆ 𝐵 → ∪ 𝑥 ∈ 𝐴 𝐶 ⊆ ∪ 𝑥 ∈ 𝐵 𝐶) | ||
Theorem | iinss1 4533* | Subclass theorem for indexed intersection. (Contributed by NM, 24-Jan-2012.) |
⊢ (𝐴 ⊆ 𝐵 → ∩ 𝑥 ∈ 𝐵 𝐶 ⊆ ∩ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iuneq1 4534* | Equality theorem for indexed union. (Contributed by NM, 27-Jun-1998.) |
⊢ (𝐴 = 𝐵 → ∪ 𝑥 ∈ 𝐴 𝐶 = ∪ 𝑥 ∈ 𝐵 𝐶) | ||
Theorem | iineq1 4535* | Equality theorem for indexed intersection. (Contributed by NM, 27-Jun-1998.) |
⊢ (𝐴 = 𝐵 → ∩ 𝑥 ∈ 𝐴 𝐶 = ∩ 𝑥 ∈ 𝐵 𝐶) | ||
Theorem | ss2iun 4536 | Subclass theorem for indexed union. (Contributed by NM, 26-Nov-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (∀𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶 → ∪ 𝑥 ∈ 𝐴 𝐵 ⊆ ∪ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iuneq2 4537 | Equality theorem for indexed union. (Contributed by NM, 22-Oct-2003.) |
⊢ (∀𝑥 ∈ 𝐴 𝐵 = 𝐶 → ∪ 𝑥 ∈ 𝐴 𝐵 = ∪ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iineq2 4538 | Equality theorem for indexed intersection. (Contributed by NM, 22-Oct-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (∀𝑥 ∈ 𝐴 𝐵 = 𝐶 → ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iuneq2i 4539 | Equality inference for indexed union. (Contributed by NM, 22-Oct-2003.) |
⊢ (𝑥 ∈ 𝐴 → 𝐵 = 𝐶) ⇒ ⊢ ∪ 𝑥 ∈ 𝐴 𝐵 = ∪ 𝑥 ∈ 𝐴 𝐶 | ||
Theorem | iineq2i 4540 | Equality inference for indexed intersection. (Contributed by NM, 22-Oct-2003.) |
⊢ (𝑥 ∈ 𝐴 → 𝐵 = 𝐶) ⇒ ⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ 𝑥 ∈ 𝐴 𝐶 | ||
Theorem | iineq2d 4541 | Equality deduction for indexed intersection. (Contributed by NM, 7-Dec-2011.) |
⊢ Ⅎ𝑥𝜑 & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iuneq2dv 4542* | Equality deduction for indexed union. (Contributed by NM, 3-Aug-2004.) |
⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → ∪ 𝑥 ∈ 𝐴 𝐵 = ∪ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iineq2dv 4543* | Equality deduction for indexed intersection. (Contributed by NM, 3-Aug-2004.) |
⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iuneq12df 4544 | Equality deduction for indexed union, deduction version. (Contributed by Thierry Arnoux, 31-Dec-2016.) |
⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐵 & ⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → ∪ 𝑥 ∈ 𝐴 𝐶 = ∪ 𝑥 ∈ 𝐵 𝐷) | ||
Theorem | iuneq1d 4545* | Equality theorem for indexed union, deduction version. (Contributed by Drahflow, 22-Oct-2015.) |
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → ∪ 𝑥 ∈ 𝐴 𝐶 = ∪ 𝑥 ∈ 𝐵 𝐶) | ||
Theorem | iuneq12d 4546* | Equality deduction for indexed union, deduction version. (Contributed by Drahflow, 22-Oct-2015.) |
⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → ∪ 𝑥 ∈ 𝐴 𝐶 = ∪ 𝑥 ∈ 𝐵 𝐷) | ||
Theorem | iuneq2d 4547* | Equality deduction for indexed union. (Contributed by Drahflow, 22-Oct-2015.) |
⊢ (𝜑 → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → ∪ 𝑥 ∈ 𝐴 𝐵 = ∪ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | nfiun 4548 | Bound-variable hypothesis builder for indexed union. (Contributed by Mario Carneiro, 25-Jan-2014.) |
⊢ Ⅎ𝑦𝐴 & ⊢ Ⅎ𝑦𝐵 ⇒ ⊢ Ⅎ𝑦∪ 𝑥 ∈ 𝐴 𝐵 | ||
Theorem | nfiin 4549 | Bound-variable hypothesis builder for indexed intersection. (Contributed by Mario Carneiro, 25-Jan-2014.) |
⊢ Ⅎ𝑦𝐴 & ⊢ Ⅎ𝑦𝐵 ⇒ ⊢ Ⅎ𝑦∩ 𝑥 ∈ 𝐴 𝐵 | ||
Theorem | nfiu1 4550 | Bound-variable hypothesis builder for indexed union. (Contributed by NM, 12-Oct-2003.) |
⊢ Ⅎ𝑥∪ 𝑥 ∈ 𝐴 𝐵 | ||
Theorem | nfii1 4551 | Bound-variable hypothesis builder for indexed intersection. (Contributed by NM, 15-Oct-2003.) |
⊢ Ⅎ𝑥∩ 𝑥 ∈ 𝐴 𝐵 | ||
Theorem | dfiun2g 4552* | 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 4553* | Alternate definition of indexed intersection when 𝐵 is a set. (Contributed by Jeff Hankins, 27-Aug-2009.) |
⊢ (∀𝑥 ∈ 𝐴 𝐵 ∈ 𝐶 → ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵}) | ||
Theorem | dfiun2 4554* | 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 4555* | 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 4556* | Define double indexed union. (Contributed by FL, 6-Nov-2013.) |
⊢ ∪ 𝑥 ∈ 𝐴 ∪ 𝑦 ∈ 𝐵 𝐶 = {𝑧 ∣ ∃𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝑧 ∈ 𝐶} | ||
Theorem | cbviun 4557* | 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 4558* | Change bound variables in an indexed intersection. (Contributed by Jeff Hankins, 26-Aug-2009.) (Revised by Mario Carneiro, 14-Oct-2016.) |
⊢ Ⅎ𝑦𝐵 & ⊢ Ⅎ𝑥𝐶 & ⊢ (𝑥 = 𝑦 → 𝐵 = 𝐶) ⇒ ⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ 𝑦 ∈ 𝐴 𝐶 | ||
Theorem | cbviunv 4559* | 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 4560* | Change bound variables in an indexed intersection. (Contributed by Jeff Hankins, 26-Aug-2009.) |
⊢ (𝑥 = 𝑦 → 𝐵 = 𝐶) ⇒ ⊢ ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ 𝑦 ∈ 𝐴 𝐶 | ||
Theorem | iunss 4561* | Subset theorem for an indexed union. (Contributed by NM, 13-Sep-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (∪ 𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶 ↔ ∀𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶) | ||
Theorem | ssiun 4562* | Subset implication for an indexed union. (Contributed by NM, 3-Sep-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (∃𝑥 ∈ 𝐴 𝐶 ⊆ 𝐵 → 𝐶 ⊆ ∪ 𝑥 ∈ 𝐴 𝐵) | ||
Theorem | ssiun2 4563 | Identity law for subset of an indexed union. (Contributed by NM, 12-Oct-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (𝑥 ∈ 𝐴 → 𝐵 ⊆ ∪ 𝑥 ∈ 𝐴 𝐵) | ||
Theorem | ssiun2s 4564* | Subset relationship for an indexed union. (Contributed by NM, 26-Oct-2003.) |
⊢ (𝑥 = 𝐶 → 𝐵 = 𝐷) ⇒ ⊢ (𝐶 ∈ 𝐴 → 𝐷 ⊆ ∪ 𝑥 ∈ 𝐴 𝐵) | ||
Theorem | iunss2 4565* | 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 4470. (Contributed by NM, 9-Dec-2004.) |
⊢ (∀𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝐶 ⊆ 𝐷 → ∪ 𝑥 ∈ 𝐴 𝐶 ⊆ ∪ 𝑦 ∈ 𝐵 𝐷) | ||
Theorem | iunab 4566* | The indexed union of a class abstraction. (Contributed by NM, 27-Dec-2004.) |
⊢ ∪ 𝑥 ∈ 𝐴 {𝑦 ∣ 𝜑} = {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝜑} | ||
Theorem | iunrab 4567* | The indexed union of a restricted class abstraction. (Contributed by NM, 3-Jan-2004.) (Proof shortened by Mario Carneiro, 14-Nov-2016.) |
⊢ ∪ 𝑥 ∈ 𝐴 {𝑦 ∈ 𝐵 ∣ 𝜑} = {𝑦 ∈ 𝐵 ∣ ∃𝑥 ∈ 𝐴 𝜑} | ||
Theorem | iunxdif2 4568* | Indexed union with a class difference as its index. (Contributed by NM, 10-Dec-2004.) |
⊢ (𝑥 = 𝑦 → 𝐶 = 𝐷) ⇒ ⊢ (∀𝑥 ∈ 𝐴 ∃𝑦 ∈ (𝐴 ∖ 𝐵)𝐶 ⊆ 𝐷 → ∪ 𝑦 ∈ (𝐴 ∖ 𝐵)𝐷 = ∪ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | ssiinf 4569 | Subset theorem for an indexed intersection. (Contributed by FL, 15-Oct-2012.) (Proof shortened by Mario Carneiro, 14-Oct-2016.) |
⊢ Ⅎ𝑥𝐶 ⇒ ⊢ (𝐶 ⊆ ∩ 𝑥 ∈ 𝐴 𝐵 ↔ ∀𝑥 ∈ 𝐴 𝐶 ⊆ 𝐵) | ||
Theorem | ssiin 4570* | Subset theorem for an indexed intersection. (Contributed by NM, 15-Oct-2003.) |
⊢ (𝐶 ⊆ ∩ 𝑥 ∈ 𝐴 𝐵 ↔ ∀𝑥 ∈ 𝐴 𝐶 ⊆ 𝐵) | ||
Theorem | iinss 4571* | Subset implication for an indexed intersection. (Contributed by NM, 15-Oct-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (∃𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶 → ∩ 𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶) | ||
Theorem | iinss2 4572 | An indexed intersection is included in any of its members. (Contributed by FL, 15-Oct-2012.) |
⊢ (𝑥 ∈ 𝐴 → ∩ 𝑥 ∈ 𝐴 𝐵 ⊆ 𝐵) | ||
Theorem | uniiun 4573* | Class union in terms of indexed union. Definition in [Stoll] p. 43. (Contributed by NM, 28-Jun-1998.) |
⊢ ∪ 𝐴 = ∪ 𝑥 ∈ 𝐴 𝑥 | ||
Theorem | intiin 4574* | Class intersection in terms of indexed intersection. Definition in [Stoll] p. 44. (Contributed by NM, 28-Jun-1998.) |
⊢ ∩ 𝐴 = ∩ 𝑥 ∈ 𝐴 𝑥 | ||
Theorem | iunid 4575* | An indexed union of singletons recovers the index set. (Contributed by NM, 6-Sep-2005.) |
⊢ ∪ 𝑥 ∈ 𝐴 {𝑥} = 𝐴 | ||
Theorem | iun0 4576 | An indexed union of the empty set is empty. (Contributed by NM, 26-Mar-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ ∪ 𝑥 ∈ 𝐴 ∅ = ∅ | ||
Theorem | 0iun 4577 | An empty indexed union is empty. (Contributed by NM, 4-Dec-2004.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ ∪ 𝑥 ∈ ∅ 𝐴 = ∅ | ||
Theorem | 0iin 4578 | An empty indexed intersection is the universal class. (Contributed by NM, 20-Oct-2005.) |
⊢ ∩ 𝑥 ∈ ∅ 𝐴 = V | ||
Theorem | viin 4579* | Indexed intersection with a universal index class. When 𝐴 doesn't depend on 𝑥, this evaluates to 𝐴 by 19.3 2069 and abid2 2745. When 𝐴 = 𝑥, this evaluates to ∅ by intiin 4574 and intv 4841. (Contributed by NM, 11-Sep-2008.) |
⊢ ∩ 𝑥 ∈ V 𝐴 = {𝑦 ∣ ∀𝑥 𝑦 ∈ 𝐴} | ||
Theorem | iunn0 4580* | There is a nonempty class in an indexed collection 𝐵(𝑥) iff the indexed union of them is nonempty. (Contributed by NM, 15-Oct-2003.) (Proof shortened by Andrew Salmon, 25-Jul-2011.) |
⊢ (∃𝑥 ∈ 𝐴 𝐵 ≠ ∅ ↔ ∪ 𝑥 ∈ 𝐴 𝐵 ≠ ∅) | ||
Theorem | iinab 4581* | Indexed intersection of a class builder. (Contributed by NM, 6-Dec-2011.) |
⊢ ∩ 𝑥 ∈ 𝐴 {𝑦 ∣ 𝜑} = {𝑦 ∣ ∀𝑥 ∈ 𝐴 𝜑} | ||
Theorem | iinrab 4582* | Indexed intersection of a restricted class builder. (Contributed by NM, 6-Dec-2011.) |
⊢ (𝐴 ≠ ∅ → ∩ 𝑥 ∈ 𝐴 {𝑦 ∈ 𝐵 ∣ 𝜑} = {𝑦 ∈ 𝐵 ∣ ∀𝑥 ∈ 𝐴 𝜑}) | ||
Theorem | iinrab2 4583* | Indexed intersection of a restricted class builder. (Contributed by NM, 6-Dec-2011.) |
⊢ (∩ 𝑥 ∈ 𝐴 {𝑦 ∈ 𝐵 ∣ 𝜑} ∩ 𝐵) = {𝑦 ∈ 𝐵 ∣ ∀𝑥 ∈ 𝐴 𝜑} | ||
Theorem | iunin2 4584* | Indexed union of intersection. Generalization of half of theorem "Distributive laws" in [Enderton] p. 30. Use uniiun 4573 to recover Enderton's theorem. (Contributed by NM, 26-Mar-2004.) |
⊢ ∪ 𝑥 ∈ 𝐴 (𝐵 ∩ 𝐶) = (𝐵 ∩ ∪ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iunin1 4585* | Indexed union of intersection. Generalization of half of theorem "Distributive laws" in [Enderton] p. 30. Use uniiun 4573 to recover Enderton's theorem. (Contributed by Mario Carneiro, 30-Aug-2015.) |
⊢ ∪ 𝑥 ∈ 𝐴 (𝐶 ∩ 𝐵) = (∪ 𝑥 ∈ 𝐴 𝐶 ∩ 𝐵) | ||
Theorem | iinun2 4586* | Indexed intersection of union. Generalization of half of theorem "Distributive laws" in [Enderton] p. 30. Use intiin 4574 to recover Enderton's theorem. (Contributed by NM, 19-Aug-2004.) |
⊢ ∩ 𝑥 ∈ 𝐴 (𝐵 ∪ 𝐶) = (𝐵 ∪ ∩ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | iundif2 4587* | Indexed union of class difference. Generalization of half of theorem "De Morgan's laws" in [Enderton] p. 31. Use intiin 4574 to recover Enderton's theorem. (Contributed by NM, 19-Aug-2004.) |
⊢ ∪ 𝑥 ∈ 𝐴 (𝐵 ∖ 𝐶) = (𝐵 ∖ ∩ 𝑥 ∈ 𝐴 𝐶) | ||
Theorem | 2iunin 4588* | Rearrange indexed unions over intersection. (Contributed by NM, 18-Dec-2008.) |
⊢ ∪ 𝑥 ∈ 𝐴 ∪ 𝑦 ∈ 𝐵 (𝐶 ∩ 𝐷) = (∪ 𝑥 ∈ 𝐴 𝐶 ∩ ∪ 𝑦 ∈ 𝐵 𝐷) | ||
Theorem | iindif2 4589* | Indexed intersection of class difference. Generalization of half of theorem "De Morgan's laws" in [Enderton] p. 31. Use uniiun 4573 to recover Enderton's theorem. (Contributed by NM, 5-Oct-2006.) |
⊢ (𝐴 ≠ ∅ → ∩ 𝑥 ∈ 𝐴 (𝐵 ∖ 𝐶) = (𝐵 ∖ ∪ 𝑥 ∈ 𝐴 𝐶)) | ||
Theorem | iinin2 4590* | Indexed intersection of intersection. Generalization of half of theorem "Distributive laws" in [Enderton] p. 30. Use intiin 4574 to recover Enderton's theorem. (Contributed by Mario Carneiro, 19-Mar-2015.) |
⊢ (𝐴 ≠ ∅ → ∩ 𝑥 ∈ 𝐴 (𝐵 ∩ 𝐶) = (𝐵 ∩ ∩ 𝑥 ∈ 𝐴 𝐶)) | ||
Theorem | iinin1 4591* | Indexed intersection of intersection. Generalization of half of theorem "Distributive laws" in [Enderton] p. 30. Use intiin 4574 to recover Enderton's theorem. (Contributed by Mario Carneiro, 19-Mar-2015.) |
⊢ (𝐴 ≠ ∅ → ∩ 𝑥 ∈ 𝐴 (𝐶 ∩ 𝐵) = (∩ 𝑥 ∈ 𝐴 𝐶 ∩ 𝐵)) | ||
Theorem | iinvdif 4592* | The indexed intersection of a complement. (Contributed by Gérard Lang, 5-Aug-2018.) |
⊢ ∩ 𝑥 ∈ 𝐴 (V ∖ 𝐵) = (V ∖ ∪ 𝑥 ∈ 𝐴 𝐵) | ||
Theorem | elriin 4593* | Elementhood in a relative intersection. (Contributed by Mario Carneiro, 30-Dec-2016.) |
⊢ (𝐵 ∈ (𝐴 ∩ ∩ 𝑥 ∈ 𝑋 𝑆) ↔ (𝐵 ∈ 𝐴 ∧ ∀𝑥 ∈ 𝑋 𝐵 ∈ 𝑆)) | ||
Theorem | riin0 4594* | Relative intersection of an empty family. (Contributed by Stefan O'Rear, 3-Apr-2015.) |
⊢ (𝑋 = ∅ → (𝐴 ∩ ∩ 𝑥 ∈ 𝑋 𝑆) = 𝐴) | ||
Theorem | riinn0 4595* | Relative intersection of a nonempty family. (Contributed by Stefan O'Rear, 3-Apr-2015.) |
⊢ ((∀𝑥 ∈ 𝑋 𝑆 ⊆ 𝐴 ∧ 𝑋 ≠ ∅) → (𝐴 ∩ ∩ 𝑥 ∈ 𝑋 𝑆) = ∩ 𝑥 ∈ 𝑋 𝑆) | ||
Theorem | riinrab 4596* | Relative intersection of a relative abstraction. (Contributed by Stefan O'Rear, 3-Apr-2015.) |
⊢ (𝐴 ∩ ∩ 𝑥 ∈ 𝑋 {𝑦 ∈ 𝐴 ∣ 𝜑}) = {𝑦 ∈ 𝐴 ∣ ∀𝑥 ∈ 𝑋 𝜑} | ||
Theorem | symdif0 4597 | Symmetric difference with the empty class. (Contributed by Scott Fenton, 24-Apr-2012.) |
⊢ (𝐴 △ ∅) = 𝐴 | ||
Theorem | symdifv 4598 | Symmetric difference with the universal class. (Contributed by Scott Fenton, 24-Apr-2012.) |
⊢ (𝐴 △ V) = (V ∖ 𝐴) | ||
Theorem | symdifid 4599 | Symmetric difference with self yields the empty class. (Contributed by Scott Fenton, 25-Apr-2012.) |
⊢ (𝐴 △ 𝐴) = ∅ | ||
Theorem | iinxsng 4600* | A singleton index picks out an instance of an indexed intersection's argument. (Contributed by NM, 15-Jan-2012.) (Proof shortened by Mario Carneiro, 17-Nov-2016.) |
⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶) ⇒ ⊢ (𝐴 ∈ 𝑉 → ∩ 𝑥 ∈ {𝐴}𝐵 = 𝐶) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |