| Metamath
Proof Explorer Theorem List (p. 325 of 497) | < 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-30845) |
(30846-32368) |
(32369-49617) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | eqtrb 32401 | A transposition of equality. (Contributed by Thierry Arnoux, 20-Aug-2023.) |
| ⊢ ((𝐴 = 𝐵 ∧ 𝐴 = 𝐶) ↔ (𝐴 = 𝐵 ∧ 𝐵 = 𝐶)) | ||
| Theorem | eqelbid 32402* | A variable elimination law for equality within a given set 𝐴. See equvel 2460. (Contributed by Thierry Arnoux, 20-Feb-2025.) |
| ⊢ (𝜑 → 𝐵 ∈ 𝐴) & ⊢ (𝜑 → 𝐶 ∈ 𝐴) ⇒ ⊢ (𝜑 → (∀𝑥 ∈ 𝐴 (𝑥 = 𝐵 ↔ 𝑥 = 𝐶) ↔ 𝐵 = 𝐶)) | ||
| Theorem | opsbc2ie 32403* | Conversion of implicit substitution to explicit class substitution for ordered pairs. (Contributed by Thierry Arnoux, 4-Jul-2023.) |
| ⊢ (𝑝 = 〈𝑎, 𝑏〉 → (𝜑 ↔ 𝜒)) ⇒ ⊢ (𝑝 = 〈𝑥, 𝑦〉 → (𝜑 ↔ [𝑦 / 𝑏][𝑥 / 𝑎]𝜒)) | ||
| Theorem | opreu2reuALT 32404* | Correspondence between uniqueness of ordered pairs and double restricted existential uniqueness quantification. Alternate proof of one direction only, use opreu2reurex 6283 instead. (Contributed by Thierry Arnoux, 4-Jul-2023.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ (𝑝 = 〈𝑎, 𝑏〉 → (𝜑 ↔ 𝜒)) ⇒ ⊢ ((∃!𝑎 ∈ 𝐴 ∃𝑏 ∈ 𝐵 𝜒 ∧ ∃!𝑏 ∈ 𝐵 ∃𝑎 ∈ 𝐴 𝜒) → ∃!𝑝 ∈ (𝐴 × 𝐵)𝜑) | ||
| Syntax | w2reu 32405 | Syntax for double restricted existential uniqueness quantification. |
| wff ∃!𝑥 ∈ 𝐴 , 𝑦 ∈ 𝐵𝜑 | ||
| Definition | df-2reu 32406 | Define the double restricted existential uniqueness quantifier. (Contributed by Thierry Arnoux, 4-Jul-2023.) |
| ⊢ (∃!𝑥 ∈ 𝐴 , 𝑦 ∈ 𝐵𝜑 ↔ (∃!𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝜑 ∧ ∃!𝑦 ∈ 𝐵 ∃𝑥 ∈ 𝐴 𝜑)) | ||
| Theorem | 2reucom 32407 | Double restricted existential uniqueness commutes. (Contributed by Thierry Arnoux, 4-Jul-2023.) |
| ⊢ (∃!𝑥 ∈ 𝐴 , 𝑦 ∈ 𝐵𝜑 ↔ ∃!𝑦 ∈ 𝐵 , 𝑥 ∈ 𝐴𝜑) | ||
| Theorem | 2reu2rex1 32408 | Double restricted existential uniqueness implies double restricted existence. (Contributed by Thierry Arnoux, 4-Jul-2023.) |
| ⊢ (∃!𝑥 ∈ 𝐴 , 𝑦 ∈ 𝐵𝜑 → ∃𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝜑) | ||
| Theorem | 2reureurex 32409 | Double restricted existential uniqueness implies restricted existential uniqueness with restricted existence. (Contributed by AV, 5-Jul-2023.) |
| ⊢ (∃!𝑥 ∈ 𝐴 , 𝑦 ∈ 𝐵𝜑 → ∃!𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝜑) | ||
| Theorem | 2reu2reu2 32410* | Double restricted existential uniqueness implies two nested restricted existential uniqueness. (Contributed by AV, 5-Jul-2023.) |
| ⊢ (∃!𝑥 ∈ 𝐴 , 𝑦 ∈ 𝐵𝜑 → ∃!𝑥 ∈ 𝐴 ∃!𝑦 ∈ 𝐵 𝜑) | ||
| Theorem | opreu2reu1 32411* | Equivalent definition of the double restricted existential uniqueness quantifier, using uniqueness of ordered pairs. (Contributed by Thierry Arnoux, 4-Jul-2023.) |
| ⊢ (𝑝 = 〈𝑥, 𝑦〉 → (𝜒 ↔ 𝜑)) ⇒ ⊢ (∃!𝑥 ∈ 𝐴 , 𝑦 ∈ 𝐵𝜑 ↔ ∃!𝑝 ∈ (𝐴 × 𝐵)𝜒) | ||
| Theorem | sq2reunnltb 32412* | There exists a unique decomposition of a prime as a sum of squares of two different positive integers iff the prime is of the form 4𝑘 + 1. Double restricted existential uniqueness variant of 2sqreunnltb 27422. (Contributed by AV, 5-Jul-2023.) |
| ⊢ (𝑃 ∈ ℙ → ((𝑃 mod 4) = 1 ↔ ∃!𝑎 ∈ ℕ , 𝑏 ∈ ℕ(𝑎 < 𝑏 ∧ ((𝑎↑2) + (𝑏↑2)) = 𝑃))) | ||
| Theorem | addsqnot2reu 32413* | For each complex number 𝐶, there does not uniquely exist two complex numbers 𝑎 and 𝑏, with 𝑏 squared and added to 𝑎 resulting in the given complex number 𝐶. Double restricted existential uniqueness variant of addsqn2reurex2 27406. (Contributed by AV, 5-Jul-2023.) |
| ⊢ (𝐶 ∈ ℂ → ¬ ∃!𝑎 ∈ ℂ , 𝑏 ∈ ℂ(𝑎 + (𝑏↑2)) = 𝐶) | ||
| Theorem | sbceqbidf 32414 | Equality theorem for class substitution. (Contributed by Thierry Arnoux, 4-Sep-2018.) |
| ⊢ Ⅎ𝑥𝜑 & ⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → ([𝐴 / 𝑥]𝜓 ↔ [𝐵 / 𝑥]𝜒)) | ||
| Theorem | sbcies 32415* | A special version of class substitution commonly used for structures. (Contributed by Thierry Arnoux, 14-Mar-2019.) |
| ⊢ 𝐴 = (𝐸‘𝑊) & ⊢ (𝑎 = 𝐴 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (𝑤 = 𝑊 → ([(𝐸‘𝑤) / 𝑎]𝜓 ↔ 𝜑)) | ||
| Theorem | mo5f 32416* | Alternate definition of "at most one." (Contributed by Thierry Arnoux, 1-Mar-2017.) |
| ⊢ Ⅎ𝑖𝜑 & ⊢ Ⅎ𝑗𝜑 ⇒ ⊢ (∃*𝑥𝜑 ↔ ∀𝑖∀𝑗(([𝑖 / 𝑥]𝜑 ∧ [𝑗 / 𝑥]𝜑) → 𝑖 = 𝑗)) | ||
| Theorem | nmo 32417* | Negation of "at most one". (Contributed by Thierry Arnoux, 26-Feb-2017.) |
| ⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (¬ ∃*𝑥𝜑 ↔ ∀𝑦∃𝑥(𝜑 ∧ 𝑥 ≠ 𝑦)) | ||
| Theorem | reuxfrdf 32418* | Transfer existential uniqueness from a variable 𝑥 to another variable 𝑦 contained in expression 𝐴. Cf. reuxfrd 3731 (Contributed by Thierry Arnoux, 7-Apr-2017.) (Revised by Thierry Arnoux, 8-Oct-2017.) (Revised by Thierry Arnoux, 30-Mar-2018.) |
| ⊢ Ⅎ𝑦𝐵 & ⊢ ((𝜑 ∧ 𝑦 ∈ 𝐶) → 𝐴 ∈ 𝐵) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐵) → ∃*𝑦 ∈ 𝐶 𝑥 = 𝐴) ⇒ ⊢ (𝜑 → (∃!𝑥 ∈ 𝐵 ∃𝑦 ∈ 𝐶 (𝑥 = 𝐴 ∧ 𝜓) ↔ ∃!𝑦 ∈ 𝐶 𝜓)) | ||
| Theorem | rexunirn 32419* | Restricted existential quantification over the union of the range of a function. Cf. rexrn 7076 and eluni2 4887. (Contributed by Thierry Arnoux, 19-Sep-2017.) |
| ⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵) & ⊢ (𝑥 ∈ 𝐴 → 𝐵 ∈ 𝑉) ⇒ ⊢ (∃𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝜑 → ∃𝑦 ∈ ∪ ran 𝐹𝜑) | ||
| Theorem | rmoxfrd 32420* | Transfer "at most one" restricted quantification from a variable 𝑥 to another variable 𝑦 contained in expression 𝐴. (Contributed by Thierry Arnoux, 7-Apr-2017.) (Revised by Thierry Arnoux, 8-Oct-2017.) |
| ⊢ ((𝜑 ∧ 𝑦 ∈ 𝐶) → 𝐴 ∈ 𝐵) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐵) → ∃!𝑦 ∈ 𝐶 𝑥 = 𝐴) & ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃*𝑥 ∈ 𝐵 𝜓 ↔ ∃*𝑦 ∈ 𝐶 𝜒)) | ||
| Theorem | rmoun 32421 | "At most one" restricted existential quantifier for a union implies the same quantifier on both sets. (Contributed by Thierry Arnoux, 27-Nov-2023.) |
| ⊢ (∃*𝑥 ∈ (𝐴 ∪ 𝐵)𝜑 → (∃*𝑥 ∈ 𝐴 𝜑 ∧ ∃*𝑥 ∈ 𝐵 𝜑)) | ||
| Theorem | rmounid 32422* | A case where an "at most one" restricted existential quantifier for a union is equivalent to such a quantifier for one of the sets. (Contributed by Thierry Arnoux, 27-Nov-2023.) |
| ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐵) → ¬ 𝜓) ⇒ ⊢ (𝜑 → (∃*𝑥 ∈ (𝐴 ∪ 𝐵)𝜓 ↔ ∃*𝑥 ∈ 𝐴 𝜓)) | ||
| Theorem | riotaeqbidva 32423* | Equivalent wff's yield equal restricted definition binders (deduction form). (raleqbidva 3311 analog.) (Contributed by Thierry Arnoux, 29-Jan-2025.) |
| ⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (℩𝑥 ∈ 𝐴 𝜓) = (℩𝑥 ∈ 𝐵 𝜒)) | ||
| Theorem | dmrab 32424* | Domain of a restricted class abstraction over a cartesian product. (Contributed by Thierry Arnoux, 3-Jul-2023.) |
| ⊢ (𝑧 = 〈𝑥, 𝑦〉 → (𝜑 ↔ 𝜓)) ⇒ ⊢ dom {𝑧 ∈ (𝐴 × 𝐵) ∣ 𝜑} = {𝑥 ∈ 𝐴 ∣ ∃𝑦 ∈ 𝐵 𝜓} | ||
| Theorem | difrab2 32425 | Difference of two restricted class abstractions. Compare with difrab 4293. (Contributed by Thierry Arnoux, 3-Jan-2022.) |
| ⊢ ({𝑥 ∈ 𝐴 ∣ 𝜑} ∖ {𝑥 ∈ 𝐵 ∣ 𝜑}) = {𝑥 ∈ (𝐴 ∖ 𝐵) ∣ 𝜑} | ||
| Theorem | rabexgfGS 32426 | Separation Scheme in terms of a restricted class abstraction. To be removed in profit of Glauco's equivalent version. (Contributed by Thierry Arnoux, 11-May-2017.) |
| ⊢ Ⅎ𝑥𝐴 ⇒ ⊢ (𝐴 ∈ 𝑉 → {𝑥 ∈ 𝐴 ∣ 𝜑} ∈ V) | ||
| Theorem | rabsnel 32427* | Truth implied by equality of a restricted class abstraction and a singleton. (Contributed by Thierry Arnoux, 15-Sep-2018.) |
| ⊢ 𝐵 ∈ V ⇒ ⊢ ({𝑥 ∈ 𝐴 ∣ 𝜑} = {𝐵} → 𝐵 ∈ 𝐴) | ||
| Theorem | rabsspr 32428* | Conditions for a restricted class abstraction to be a subset of an unordered pair. (Contributed by Thierry Arnoux, 6-Jul-2025.) |
| ⊢ ({𝑥 ∈ 𝑉 ∣ 𝜑} ⊆ {𝑋, 𝑌} ↔ ∀𝑥 ∈ 𝑉 (𝜑 → (𝑥 = 𝑋 ∨ 𝑥 = 𝑌))) | ||
| Theorem | rabsstp 32429* | Conditions for a restricted class abstraction to be a subset of an unordered triple. (Contributed by Thierry Arnoux, 6-Jul-2025.) |
| ⊢ ({𝑥 ∈ 𝑉 ∣ 𝜑} ⊆ {𝑋, 𝑌, 𝑍} ↔ ∀𝑥 ∈ 𝑉 (𝜑 → (𝑥 = 𝑋 ∨ 𝑥 = 𝑌 ∨ 𝑥 = 𝑍))) | ||
| Theorem | 3unrab 32430 | Union of three restricted class abstractions. (Contributed by Thierry Arnoux, 6-Jul-2025.) |
| ⊢ (({𝑥 ∈ 𝐴 ∣ 𝜑} ∪ {𝑥 ∈ 𝐴 ∣ 𝜓}) ∪ {𝑥 ∈ 𝐴 ∣ 𝜒}) = {𝑥 ∈ 𝐴 ∣ (𝜑 ∨ 𝜓 ∨ 𝜒)} | ||
| Theorem | foresf1o 32431* | From a surjective function, *choose* a subset of the domain, such that the restricted function is bijective. (Contributed by Thierry Arnoux, 27-Jan-2020.) |
| ⊢ ((𝐴 ∈ 𝑉 ∧ 𝐹:𝐴–onto→𝐵) → ∃𝑥 ∈ 𝒫 𝐴(𝐹 ↾ 𝑥):𝑥–1-1-onto→𝐵) | ||
| Theorem | rabfodom 32432* | Domination relation for restricted abstract class builders, based on a surjective function. (Contributed by Thierry Arnoux, 27-Jan-2020.) |
| ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴 ∧ 𝑦 = (𝐹‘𝑥)) → (𝜒 ↔ 𝜓)) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝐹:𝐴–onto→𝐵) ⇒ ⊢ (𝜑 → {𝑦 ∈ 𝐵 ∣ 𝜒} ≼ {𝑥 ∈ 𝐴 ∣ 𝜓}) | ||
| Theorem | rabrexfi 32433* | Conditions for a class abstraction with a restricted existential quantification to be finite. (Contributed by Thierry Arnoux, 6-Jul-2025.) |
| ⊢ (𝜑 → 𝐵 ∈ Fin) & ⊢ ((𝜑 ∧ 𝑦 ∈ 𝐵) → {𝑥 ∈ 𝐴 ∣ 𝜓} ∈ Fin) ⇒ ⊢ (𝜑 → {𝑥 ∈ 𝐴 ∣ ∃𝑦 ∈ 𝐵 𝜓} ∈ Fin) | ||
| Theorem | abrexdomjm 32434* | An indexed set is dominated by the indexing set. (Contributed by Jeff Madsen, 2-Sep-2009.) |
| ⊢ (𝑦 ∈ 𝐴 → ∃*𝑥𝜑) ⇒ ⊢ (𝐴 ∈ 𝑉 → {𝑥 ∣ ∃𝑦 ∈ 𝐴 𝜑} ≼ 𝐴) | ||
| Theorem | abrexdom2jm 32435* | An indexed set is dominated by the indexing set. (Contributed by Jeff Madsen, 2-Sep-2009.) |
| ⊢ (𝐴 ∈ 𝑉 → {𝑥 ∣ ∃𝑦 ∈ 𝐴 𝑥 = 𝐵} ≼ 𝐴) | ||
| Theorem | abrexexd 32436* | Existence of a class abstraction of existentially restricted sets. (Contributed by Thierry Arnoux, 10-May-2017.) |
| ⊢ Ⅎ𝑥𝐴 & ⊢ (𝜑 → 𝐴 ∈ V) ⇒ ⊢ (𝜑 → {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵} ∈ V) | ||
| Theorem | elabreximd 32437* | Class substitution in an image set. (Contributed by Thierry Arnoux, 30-Dec-2016.) |
| ⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑥𝜒 & ⊢ (𝐴 = 𝐵 → (𝜒 ↔ 𝜓)) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐶) → 𝜓) ⇒ ⊢ ((𝜑 ∧ 𝐴 ∈ {𝑦 ∣ ∃𝑥 ∈ 𝐶 𝑦 = 𝐵}) → 𝜒) | ||
| Theorem | elabreximdv 32438* | Class substitution in an image set. (Contributed by Thierry Arnoux, 30-Dec-2016.) |
| ⊢ (𝐴 = 𝐵 → (𝜒 ↔ 𝜓)) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐶) → 𝜓) ⇒ ⊢ ((𝜑 ∧ 𝐴 ∈ {𝑦 ∣ ∃𝑥 ∈ 𝐶 𝑦 = 𝐵}) → 𝜒) | ||
| Theorem | abrexss 32439* | A necessary condition for an image set to be a subset. (Contributed by Thierry Arnoux, 6-Feb-2017.) |
| ⊢ Ⅎ𝑥𝐶 ⇒ ⊢ (∀𝑥 ∈ 𝐴 𝐵 ∈ 𝐶 → {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵} ⊆ 𝐶) | ||
| Theorem | nelun 32440 | Negated membership for a union. (Contributed by Thierry Arnoux, 13-Dec-2023.) |
| ⊢ (𝐴 = (𝐵 ∪ 𝐶) → (¬ 𝑋 ∈ 𝐴 ↔ (¬ 𝑋 ∈ 𝐵 ∧ ¬ 𝑋 ∈ 𝐶))) | ||
| Theorem | snsssng 32441 | If a singleton is a subset of another, their members are equal. (Contributed by NM, 28-May-2006.) (Revised by Thierry Arnoux, 11-Apr-2024.) |
| ⊢ ((𝐴 ∈ 𝑉 ∧ {𝐴} ⊆ {𝐵}) → 𝐴 = 𝐵) | ||
| Theorem | n0nsnel 32442* | If a class with one element is not a singleton, there is at least another element in this class. (Contributed by AV, 6-Mar-2025.) (Revised by Thierry Arnoux, 28-May-2025.) |
| ⊢ ((𝐶 ∈ 𝐵 ∧ 𝐵 ≠ {𝐴}) → ∃𝑥 ∈ 𝐵 𝑥 ≠ 𝐴) | ||
| Theorem | inin 32443 | Intersection with an intersection. (Contributed by Thierry Arnoux, 27-Dec-2016.) |
| ⊢ (𝐴 ∩ (𝐴 ∩ 𝐵)) = (𝐴 ∩ 𝐵) | ||
| Theorem | difininv 32444 | Condition for the intersections of two sets with a given set to be equal. (Contributed by Thierry Arnoux, 28-Dec-2021.) |
| ⊢ ((((𝐴 ∖ 𝐶) ∩ 𝐵) = ∅ ∧ ((𝐶 ∖ 𝐴) ∩ 𝐵) = ∅) → (𝐴 ∩ 𝐵) = (𝐶 ∩ 𝐵)) | ||
| Theorem | difeq 32445 | Rewriting an equation with class difference, without using quantifiers. (Contributed by Thierry Arnoux, 24-Sep-2017.) |
| ⊢ ((𝐴 ∖ 𝐵) = 𝐶 ↔ ((𝐶 ∩ 𝐵) = ∅ ∧ (𝐶 ∪ 𝐵) = (𝐴 ∪ 𝐵))) | ||
| Theorem | eqdif 32446 | If both set differences of two sets are empty, those sets are equal. (Contributed by Thierry Arnoux, 16-Nov-2023.) |
| ⊢ (((𝐴 ∖ 𝐵) = ∅ ∧ (𝐵 ∖ 𝐴) = ∅) → 𝐴 = 𝐵) | ||
| Theorem | indifbi 32447 | Two ways to express equality relative to a class 𝐴. (Contributed by Thierry Arnoux, 23-Jun-2024.) |
| ⊢ ((𝐴 ∩ 𝐵) = (𝐴 ∩ 𝐶) ↔ (𝐴 ∖ 𝐵) = (𝐴 ∖ 𝐶)) | ||
| Theorem | diffib 32448 | Case where diffi 9187 is a biconditional. (Contributed by Thierry Arnoux, 27-Jun-2024.) |
| ⊢ (𝐵 ∈ Fin → (𝐴 ∈ Fin ↔ (𝐴 ∖ 𝐵) ∈ Fin)) | ||
| Theorem | difxp1ss 32449 | Difference law for Cartesian products. (Contributed by Thierry Arnoux, 24-Jul-2023.) |
| ⊢ ((𝐴 ∖ 𝐶) × 𝐵) ⊆ (𝐴 × 𝐵) | ||
| Theorem | difxp2ss 32450 | Difference law for Cartesian products. (Contributed by Thierry Arnoux, 24-Jul-2023.) |
| ⊢ (𝐴 × (𝐵 ∖ 𝐶)) ⊆ (𝐴 × 𝐵) | ||
| Theorem | indifundif 32451 | A remarkable equation with sets. (Contributed by Thierry Arnoux, 18-May-2020.) |
| ⊢ (((𝐴 ∩ 𝐵) ∖ 𝐶) ∪ (𝐴 ∖ 𝐵)) = (𝐴 ∖ (𝐵 ∩ 𝐶)) | ||
| Theorem | elpwincl1 32452 | Closure of intersection with regard to elementhood to a power set. (Contributed by Thierry Arnoux, 18-May-2020.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝒫 𝐶) ⇒ ⊢ (𝜑 → (𝐴 ∩ 𝐵) ∈ 𝒫 𝐶) | ||
| Theorem | elpwdifcl 32453 | Closure of class difference with regard to elementhood to a power set. (Contributed by Thierry Arnoux, 18-May-2020.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝒫 𝐶) ⇒ ⊢ (𝜑 → (𝐴 ∖ 𝐵) ∈ 𝒫 𝐶) | ||
| Theorem | elpwiuncl 32454* | Closure of indexed union with regard to elementhood to a power set. (Contributed by Thierry Arnoux, 27-May-2020.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ ((𝜑 ∧ 𝑘 ∈ 𝐴) → 𝐵 ∈ 𝒫 𝐶) ⇒ ⊢ (𝜑 → ∪ 𝑘 ∈ 𝐴 𝐵 ∈ 𝒫 𝐶) | ||
| Theorem | elpreq 32455 | Equality wihin a pair. (Contributed by Thierry Arnoux, 23-Aug-2017.) |
| ⊢ (𝜑 → 𝑋 ∈ {𝐴, 𝐵}) & ⊢ (𝜑 → 𝑌 ∈ {𝐴, 𝐵}) & ⊢ (𝜑 → (𝑋 = 𝐴 ↔ 𝑌 = 𝐴)) ⇒ ⊢ (𝜑 → 𝑋 = 𝑌) | ||
| Theorem | prssad 32456 | If a pair is a subset of a class, the first element of the pair is an element of that class. (Contributed by Thierry Arnoux, 2-Nov-2025.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → {𝐴, 𝐵} ⊆ 𝐶) ⇒ ⊢ (𝜑 → 𝐴 ∈ 𝐶) | ||
| Theorem | prssbd 32457 | If a pair is a subset of a class, the second element of the pair is an element of that class. (Contributed by Thierry Arnoux, 2-Nov-2025.) |
| ⊢ (𝜑 → 𝐵 ∈ 𝑉) & ⊢ (𝜑 → {𝐴, 𝐵} ⊆ 𝐶) ⇒ ⊢ (𝜑 → 𝐵 ∈ 𝐶) | ||
| Theorem | nelpr 32458 | A set 𝐴 not in a pair is neither element of the pair. (Contributed by Thierry Arnoux, 20-Nov-2023.) |
| ⊢ (𝐴 ∈ 𝑉 → (¬ 𝐴 ∈ {𝐵, 𝐶} ↔ (𝐴 ≠ 𝐵 ∧ 𝐴 ≠ 𝐶))) | ||
| Theorem | inpr0 32459 | Rewrite an empty intersection with a pair. (Contributed by Thierry Arnoux, 20-Nov-2023.) |
| ⊢ ((𝐴 ∩ {𝐵, 𝐶}) = ∅ ↔ (¬ 𝐵 ∈ 𝐴 ∧ ¬ 𝐶 ∈ 𝐴)) | ||
| Theorem | neldifpr1 32460 | The first element of a pair is not an element of a difference with this pair. (Contributed by Thierry Arnoux, 20-Nov-2023.) |
| ⊢ ¬ 𝐴 ∈ (𝐶 ∖ {𝐴, 𝐵}) | ||
| Theorem | neldifpr2 32461 | The second element of a pair is not an element of a difference with this pair. (Contributed by Thierry Arnoux, 20-Nov-2023.) |
| ⊢ ¬ 𝐵 ∈ (𝐶 ∖ {𝐴, 𝐵}) | ||
| Theorem | unidifsnel 32462 | The other element of a pair is an element of the pair. (Contributed by Thierry Arnoux, 26-Aug-2017.) |
| ⊢ ((𝑋 ∈ 𝑃 ∧ 𝑃 ≈ 2o) → ∪ (𝑃 ∖ {𝑋}) ∈ 𝑃) | ||
| Theorem | unidifsnne 32463 | The other element of a pair is not the known element. (Contributed by Thierry Arnoux, 26-Aug-2017.) |
| ⊢ ((𝑋 ∈ 𝑃 ∧ 𝑃 ≈ 2o) → ∪ (𝑃 ∖ {𝑋}) ≠ 𝑋) | ||
| Theorem | tpssg 32464 | An unordered triple of elements of a class is a subset of the class. (Contributed by Thierry Arnoux, 2-Nov-2025.) |
| ⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊 ∧ 𝐶 ∈ 𝑋) → ((𝐴 ∈ 𝐷 ∧ 𝐵 ∈ 𝐷 ∧ 𝐶 ∈ 𝐷) ↔ {𝐴, 𝐵, 𝐶} ⊆ 𝐷)) | ||
| Theorem | tpssd 32465 | Deduction version of tpssi : An unordered triple of elements of a class is a subset of that class. (Contributed by Thierry Arnoux, 2-Nov-2025.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝐷) & ⊢ (𝜑 → 𝐵 ∈ 𝐷) & ⊢ (𝜑 → 𝐶 ∈ 𝐷) ⇒ ⊢ (𝜑 → {𝐴, 𝐵, 𝐶} ⊆ 𝐷) | ||
| Theorem | tpssad 32466 | If an ordered triple is a subset of a class, the first element of the triple is an element of that class. (Contributed by Thierry Arnoux, 2-Nov-2025.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → {𝐴, 𝐵, 𝐶} ⊆ 𝐷) ⇒ ⊢ (𝜑 → 𝐴 ∈ 𝐷) | ||
| Theorem | tpssbd 32467 | If an ordered triple is a subset of a class, the second element of the triple is an element of that class. (Contributed by Thierry Arnoux, 2-Nov-2025.) |
| ⊢ (𝜑 → 𝐵 ∈ 𝑉) & ⊢ (𝜑 → {𝐴, 𝐵, 𝐶} ⊆ 𝐷) ⇒ ⊢ (𝜑 → 𝐵 ∈ 𝐷) | ||
| Theorem | tpsscd 32468 | If an ordered triple is a subset of a class, the third element of the triple is an element of that class. (Contributed by Thierry Arnoux, 2-Nov-2025.) |
| ⊢ (𝜑 → 𝐶 ∈ 𝑉) & ⊢ (𝜑 → {𝐴, 𝐵, 𝐶} ⊆ 𝐷) ⇒ ⊢ (𝜑 → 𝐶 ∈ 𝐷) | ||
| Theorem | ifeqeqx 32469* | An equality theorem tailored for ballotlemsf1o 34492. (Contributed by Thierry Arnoux, 14-Apr-2017.) |
| ⊢ (𝑥 = 𝑋 → 𝐴 = 𝐶) & ⊢ (𝑥 = 𝑌 → 𝐵 = 𝑎) & ⊢ (𝑥 = 𝑋 → (𝜒 ↔ 𝜃)) & ⊢ (𝑥 = 𝑌 → (𝜒 ↔ 𝜓)) & ⊢ (𝜑 → 𝑎 = 𝐶) & ⊢ ((𝜑 ∧ 𝜓) → 𝜃) & ⊢ (𝜑 → 𝑌 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝑊) ⇒ ⊢ ((𝜑 ∧ 𝑥 = if(𝜓, 𝑋, 𝑌)) → 𝑎 = if(𝜒, 𝐴, 𝐵)) | ||
| Theorem | elimifd 32470 | Elimination of a conditional operator contained in a wff 𝜒. (Contributed by Thierry Arnoux, 25-Jan-2017.) |
| ⊢ (𝜑 → (if(𝜓, 𝐴, 𝐵) = 𝐴 → (𝜒 ↔ 𝜃))) & ⊢ (𝜑 → (if(𝜓, 𝐴, 𝐵) = 𝐵 → (𝜒 ↔ 𝜏))) ⇒ ⊢ (𝜑 → (𝜒 ↔ ((𝜓 ∧ 𝜃) ∨ (¬ 𝜓 ∧ 𝜏)))) | ||
| Theorem | elim2if 32471 | Elimination of two conditional operators contained in a wff 𝜒. (Contributed by Thierry Arnoux, 25-Jan-2017.) |
| ⊢ (if(𝜑, 𝐴, if(𝜓, 𝐵, 𝐶)) = 𝐴 → (𝜒 ↔ 𝜃)) & ⊢ (if(𝜑, 𝐴, if(𝜓, 𝐵, 𝐶)) = 𝐵 → (𝜒 ↔ 𝜏)) & ⊢ (if(𝜑, 𝐴, if(𝜓, 𝐵, 𝐶)) = 𝐶 → (𝜒 ↔ 𝜂)) ⇒ ⊢ (𝜒 ↔ ((𝜑 ∧ 𝜃) ∨ (¬ 𝜑 ∧ ((𝜓 ∧ 𝜏) ∨ (¬ 𝜓 ∧ 𝜂))))) | ||
| Theorem | elim2ifim 32472 | Elimination of two conditional operators for an implication. (Contributed by Thierry Arnoux, 25-Jan-2017.) |
| ⊢ (if(𝜑, 𝐴, if(𝜓, 𝐵, 𝐶)) = 𝐴 → (𝜒 ↔ 𝜃)) & ⊢ (if(𝜑, 𝐴, if(𝜓, 𝐵, 𝐶)) = 𝐵 → (𝜒 ↔ 𝜏)) & ⊢ (if(𝜑, 𝐴, if(𝜓, 𝐵, 𝐶)) = 𝐶 → (𝜒 ↔ 𝜂)) & ⊢ (𝜑 → 𝜃) & ⊢ ((¬ 𝜑 ∧ 𝜓) → 𝜏) & ⊢ ((¬ 𝜑 ∧ ¬ 𝜓) → 𝜂) ⇒ ⊢ 𝜒 | ||
| Theorem | ifeq3da 32473 | Given an expression 𝐶 containing if(𝜓, 𝐸, 𝐹), substitute (hypotheses .1 and .2) and evaluate (hypotheses .3 and .4) it for both cases at the same time. (Contributed by Thierry Arnoux, 13-Dec-2021.) |
| ⊢ (if(𝜓, 𝐸, 𝐹) = 𝐸 → 𝐶 = 𝐺) & ⊢ (if(𝜓, 𝐸, 𝐹) = 𝐹 → 𝐶 = 𝐻) & ⊢ (𝜑 → 𝐺 = 𝐴) & ⊢ (𝜑 → 𝐻 = 𝐵) ⇒ ⊢ (𝜑 → if(𝜓, 𝐴, 𝐵) = 𝐶) | ||
| Theorem | ifnetrue 32474 | Deduce truth from a conditional operator value. (Contributed by Thierry Arnoux, 20-Feb-2025.) |
| ⊢ ((𝐴 ≠ 𝐵 ∧ if(𝜑, 𝐴, 𝐵) = 𝐴) → 𝜑) | ||
| Theorem | ifnefals 32475 | Deduce falsehood from a conditional operator value. (Contributed by Thierry Arnoux, 20-Feb-2025.) |
| ⊢ ((𝐴 ≠ 𝐵 ∧ if(𝜑, 𝐴, 𝐵) = 𝐵) → ¬ 𝜑) | ||
| Theorem | ifnebib 32476 | The converse of ifbi 4523 holds if the two values are not equal. (Contributed by Thierry Arnoux, 20-Feb-2025.) |
| ⊢ (𝐴 ≠ 𝐵 → (if(𝜑, 𝐴, 𝐵) = if(𝜓, 𝐴, 𝐵) ↔ (𝜑 ↔ 𝜓))) | ||
| Theorem | uniinn0 32477* | Sufficient and necessary condition for a union to intersect with a given set. (Contributed by Thierry Arnoux, 27-Jan-2020.) |
| ⊢ ((∪ 𝐴 ∩ 𝐵) ≠ ∅ ↔ ∃𝑥 ∈ 𝐴 (𝑥 ∩ 𝐵) ≠ ∅) | ||
| Theorem | uniin1 32478* | Union of intersection. Generalization of half of theorem "Distributive laws" in [Enderton] p. 30. (Contributed by Thierry Arnoux, 21-Jun-2020.) |
| ⊢ ∪ 𝑥 ∈ 𝐴 (𝑥 ∩ 𝐵) = (∪ 𝐴 ∩ 𝐵) | ||
| Theorem | uniin2 32479* | Union of intersection. Generalization of half of theorem "Distributive laws" in [Enderton] p. 30. (Contributed by Thierry Arnoux, 21-Jun-2020.) |
| ⊢ ∪ 𝑥 ∈ 𝐵 (𝐴 ∩ 𝑥) = (𝐴 ∩ ∪ 𝐵) | ||
| Theorem | difuncomp 32480 | Express a class difference using unions and class complements. (Contributed by Thierry Arnoux, 21-Jun-2020.) |
| ⊢ (𝐴 ⊆ 𝐶 → (𝐴 ∖ 𝐵) = (𝐶 ∖ ((𝐶 ∖ 𝐴) ∪ 𝐵))) | ||
| Theorem | elpwunicl 32481 | Closure of a set union with regard to elementhood to a power set. (Contributed by Thierry Arnoux, 21-Jun-2020.) (Proof shortened by BJ, 6-Apr-2024.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝒫 𝒫 𝐵) ⇒ ⊢ (𝜑 → ∪ 𝐴 ∈ 𝒫 𝐵) | ||
| Theorem | cbviunf 32482* | 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 | iuneq12daf 32483 | Equality deduction for indexed union, deduction version. (Contributed by Thierry Arnoux, 13-Mar-2017.) |
| ⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐵 & ⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → ∪ 𝑥 ∈ 𝐴 𝐶 = ∪ 𝑥 ∈ 𝐵 𝐷) | ||
| Theorem | iunin1f 32484 | Indexed union of intersection. Generalization of half of theorem "Distributive laws" in [Enderton] p. 30. Use uniiun 5034 to recover Enderton's theorem. (Contributed by NM, 26-Mar-2004.) (Revised by Thierry Arnoux, 2-May-2020.) |
| ⊢ Ⅎ𝑥𝐶 ⇒ ⊢ ∪ 𝑥 ∈ 𝐴 (𝐵 ∩ 𝐶) = (∪ 𝑥 ∈ 𝐴 𝐵 ∩ 𝐶) | ||
| Theorem | ssiun3 32485* | Subset equivalence for an indexed union. (Contributed by Thierry Arnoux, 17-Oct-2016.) |
| ⊢ (∀𝑦 ∈ 𝐶 ∃𝑥 ∈ 𝐴 𝑦 ∈ 𝐵 ↔ 𝐶 ⊆ ∪ 𝑥 ∈ 𝐴 𝐵) | ||
| Theorem | ssiun2sf 32486 | Subset relationship for an indexed union. (Contributed by Thierry Arnoux, 31-Dec-2016.) |
| ⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐶 & ⊢ Ⅎ𝑥𝐷 & ⊢ (𝑥 = 𝐶 → 𝐵 = 𝐷) ⇒ ⊢ (𝐶 ∈ 𝐴 → 𝐷 ⊆ ∪ 𝑥 ∈ 𝐴 𝐵) | ||
| Theorem | iuninc 32487* | The union of an increasing collection of sets is its last element. (Contributed by Thierry Arnoux, 22-Jan-2017.) |
| ⊢ (𝜑 → 𝐹 Fn ℕ) & ⊢ ((𝜑 ∧ 𝑛 ∈ ℕ) → (𝐹‘𝑛) ⊆ (𝐹‘(𝑛 + 1))) ⇒ ⊢ ((𝜑 ∧ 𝑖 ∈ ℕ) → ∪ 𝑛 ∈ (1...𝑖)(𝐹‘𝑛) = (𝐹‘𝑖)) | ||
| Theorem | iundifdifd 32488* | The intersection of a set is the complement of the union of the complements. (Contributed by Thierry Arnoux, 19-Dec-2016.) |
| ⊢ (𝐴 ⊆ 𝒫 𝑂 → (𝐴 ≠ ∅ → ∩ 𝐴 = (𝑂 ∖ ∪ 𝑥 ∈ 𝐴 (𝑂 ∖ 𝑥)))) | ||
| Theorem | iundifdif 32489* | The intersection of a set is the complement of the union of the complements. TODO: shorten using iundifdifd 32488. (Contributed by Thierry Arnoux, 4-Sep-2016.) |
| ⊢ 𝑂 ∈ V & ⊢ 𝐴 ⊆ 𝒫 𝑂 ⇒ ⊢ (𝐴 ≠ ∅ → ∩ 𝐴 = (𝑂 ∖ ∪ 𝑥 ∈ 𝐴 (𝑂 ∖ 𝑥))) | ||
| Theorem | iunrdx 32490* | Re-index an indexed union. (Contributed by Thierry Arnoux, 6-Apr-2017.) |
| ⊢ (𝜑 → 𝐹:𝐴–onto→𝐶) & ⊢ ((𝜑 ∧ 𝑦 = (𝐹‘𝑥)) → 𝐷 = 𝐵) ⇒ ⊢ (𝜑 → ∪ 𝑥 ∈ 𝐴 𝐵 = ∪ 𝑦 ∈ 𝐶 𝐷) | ||
| Theorem | iunpreima 32491* | Preimage of an indexed union. (Contributed by Thierry Arnoux, 27-Mar-2018.) |
| ⊢ (Fun 𝐹 → (◡𝐹 “ ∪ 𝑥 ∈ 𝐴 𝐵) = ∪ 𝑥 ∈ 𝐴 (◡𝐹 “ 𝐵)) | ||
| Theorem | iunrnmptss 32492* | A subset relation for an indexed union over the range of function expressed as a mapping. (Contributed by Thierry Arnoux, 27-Mar-2018.) |
| ⊢ (𝑦 = 𝐵 → 𝐶 = 𝐷) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 ∈ 𝑉) ⇒ ⊢ (𝜑 → ∪ 𝑦 ∈ ran (𝑥 ∈ 𝐴 ↦ 𝐵)𝐶 ⊆ ∪ 𝑥 ∈ 𝐴 𝐷) | ||
| Theorem | iunxunsn 32493* | Appending a set to an indexed union. (Contributed by Thierry Arnoux, 20-Nov-2023.) |
| ⊢ (𝑥 = 𝑋 → 𝐵 = 𝐶) ⇒ ⊢ (𝑋 ∈ 𝑉 → ∪ 𝑥 ∈ (𝐴 ∪ {𝑋})𝐵 = (∪ 𝑥 ∈ 𝐴 𝐵 ∪ 𝐶)) | ||
| Theorem | iunxunpr 32494* | Appending two sets to an indexed union. (Contributed by Thierry Arnoux, 20-Nov-2023.) |
| ⊢ (𝑥 = 𝑋 → 𝐵 = 𝐶) & ⊢ (𝑥 = 𝑌 → 𝐵 = 𝐷) ⇒ ⊢ ((𝑋 ∈ 𝑉 ∧ 𝑌 ∈ 𝑊) → ∪ 𝑥 ∈ (𝐴 ∪ {𝑋, 𝑌})𝐵 = (∪ 𝑥 ∈ 𝐴 𝐵 ∪ (𝐶 ∪ 𝐷))) | ||
| Theorem | iunxpssiun1 32495* | Provide an upper bound for the indexed union of cartesian products. (Contributed by Thierry Arnoux, 13-Oct-2025.) |
| ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐶 ⊆ 𝐸) ⇒ ⊢ (𝜑 → ∪ 𝑥 ∈ 𝐴 (𝐵 × 𝐶) ⊆ (∪ 𝑥 ∈ 𝐴 𝐵 × 𝐸)) | ||
| Theorem | iinabrex 32496* | Rewriting an indexed intersection into an intersection of its image set. (Contributed by Thierry Arnoux, 15-Jun-2024.) |
| ⊢ (∀𝑥 ∈ 𝐴 𝐵 ∈ 𝑉 → ∩ 𝑥 ∈ 𝐴 𝐵 = ∩ {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵}) | ||
| Theorem | disjnf 32497* | In case 𝑥 is not free in 𝐵, disjointness is not so interesting since it reduces to cases where 𝐴 is a singleton. (Google Groups discussion with Peter Mazsa.) (Contributed by Thierry Arnoux, 26-Jul-2018.) |
| ⊢ (Disj 𝑥 ∈ 𝐴 𝐵 ↔ (𝐵 = ∅ ∨ ∃*𝑥 𝑥 ∈ 𝐴)) | ||
| Theorem | cbvdisjf 32498* | Change bound variables in a disjoint collection. (Contributed by Thierry Arnoux, 6-Apr-2017.) |
| ⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑦𝐵 & ⊢ Ⅎ𝑥𝐶 & ⊢ (𝑥 = 𝑦 → 𝐵 = 𝐶) ⇒ ⊢ (Disj 𝑥 ∈ 𝐴 𝐵 ↔ Disj 𝑦 ∈ 𝐴 𝐶) | ||
| Theorem | disjss1f 32499 | A subset of a disjoint collection is disjoint. (Contributed by Thierry Arnoux, 6-Apr-2017.) |
| ⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ (𝐴 ⊆ 𝐵 → (Disj 𝑥 ∈ 𝐵 𝐶 → Disj 𝑥 ∈ 𝐴 𝐶)) | ||
| Theorem | disjeq1f 32500 | Equality theorem for disjoint collection. (Contributed by Mario Carneiro, 14-Nov-2016.) |
| ⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ (𝐴 = 𝐵 → (Disj 𝑥 ∈ 𝐴 𝐶 ↔ Disj 𝑥 ∈ 𝐵 𝐶)) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |