HomeHome Intuitionistic Logic Explorer
Theorem List (p. 36 of 156)
< Previous  Next >
Bad symbols? Try the
GIF version.

Mirrors  >  Metamath Home Page  >  ILE Home Page  >  Theorem List Contents  >  Recent Proofs       This page: Page List

Theorem List for Intuitionistic Logic Explorer - 3501-3600   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theoremdisjel 3501 A set can't belong to both members of disjoint classes. (Contributed by NM, 28-Feb-2015.)
(((𝐴𝐵) = ∅ ∧ 𝐶𝐴) → ¬ 𝐶𝐵)
 
Theoremdisj2 3502 Two ways of saying that two classes are disjoint. (Contributed by NM, 17-May-1998.)
((𝐴𝐵) = ∅ ↔ 𝐴 ⊆ (V ∖ 𝐵))
 
Theoremssdisj 3503 Intersection with a subclass of a disjoint class. (Contributed by FL, 24-Jan-2007.)
((𝐴𝐵 ∧ (𝐵𝐶) = ∅) → (𝐴𝐶) = ∅)
 
Theoremundisj1 3504 The union of disjoint classes is disjoint. (Contributed by NM, 26-Sep-2004.)
(((𝐴𝐶) = ∅ ∧ (𝐵𝐶) = ∅) ↔ ((𝐴𝐵) ∩ 𝐶) = ∅)
 
Theoremundisj2 3505 The union of disjoint classes is disjoint. (Contributed by NM, 13-Sep-2004.)
(((𝐴𝐵) = ∅ ∧ (𝐴𝐶) = ∅) ↔ (𝐴 ∩ (𝐵𝐶)) = ∅)
 
Theoremssindif0im 3506 Subclass implies empty intersection with difference from the universal class. (Contributed by NM, 17-Sep-2003.)
(𝐴𝐵 → (𝐴 ∩ (V ∖ 𝐵)) = ∅)
 
Theoreminelcm 3507 The intersection of classes with a common member is nonempty. (Contributed by NM, 7-Apr-1994.)
((𝐴𝐵𝐴𝐶) → (𝐵𝐶) ≠ ∅)
 
Theoremminel 3508 A minimum element of a class has no elements in common with the class. (Contributed by NM, 22-Jun-1994.)
((𝐴𝐵 ∧ (𝐶𝐵) = ∅) → ¬ 𝐴𝐶)
 
Theoremundif4 3509 Distribute union over difference. (Contributed by NM, 17-May-1998.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
((𝐴𝐶) = ∅ → (𝐴 ∪ (𝐵𝐶)) = ((𝐴𝐵) ∖ 𝐶))
 
Theoremdisjssun 3510 Subset relation for disjoint classes. (Contributed by NM, 25-Oct-2005.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
((𝐴𝐵) = ∅ → (𝐴 ⊆ (𝐵𝐶) ↔ 𝐴𝐶))
 
Theoremssdif0im 3511 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.)
(𝐴𝐵 → (𝐴𝐵) = ∅)
 
Theoremvdif0im 3512 Universal class equality in terms of empty difference. (Contributed by Jim Kingdon, 3-Aug-2018.)
(𝐴 = V → (V ∖ 𝐴) = ∅)
 
Theoremdifrab0eqim 3513* 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.)
(𝑉 = {𝑥𝑉𝜑} → (𝑉 ∖ {𝑥𝑉𝜑}) = ∅)
 
Theoreminssdif0im 3514 Intersection, subclass, and difference relationship. In classical logic the converse would also hold. (Contributed by Jim Kingdon, 3-Aug-2018.)
((𝐴𝐵) ⊆ 𝐶 → (𝐴 ∩ (𝐵𝐶)) = ∅)
 
Theoremdifid 3515 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.)
(𝐴𝐴) = ∅
 
TheoremdifidALT 3516 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 3515. (Contributed by David Abernethy, 17-Jun-2012.) (Proof modification is discouraged.) (New usage is discouraged.)
(𝐴𝐴) = ∅
 
Theoremdif0 3517 The difference between a class and the empty set. Part of Exercise 4.4 of [Stoll] p. 16. (Contributed by NM, 17-Aug-2004.)
(𝐴 ∖ ∅) = 𝐴
 
Theorem0dif 3518 The difference between the empty set and a class. Part of Exercise 4.4 of [Stoll] p. 16. (Contributed by NM, 17-Aug-2004.)
(∅ ∖ 𝐴) = ∅
 
Theoremdisjdif 3519 A class and its relative complement are disjoint. Theorem 38 of [Suppes] p. 29. (Contributed by NM, 24-Mar-1998.)
(𝐴 ∩ (𝐵𝐴)) = ∅
 
Theoremdifin0 3520 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.)
((𝐴𝐵) ∖ 𝐵) = ∅
 
Theoremundif1ss 3521 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.)
((𝐴𝐵) ∪ 𝐵) ⊆ (𝐴𝐵)
 
Theoremundif2ss 3522 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.)
(𝐴 ∪ (𝐵𝐴)) ⊆ (𝐴𝐵)
 
Theoremundifabs 3523 Absorption of difference by union. (Contributed by NM, 18-Aug-2013.)
(𝐴 ∪ (𝐴𝐵)) = 𝐴
 
Theoreminundifss 3524 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.)
((𝐴𝐵) ∪ (𝐴𝐵)) ⊆ 𝐴
 
Theoremdisjdif2 3525 The difference of a class and a class disjoint from it is the original class. (Contributed by BJ, 21-Apr-2019.)
((𝐴𝐵) = ∅ → (𝐴𝐵) = 𝐴)
 
Theoremdifun2 3526 Absorption of union by difference. Theorem 36 of [Suppes] p. 29. (Contributed by NM, 19-May-1998.)
((𝐴𝐵) ∖ 𝐵) = (𝐴𝐵)
 
Theoremundifss 3527 Union of complementary parts into whole. (Contributed by Jim Kingdon, 4-Aug-2018.)
(𝐴𝐵 ↔ (𝐴 ∪ (𝐵𝐴)) ⊆ 𝐵)
 
Theoremssdifin0 3528 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.)
(𝐴 ⊆ (𝐵𝐶) → (𝐴𝐶) = ∅)
 
Theoremssdifeq0 3529 A class is a subclass of itself subtracted from another iff it is the empty set. (Contributed by Steve Rodriguez, 20-Nov-2015.)
(𝐴 ⊆ (𝐵𝐴) ↔ 𝐴 = ∅)
 
Theoremssundifim 3530 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.)
(𝐴 ⊆ (𝐵𝐶) → (𝐴𝐵) ⊆ 𝐶)
 
Theoremdifdifdirss 3531 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.)
((𝐴𝐵) ∖ 𝐶) ⊆ ((𝐴𝐶) ∖ (𝐵𝐶))
 
Theoremuneqdifeqim 3532 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.)
((𝐴𝐶 ∧ (𝐴𝐵) = ∅) → ((𝐴𝐵) = 𝐶 → (𝐶𝐴) = 𝐵))
 
Theoremr19.2m 3533* Theorem 19.2 of [Margaris] p. 89 with restricted quantifiers (compare 19.2 1649). 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.)
((∃𝑦 𝑦𝐴 ∧ ∀𝑥𝐴 𝜑) → ∃𝑥𝐴 𝜑)
 
Theoremr19.2mOLD 3534* Theorem 19.2 of [Margaris] p. 89 with restricted quantifiers (compare 19.2 1649). 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 3533 as of 7-Apr-2023. (Proof modification is discouraged.) (New usage is discouraged.)
((∃𝑥 𝑥𝐴 ∧ ∀𝑥𝐴 𝜑) → ∃𝑥𝐴 𝜑)
 
Theoremr19.3rm 3535* Restricted quantification of wff not containing quantified variable. (Contributed by Jim Kingdon, 19-Dec-2018.)
𝑥𝜑       (∃𝑦 𝑦𝐴 → (𝜑 ↔ ∀𝑥𝐴 𝜑))
 
Theoremr19.28m 3536* 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.)
𝑥𝜑       (∃𝑥 𝑥𝐴 → (∀𝑥𝐴 (𝜑𝜓) ↔ (𝜑 ∧ ∀𝑥𝐴 𝜓)))
 
Theoremr19.3rmv 3537* Restricted quantification of wff not containing quantified variable. (Contributed by Jim Kingdon, 6-Aug-2018.)
(∃𝑦 𝑦𝐴 → (𝜑 ↔ ∀𝑥𝐴 𝜑))
 
Theoremr19.9rmv 3538* Restricted quantification of wff not containing quantified variable. (Contributed by Jim Kingdon, 5-Aug-2018.)
(∃𝑦 𝑦𝐴 → (𝜑 ↔ ∃𝑥𝐴 𝜑))
 
Theoremr19.28mv 3539* 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, 6-Aug-2018.)
(∃𝑥 𝑥𝐴 → (∀𝑥𝐴 (𝜑𝜓) ↔ (𝜑 ∧ ∀𝑥𝐴 𝜓)))
 
Theoremr19.45mv 3540* Restricted version of Theorem 19.45 of [Margaris] p. 90. (Contributed by NM, 27-May-1998.)
(∃𝑥 𝑥𝐴 → (∃𝑥𝐴 (𝜑𝜓) ↔ (𝜑 ∨ ∃𝑥𝐴 𝜓)))
 
Theoremr19.44mv 3541* Restricted version of Theorem 19.44 of [Margaris] p. 90. (Contributed by NM, 27-May-1998.)
(∃𝑦 𝑦𝐴 → (∃𝑥𝐴 (𝜑𝜓) ↔ (∃𝑥𝐴 𝜑𝜓)))
 
Theoremr19.27m 3542* Restricted quantifier version of Theorem 19.27 of [Margaris] p. 90. It is valid only when the domain of quantification is inhabited. (Contributed by Jim Kingdon, 5-Aug-2018.)
𝑥𝜓       (∃𝑥 𝑥𝐴 → (∀𝑥𝐴 (𝜑𝜓) ↔ (∀𝑥𝐴 𝜑𝜓)))
 
Theoremr19.27mv 3543* Restricted quantifier version of Theorem 19.27 of [Margaris] p. 90. It is valid only when the domain of quantification is inhabited. (Contributed by Jim Kingdon, 5-Aug-2018.)
(∃𝑥 𝑥𝐴 → (∀𝑥𝐴 (𝜑𝜓) ↔ (∀𝑥𝐴 𝜑𝜓)))
 
Theoremrzal 3544* Vacuous quantification is always true. (Contributed by NM, 11-Mar-1997.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
(𝐴 = ∅ → ∀𝑥𝐴 𝜑)
 
Theoremrexn0 3545* Restricted existential quantification implies its restriction is nonempty (it is also inhabited as shown in rexm 3546). (Contributed by Szymon Jaroszewicz, 3-Apr-2007.)
(∃𝑥𝐴 𝜑𝐴 ≠ ∅)
 
Theoremrexm 3546* Restricted existential quantification implies its restriction is inhabited. (Contributed by Jim Kingdon, 16-Oct-2018.)
(∃𝑥𝐴 𝜑 → ∃𝑥 𝑥𝐴)
 
Theoremralidm 3547* Idempotent law for restricted quantifier. (Contributed by NM, 28-Mar-1997.)
(∀𝑥𝐴𝑥𝐴 𝜑 ↔ ∀𝑥𝐴 𝜑)
 
Theoremral0 3548 Vacuous universal quantification is always true. (Contributed by NM, 20-Oct-2005.)
𝑥 ∈ ∅ 𝜑
 
Theoremralf0 3549* The quantification of a falsehood is vacuous when true. (Contributed by NM, 26-Nov-2005.)
¬ 𝜑       (∀𝑥𝐴 𝜑𝐴 = ∅)
 
Theoremralm 3550 Inhabited classes and restricted quantification. (Contributed by Jim Kingdon, 6-Aug-2018.)
((∃𝑥 𝑥𝐴 → ∀𝑥𝐴 𝜑) ↔ ∀𝑥𝐴 𝜑)
 
Theoremraaanlem 3551* Special case of raaan 3552 where 𝐴 is inhabited. (Contributed by Jim Kingdon, 6-Aug-2018.)
𝑦𝜑    &   𝑥𝜓       (∃𝑥 𝑥𝐴 → (∀𝑥𝐴𝑦𝐴 (𝜑𝜓) ↔ (∀𝑥𝐴 𝜑 ∧ ∀𝑦𝐴 𝜓)))
 
Theoremraaan 3552* Rearrange restricted quantifiers. (Contributed by NM, 26-Oct-2010.)
𝑦𝜑    &   𝑥𝜓       (∀𝑥𝐴𝑦𝐴 (𝜑𝜓) ↔ (∀𝑥𝐴 𝜑 ∧ ∀𝑦𝐴 𝜓))
 
Theoremraaanv 3553* Rearrange restricted quantifiers. (Contributed by NM, 11-Mar-1997.)
(∀𝑥𝐴𝑦𝐴 (𝜑𝜓) ↔ (∀𝑥𝐴 𝜑 ∧ ∀𝑦𝐴 𝜓))
 
Theoremsbss 3554* Set substitution into the first argument of a subset relation. (Contributed by Rodolfo Medina, 7-Jul-2010.) (Proof shortened by Mario Carneiro, 14-Nov-2016.)
([𝑦 / 𝑥]𝑥𝐴𝑦𝐴)
 
Theoremsbcssg 3555 Distribute proper substitution through a subclass relation. (Contributed by Alan Sare, 22-Jul-2012.) (Proof shortened by Alexander van der Vekens, 23-Jul-2017.)
(𝐴𝑉 → ([𝐴 / 𝑥]𝐵𝐶𝐴 / 𝑥𝐵𝐴 / 𝑥𝐶))
 
Theoremdcun 3556 The union of two decidable classes is decidable. (Contributed by Jim Kingdon, 5-Oct-2022.)
(𝜑DECID 𝑘𝐴)    &   (𝜑DECID 𝑘𝐵)       (𝜑DECID 𝑘 ∈ (𝐴𝐵))
 
2.1.15  Conditional operator
 
Syntaxcif 3557 Extend class notation to include the conditional operator. See df-if 3558 for a description. (In older databases this was denoted "ded".)
class if(𝜑, 𝐴, 𝐵)
 
Definitiondf-if 3558* Define the conditional operator. Read if(𝜑, 𝐴, 𝐵) as "if 𝜑 then 𝐴 else 𝐵". See iftrue 3562 and iffalse 3565 for its values. In mathematical literature, this operator is rarely defined formally but is implicit in informal definitions such as "let f(x)=0 if x=0 and 1/x otherwise."

In the absence of excluded middle, this will tend to be useful where 𝜑 is decidable (in the sense of df-dc 836). (Contributed by NM, 15-May-1999.)

if(𝜑, 𝐴, 𝐵) = {𝑥 ∣ ((𝑥𝐴𝜑) ∨ (𝑥𝐵 ∧ ¬ 𝜑))}
 
Theoremdfif6 3559* An alternate definition of the conditional operator df-if 3558 as a simple class abstraction. (Contributed by Mario Carneiro, 8-Sep-2013.)
if(𝜑, 𝐴, 𝐵) = ({𝑥𝐴𝜑} ∪ {𝑥𝐵 ∣ ¬ 𝜑})
 
Theoremifeq1 3560 Equality theorem for conditional operator. (Contributed by NM, 1-Sep-2004.) (Revised by Mario Carneiro, 8-Sep-2013.)
(𝐴 = 𝐵 → if(𝜑, 𝐴, 𝐶) = if(𝜑, 𝐵, 𝐶))
 
Theoremifeq2 3561 Equality theorem for conditional operator. (Contributed by NM, 1-Sep-2004.) (Revised by Mario Carneiro, 8-Sep-2013.)
(𝐴 = 𝐵 → if(𝜑, 𝐶, 𝐴) = if(𝜑, 𝐶, 𝐵))
 
Theoremiftrue 3562 Value of the conditional operator when its first argument is true. (Contributed by NM, 15-May-1999.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
(𝜑 → if(𝜑, 𝐴, 𝐵) = 𝐴)
 
Theoremiftruei 3563 Inference associated with iftrue 3562. (Contributed by BJ, 7-Oct-2018.)
𝜑       if(𝜑, 𝐴, 𝐵) = 𝐴
 
Theoremiftrued 3564 Value of the conditional operator when its first argument is true. (Contributed by Glauco Siliprandi, 11-Dec-2019.)
(𝜑𝜒)       (𝜑 → if(𝜒, 𝐴, 𝐵) = 𝐴)
 
Theoremiffalse 3565 Value of the conditional operator when its first argument is false. (Contributed by NM, 14-Aug-1999.)
𝜑 → if(𝜑, 𝐴, 𝐵) = 𝐵)
 
Theoremiffalsei 3566 Inference associated with iffalse 3565. (Contributed by BJ, 7-Oct-2018.)
¬ 𝜑       if(𝜑, 𝐴, 𝐵) = 𝐵
 
Theoremiffalsed 3567 Value of the conditional operator when its first argument is false. (Contributed by Glauco Siliprandi, 11-Dec-2019.)
(𝜑 → ¬ 𝜒)       (𝜑 → if(𝜒, 𝐴, 𝐵) = 𝐵)
 
Theoremifnefalse 3568 When values are unequal, but an "if" condition checks if they are equal, then the "false" branch results. This is a simple utility to provide a slight shortening and simplification of proofs versus applying iffalse 3565 directly in this case. (Contributed by David A. Wheeler, 15-May-2015.)
(𝐴𝐵 → if(𝐴 = 𝐵, 𝐶, 𝐷) = 𝐷)
 
Theoremifsbdc 3569 Distribute a function over an if-clause. (Contributed by Jim Kingdon, 1-Jan-2022.)
(if(𝜑, 𝐴, 𝐵) = 𝐴𝐶 = 𝐷)    &   (if(𝜑, 𝐴, 𝐵) = 𝐵𝐶 = 𝐸)       (DECID 𝜑𝐶 = if(𝜑, 𝐷, 𝐸))
 
Theoremdfif3 3570* Alternate definition of the conditional operator df-if 3558. Note that 𝜑 is independent of 𝑥 i.e. a constant true or false. (Contributed by NM, 25-Aug-2013.) (Revised by Mario Carneiro, 8-Sep-2013.)
𝐶 = {𝑥𝜑}       if(𝜑, 𝐴, 𝐵) = ((𝐴𝐶) ∪ (𝐵 ∩ (V ∖ 𝐶)))
 
Theoremifssun 3571 A conditional class is included in the union of its two alternatives. (Contributed by BJ, 15-Aug-2024.)
if(𝜑, 𝐴, 𝐵) ⊆ (𝐴𝐵)
 
Theoremifidss 3572 A conditional class whose two alternatives are equal is included in that alternative. With excluded middle, we can prove it is equal to it. (Contributed by BJ, 15-Aug-2024.)
if(𝜑, 𝐴, 𝐴) ⊆ 𝐴
 
Theoremifeq12 3573 Equality theorem for conditional operators. (Contributed by NM, 1-Sep-2004.)
((𝐴 = 𝐵𝐶 = 𝐷) → if(𝜑, 𝐴, 𝐶) = if(𝜑, 𝐵, 𝐷))
 
Theoremifeq1d 3574 Equality deduction for conditional operator. (Contributed by NM, 16-Feb-2005.)
(𝜑𝐴 = 𝐵)       (𝜑 → if(𝜓, 𝐴, 𝐶) = if(𝜓, 𝐵, 𝐶))
 
Theoremifeq2d 3575 Equality deduction for conditional operator. (Contributed by NM, 16-Feb-2005.)
(𝜑𝐴 = 𝐵)       (𝜑 → if(𝜓, 𝐶, 𝐴) = if(𝜓, 𝐶, 𝐵))
 
Theoremifeq12d 3576 Equality deduction for conditional operator. (Contributed by NM, 24-Mar-2015.)
(𝜑𝐴 = 𝐵)    &   (𝜑𝐶 = 𝐷)       (𝜑 → if(𝜓, 𝐴, 𝐶) = if(𝜓, 𝐵, 𝐷))
 
Theoremifbi 3577 Equivalence theorem for conditional operators. (Contributed by Raph Levien, 15-Jan-2004.)
((𝜑𝜓) → if(𝜑, 𝐴, 𝐵) = if(𝜓, 𝐴, 𝐵))
 
Theoremifbid 3578 Equivalence deduction for conditional operators. (Contributed by NM, 18-Apr-2005.)
(𝜑 → (𝜓𝜒))       (𝜑 → if(𝜓, 𝐴, 𝐵) = if(𝜒, 𝐴, 𝐵))
 
Theoremifbieq1d 3579 Equivalence/equality deduction for conditional operators. (Contributed by JJ, 25-Sep-2018.)
(𝜑 → (𝜓𝜒))    &   (𝜑𝐴 = 𝐵)       (𝜑 → if(𝜓, 𝐴, 𝐶) = if(𝜒, 𝐵, 𝐶))
 
Theoremifbieq2i 3580 Equivalence/equality inference for conditional operators. (Contributed by Paul Chapman, 22-Jun-2011.)
(𝜑𝜓)    &   𝐴 = 𝐵       if(𝜑, 𝐶, 𝐴) = if(𝜓, 𝐶, 𝐵)
 
Theoremifbieq2d 3581 Equivalence/equality deduction for conditional operators. (Contributed by Paul Chapman, 22-Jun-2011.)
(𝜑 → (𝜓𝜒))    &   (𝜑𝐴 = 𝐵)       (𝜑 → if(𝜓, 𝐶, 𝐴) = if(𝜒, 𝐶, 𝐵))
 
Theoremifbieq12i 3582 Equivalence deduction for conditional operators. (Contributed by NM, 18-Mar-2013.)
(𝜑𝜓)    &   𝐴 = 𝐶    &   𝐵 = 𝐷       if(𝜑, 𝐴, 𝐵) = if(𝜓, 𝐶, 𝐷)
 
Theoremifbieq12d 3583 Equivalence deduction for conditional operators. (Contributed by Jeff Madsen, 2-Sep-2009.)
(𝜑 → (𝜓𝜒))    &   (𝜑𝐴 = 𝐶)    &   (𝜑𝐵 = 𝐷)       (𝜑 → if(𝜓, 𝐴, 𝐵) = if(𝜒, 𝐶, 𝐷))
 
Theoremnfifd 3584 Deduction version of nfif 3585. (Contributed by NM, 15-Feb-2013.) (Revised by Mario Carneiro, 13-Oct-2016.)
(𝜑 → Ⅎ𝑥𝜓)    &   (𝜑𝑥𝐴)    &   (𝜑𝑥𝐵)       (𝜑𝑥if(𝜓, 𝐴, 𝐵))
 
Theoremnfif 3585 Bound-variable hypothesis builder for a conditional operator. (Contributed by NM, 16-Feb-2005.) (Proof shortened by Andrew Salmon, 26-Jun-2011.)
𝑥𝜑    &   𝑥𝐴    &   𝑥𝐵       𝑥if(𝜑, 𝐴, 𝐵)
 
Theoremifcldadc 3586 Conditional closure. (Contributed by Jim Kingdon, 11-Jan-2022.)
((𝜑𝜓) → 𝐴𝐶)    &   ((𝜑 ∧ ¬ 𝜓) → 𝐵𝐶)    &   (𝜑DECID 𝜓)       (𝜑 → if(𝜓, 𝐴, 𝐵) ∈ 𝐶)
 
Theoremifeq1dadc 3587 Conditional equality. (Contributed by Jeff Madsen, 2-Sep-2009.)
((𝜑𝜓) → 𝐴 = 𝐵)    &   (𝜑DECID 𝜓)       (𝜑 → if(𝜓, 𝐴, 𝐶) = if(𝜓, 𝐵, 𝐶))
 
Theoremifeq2dadc 3588 Conditional equality. (Contributed by Jeff Madsen, 2-Sep-2009.)
((𝜑 ∧ ¬ 𝜓) → 𝐴 = 𝐵)    &   (𝜑DECID 𝜓)       (𝜑 → if(𝜓, 𝐶, 𝐴) = if(𝜓, 𝐶, 𝐵))
 
Theoremifbothdadc 3589 A formula 𝜃 containing a decidable conditional operator is true when both of its cases are true. (Contributed by Jim Kingdon, 3-Jun-2022.)
(𝐴 = if(𝜑, 𝐴, 𝐵) → (𝜓𝜃))    &   (𝐵 = if(𝜑, 𝐴, 𝐵) → (𝜒𝜃))    &   ((𝜂𝜑) → 𝜓)    &   ((𝜂 ∧ ¬ 𝜑) → 𝜒)    &   (𝜂DECID 𝜑)       (𝜂𝜃)
 
Theoremifbothdc 3590 A wff 𝜃 containing a conditional operator is true when both of its cases are true. (Contributed by Jim Kingdon, 8-Aug-2021.)
(𝐴 = if(𝜑, 𝐴, 𝐵) → (𝜓𝜃))    &   (𝐵 = if(𝜑, 𝐴, 𝐵) → (𝜒𝜃))       ((𝜓𝜒DECID 𝜑) → 𝜃)
 
Theoremifiddc 3591 Identical true and false arguments in the conditional operator. (Contributed by NM, 18-Apr-2005.)
(DECID 𝜑 → if(𝜑, 𝐴, 𝐴) = 𝐴)
 
Theoremeqifdc 3592 Expansion of an equality with a conditional operator. (Contributed by Jim Kingdon, 28-Jul-2022.)
(DECID 𝜑 → (𝐴 = if(𝜑, 𝐵, 𝐶) ↔ ((𝜑𝐴 = 𝐵) ∨ (¬ 𝜑𝐴 = 𝐶))))
 
Theoremifcldcd 3593 Membership (closure) of a conditional operator, deduction form. (Contributed by Jim Kingdon, 8-Aug-2021.)
(𝜑𝐴𝐶)    &   (𝜑𝐵𝐶)    &   (𝜑DECID 𝜓)       (𝜑 → if(𝜓, 𝐴, 𝐵) ∈ 𝐶)
 
Theoremifnotdc 3594 Negating the first argument swaps the last two arguments of a conditional operator. (Contributed by NM, 21-Jun-2007.)
(DECID 𝜑 → if(¬ 𝜑, 𝐴, 𝐵) = if(𝜑, 𝐵, 𝐴))
 
Theoremifandc 3595 Rewrite a conjunction in a conditional as two nested conditionals. (Contributed by Mario Carneiro, 28-Jul-2014.)
(DECID 𝜑 → if((𝜑𝜓), 𝐴, 𝐵) = if(𝜑, if(𝜓, 𝐴, 𝐵), 𝐵))
 
Theoremifordc 3596 Rewrite a disjunction in a conditional as two nested conditionals. (Contributed by Mario Carneiro, 28-Jul-2014.)
(DECID 𝜑 → if((𝜑𝜓), 𝐴, 𝐵) = if(𝜑, 𝐴, if(𝜓, 𝐴, 𝐵)))
 
Theoremifmdc 3597 If a conditional class is inhabited, then the condition is decidable. This shows that conditionals are not very useful unless one can prove the condition decidable. (Contributed by BJ, 24-Sep-2022.)
(𝐴 ∈ if(𝜑, 𝐵, 𝐶) → DECID 𝜑)
 
Theoremifnetruedc 3598 Deduce truth from a conditional operator value. (Contributed by Thierry Arnoux, 20-Feb-2025.)
((DECID 𝜑𝐴𝐵 ∧ if(𝜑, 𝐴, 𝐵) = 𝐴) → 𝜑)
 
Theoremifnefals 3599 Deduce falsehood from a conditional operator value. (Contributed by Thierry Arnoux, 20-Feb-2025.)
((𝐴𝐵 ∧ if(𝜑, 𝐴, 𝐵) = 𝐵) → ¬ 𝜑)
 
Theoremifnebibdc 3600 The converse of ifbi 3577 holds if the two values are not equal. (Contributed by Thierry Arnoux, 20-Feb-2025.)
((DECID 𝜑DECID 𝜓𝐴𝐵) → (if(𝜑, 𝐴, 𝐵) = if(𝜓, 𝐴, 𝐵) ↔ (𝜑𝜓)))
    < Previous  Next >

Page List
Jump to page: Contents  1 1-100 2 101-200 3 201-300 4 301-400 5 401-500 6 501-600 7 601-700 8 701-800 9 801-900 10 901-1000 11 1001-1100 12 1101-1200 13 1201-1300 14 1301-1400 15 1401-1500 16 1501-1600 17 1601-1700 18 1701-1800 19 1801-1900 20 1901-2000 21 2001-2100 22 2101-2200 23 2201-2300 24 2301-2400 25 2401-2500 26 2501-2600 27 2601-2700 28 2701-2800 29 2801-2900 30 2901-3000 31 3001-3100 32 3101-3200 33 3201-3300 34 3301-3400 35 3401-3500 36 3501-3600 37 3601-3700 38 3701-3800 39 3801-3900 40 3901-4000 41 4001-4100 42 4101-4200 43 4201-4300 44 4301-4400 45 4401-4500 46 4501-4600 47 4601-4700 48 4701-4800 49 4801-4900 50 4901-5000 51 5001-5100 52 5101-5200 53 5201-5300 54 5301-5400 55 5401-5500 56 5501-5600 57 5601-5700 58 5701-5800 59 5801-5900 60 5901-6000 61 6001-6100 62 6101-6200 63 6201-6300 64 6301-6400 65 6401-6500 66 6501-6600 67 6601-6700 68 6701-6800 69 6801-6900 70 6901-7000 71 7001-7100 72 7101-7200 73 7201-7300 74 7301-7400 75 7401-7500 76 7501-7600 77 7601-7700 78 7701-7800 79 7801-7900 80 7901-8000 81 8001-8100 82 8101-8200 83 8201-8300 84 8301-8400 85 8401-8500 86 8501-8600 87 8601-8700 88 8701-8800 89 8801-8900 90 8901-9000 91 9001-9100 92 9101-9200 93 9201-9300 94 9301-9400 95 9401-9500 96 9501-9600 97 9601-9700 98 9701-9800 99 9801-9900 100 9901-10000 101 10001-10100 102 10101-10200 103 10201-10300 104 10301-10400 105 10401-10500 106 10501-10600 107 10601-10700 108 10701-10800 109 10801-10900 110 10901-11000 111 11001-11100 112 11101-11200 113 11201-11300 114 11301-11400 115 11401-11500 116 11501-11600 117 11601-11700 118 11701-11800 119 11801-11900 120 11901-12000 121 12001-12100 122 12101-12200 123 12201-12300 124 12301-12400 125 12401-12500 126 12501-12600 127 12601-12700 128 12701-12800 129 12801-12900 130 12901-13000 131 13001-13100 132 13101-13200 133 13201-13300 134 13301-13400 135 13401-13500 136 13501-13600 137 13601-13700 138 13701-13800 139 13801-13900 140 13901-14000 141 14001-14100 142 14101-14200 143 14201-14300 144 14301-14400 145 14401-14500 146 14501-14600 147 14601-14700 148 14701-14800 149 14801-14900 150 14901-15000 151 15001-15100 152 15101-15200 153 15201-15300 154 15301-15400 155 15401-15500 156 15501-15574
  Copyright terms: Public domain < Previous  Next >