HomeHome Intuitionistic Logic Explorer
Theorem List (p. 21 of 140)
< 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 - 2001-2100   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theoremhbsb4t 2001 A variable not free remains so after substitution with a distinct variable (closed form of hbsb4 2000). (Contributed by NM, 7-Apr-2004.) (Proof shortened by Andrew Salmon, 25-May-2011.)
(∀𝑥𝑧(𝜑 → ∀𝑧𝜑) → (¬ ∀𝑧 𝑧 = 𝑦 → ([𝑦 / 𝑥]𝜑 → ∀𝑧[𝑦 / 𝑥]𝜑)))
 
Theoremnfsb4t 2002 A variable not free remains so after substitution with a distinct variable (closed form of hbsb4 2000). (Contributed by NM, 7-Apr-2004.) (Revised by Mario Carneiro, 4-Oct-2016.) (Proof rewritten by Jim Kingdon, 9-May-2018.)
(∀𝑥𝑧𝜑 → (¬ ∀𝑧 𝑧 = 𝑦 → Ⅎ𝑧[𝑦 / 𝑥]𝜑))
 
Theoremdvelimf 2003 Version of dvelim 2005 without any variable restrictions. (Contributed by NM, 1-Oct-2002.)
(𝜑 → ∀𝑥𝜑)    &   (𝜓 → ∀𝑧𝜓)    &   (𝑧 = 𝑦 → (𝜑𝜓))       (¬ ∀𝑥 𝑥 = 𝑦 → (𝜓 → ∀𝑥𝜓))
 
Theoremdvelimdf 2004 Deduction form of dvelimf 2003. This version may be useful if we want to avoid ax-17 1514 and use ax-16 1802 instead. (Contributed by NM, 7-Apr-2004.) (Revised by Mario Carneiro, 6-Oct-2016.) (Proof shortened by Wolf Lammen, 11-May-2018.)
𝑥𝜑    &   𝑧𝜑    &   (𝜑 → Ⅎ𝑥𝜓)    &   (𝜑 → Ⅎ𝑧𝜒)    &   (𝜑 → (𝑧 = 𝑦 → (𝜓𝜒)))       (𝜑 → (¬ ∀𝑥 𝑥 = 𝑦 → Ⅎ𝑥𝜒))
 
Theoremdvelim 2005* This theorem can be used to eliminate a distinct variable restriction on 𝑥 and 𝑧 and replace it with the "distinctor" ¬ ∀𝑥𝑥 = 𝑦 as an antecedent. 𝜑 normally has 𝑧 free and can be read 𝜑(𝑧), and 𝜓 substitutes 𝑦 for 𝑧 and can be read 𝜑(𝑦). We don't require that 𝑥 and 𝑦 be distinct: if they aren't, the distinctor will become false (in multiple-element domains of discourse) and "protect" the consequent.

To obtain a closed-theorem form of this inference, prefix the hypotheses with 𝑥𝑧, conjoin them, and apply dvelimdf 2004.

Other variants of this theorem are dvelimf 2003 (with no distinct variable restrictions) and dvelimALT 1998 (that avoids ax-10 1493). (Contributed by NM, 23-Nov-1994.)

(𝜑 → ∀𝑥𝜑)    &   (𝑧 = 𝑦 → (𝜑𝜓))       (¬ ∀𝑥 𝑥 = 𝑦 → (𝜓 → ∀𝑥𝜓))
 
Theoremdvelimor 2006* Disjunctive distinct variable constraint elimination. A user of this theorem starts with a formula 𝜑 (containing 𝑧) and a distinct variable constraint between 𝑥 and 𝑧. The theorem makes it possible to replace the distinct variable constraint with the disjunct 𝑥𝑥 = 𝑦 (𝜓 is just a version of 𝜑 with 𝑦 substituted for 𝑧). (Contributed by Jim Kingdon, 11-May-2018.)
𝑥𝜑    &   (𝑧 = 𝑦 → (𝜑𝜓))       (∀𝑥 𝑥 = 𝑦 ∨ Ⅎ𝑥𝜓)
 
Theoremdveeq1 2007* Quantifier introduction when one pair of variables is distinct. (Contributed by NM, 2-Jan-2002.) (Proof rewritten by Jim Kingdon, 19-Feb-2018.)
(¬ ∀𝑥 𝑥 = 𝑦 → (𝑦 = 𝑧 → ∀𝑥 𝑦 = 𝑧))
 
Theoremsbal2 2008* Move quantifier in and out of substitution. (Contributed by NM, 2-Jan-2002.)
(¬ ∀𝑥 𝑥 = 𝑦 → ([𝑧 / 𝑦]∀𝑥𝜑 ↔ ∀𝑥[𝑧 / 𝑦]𝜑))
 
Theoremnfsb4or 2009 A variable not free remains so after substitution with a distinct variable. (Contributed by Jim Kingdon, 11-May-2018.)
𝑧𝜑       (∀𝑧 𝑧 = 𝑦 ∨ Ⅎ𝑧[𝑦 / 𝑥]𝜑)
 
Theoremnfd2 2010 Deduce that 𝑥 is not free in 𝜓 in a context. (Contributed by Wolf Lammen, 16-Sep-2021.)
(𝜑 → (∃𝑥𝜓 → ∀𝑥𝜓))       (𝜑 → Ⅎ𝑥𝜓)
 
Theoremhbe1a 2011 Dual statement of hbe1 1483. (Contributed by Wolf Lammen, 15-Sep-2021.)
(∃𝑥𝑥𝜑 → ∀𝑥𝜑)
 
Theoremnf5-1 2012 One direction of nf5 . (Contributed by Wolf Lammen, 16-Sep-2021.)
(∀𝑥(𝜑 → ∀𝑥𝜑) → Ⅎ𝑥𝜑)
 
Theoremnf5d 2013 Deduce that 𝑥 is not free in 𝜓 in a context. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   (𝜑 → (𝜓 → ∀𝑥𝜓))       (𝜑 → Ⅎ𝑥𝜓)
 
1.4.6  Existential uniqueness
 
Syntaxweu 2014 Extend wff definition to include existential uniqueness ("there exists a unique 𝑥 such that 𝜑").
wff ∃!𝑥𝜑
 
Syntaxwmo 2015 Extend wff definition to include uniqueness ("there exists at most one 𝑥 such that 𝜑").
wff ∃*𝑥𝜑
 
Theoremeujust 2016* A soundness justification theorem for df-eu 2017, showing that the definition is equivalent to itself with its dummy variable renamed. Note that 𝑦 and 𝑧 needn't be distinct variables. (Contributed by NM, 11-Mar-2010.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
(∃𝑦𝑥(𝜑𝑥 = 𝑦) ↔ ∃𝑧𝑥(𝜑𝑥 = 𝑧))
 
Definitiondf-eu 2017* Define existential uniqueness, i.e., "there exists exactly one 𝑥 such that 𝜑". Definition 10.1 of [BellMachover] p. 97; also Definition *14.02 of [WhiteheadRussell] p. 175. Other possible definitions are given by eu1 2039, eu2 2058, eu3 2060, and eu5 2061 (which in some cases we show with a hypothesis 𝜑 → ∀𝑦𝜑 in place of a distinct variable condition on 𝑦 and 𝜑). Double uniqueness is tricky: ∃!𝑥∃!𝑦𝜑 does not mean "exactly one 𝑥 and one 𝑦 " (see 2eu4 2107). (Contributed by NM, 5-Aug-1993.)
(∃!𝑥𝜑 ↔ ∃𝑦𝑥(𝜑𝑥 = 𝑦))
 
Definitiondf-mo 2018 Define "there exists at most one 𝑥 such that 𝜑". Here we define it in terms of existential uniqueness. Notation of [BellMachover] p. 460, whose definition we show as mo3 2068. For another possible definition see mo4 2075. (Contributed by NM, 5-Aug-1993.)
(∃*𝑥𝜑 ↔ (∃𝑥𝜑 → ∃!𝑥𝜑))
 
Theoremeuf 2019* A version of the existential uniqueness definition with a hypothesis instead of a distinct variable condition. (Contributed by NM, 12-Aug-1993.)
(𝜑 → ∀𝑦𝜑)       (∃!𝑥𝜑 ↔ ∃𝑦𝑥(𝜑𝑥 = 𝑦))
 
Theoremeubidh 2020 Formula-building rule for unique existential quantifier (deduction form). (Contributed by NM, 9-Jul-1994.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃!𝑥𝜓 ↔ ∃!𝑥𝜒))
 
Theoremeubid 2021 Formula-building rule for unique existential quantifier (deduction form). (Contributed by NM, 9-Jul-1994.)
𝑥𝜑    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃!𝑥𝜓 ↔ ∃!𝑥𝜒))
 
Theoremeubidv 2022* Formula-building rule for unique existential quantifier (deduction form). (Contributed by NM, 9-Jul-1994.)
(𝜑 → (𝜓𝜒))       (𝜑 → (∃!𝑥𝜓 ↔ ∃!𝑥𝜒))
 
Theoremeubii 2023 Introduce unique existential quantifier to both sides of an equivalence. (Contributed by NM, 9-Jul-1994.) (Revised by Mario Carneiro, 6-Oct-2016.)
(𝜑𝜓)       (∃!𝑥𝜑 ↔ ∃!𝑥𝜓)
 
Theoremhbeu1 2024 Bound-variable hypothesis builder for uniqueness. (Contributed by NM, 9-Jul-1994.)
(∃!𝑥𝜑 → ∀𝑥∃!𝑥𝜑)
 
Theoremnfeu1 2025 Bound-variable hypothesis builder for uniqueness. (Contributed by NM, 9-Jul-1994.) (Revised by Mario Carneiro, 7-Oct-2016.)
𝑥∃!𝑥𝜑
 
Theoremnfmo1 2026 Bound-variable hypothesis builder for "at most one". (Contributed by NM, 8-Mar-1995.) (Revised by Mario Carneiro, 7-Oct-2016.)
𝑥∃*𝑥𝜑
 
Theoremsb8eu 2027 Variable substitution in unique existential quantifier. (Contributed by NM, 7-Aug-1994.) (Revised by Mario Carneiro, 7-Oct-2016.)
𝑦𝜑       (∃!𝑥𝜑 ↔ ∃!𝑦[𝑦 / 𝑥]𝜑)
 
Theoremsb8mo 2028 Variable substitution for "at most one". (Contributed by Alexander van der Vekens, 17-Jun-2017.)
𝑦𝜑       (∃*𝑥𝜑 ↔ ∃*𝑦[𝑦 / 𝑥]𝜑)
 
Theoremnfeudv 2029* Deduction version of nfeu 2033. Similar to nfeud 2030 but has the additional constraint that 𝑥 and 𝑦 must be distinct. (Contributed by Jim Kingdon, 25-May-2018.)
𝑦𝜑    &   (𝜑 → Ⅎ𝑥𝜓)       (𝜑 → Ⅎ𝑥∃!𝑦𝜓)
 
Theoremnfeud 2030 Deduction version of nfeu 2033. (Contributed by NM, 15-Feb-2013.) (Revised by Mario Carneiro, 7-Oct-2016.) (Proof rewritten by Jim Kingdon, 25-May-2018.)
𝑦𝜑    &   (𝜑 → Ⅎ𝑥𝜓)       (𝜑 → Ⅎ𝑥∃!𝑦𝜓)
 
Theoremnfmod 2031 Bound-variable hypothesis builder for "at most one". (Contributed by Mario Carneiro, 14-Nov-2016.)
𝑦𝜑    &   (𝜑 → Ⅎ𝑥𝜓)       (𝜑 → Ⅎ𝑥∃*𝑦𝜓)
 
Theoremnfeuv 2032* Bound-variable hypothesis builder for existential uniqueness. This is similar to nfeu 2033 but has the additional condition that 𝑥 and 𝑦 must be distinct. (Contributed by Jim Kingdon, 23-May-2018.)
𝑥𝜑       𝑥∃!𝑦𝜑
 
Theoremnfeu 2033 Bound-variable hypothesis builder for existential uniqueness. Note that 𝑥 and 𝑦 needn't be distinct. (Contributed by NM, 8-Mar-1995.) (Revised by Mario Carneiro, 7-Oct-2016.) (Proof rewritten by Jim Kingdon, 23-May-2018.)
𝑥𝜑       𝑥∃!𝑦𝜑
 
Theoremnfmo 2034 Bound-variable hypothesis builder for "at most one". (Contributed by NM, 9-Mar-1995.)
𝑥𝜑       𝑥∃*𝑦𝜑
 
Theoremhbeu 2035 Bound-variable hypothesis builder for uniqueness. Note that 𝑥 and 𝑦 needn't be distinct. (Contributed by NM, 8-Mar-1995.) (Proof rewritten by Jim Kingdon, 24-May-2018.)
(𝜑 → ∀𝑥𝜑)       (∃!𝑦𝜑 → ∀𝑥∃!𝑦𝜑)
 
Theoremhbeud 2036 Deduction version of hbeu 2035. (Contributed by NM, 15-Feb-2013.) (Proof rewritten by Jim Kingdon, 25-May-2018.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → ∀𝑦𝜑)    &   (𝜑 → (𝜓 → ∀𝑥𝜓))       (𝜑 → (∃!𝑦𝜓 → ∀𝑥∃!𝑦𝜓))
 
Theoremsb8euh 2037 Variable substitution in unique existential quantifier. (Contributed by NM, 7-Aug-1994.) (Revised by Andrew Salmon, 9-Jul-2011.)
(𝜑 → ∀𝑦𝜑)       (∃!𝑥𝜑 ↔ ∃!𝑦[𝑦 / 𝑥]𝜑)
 
Theoremcbveu 2038 Rule used to change bound variables, using implicit substitution. (Contributed by NM, 25-Nov-1994.) (Revised by Mario Carneiro, 7-Oct-2016.)
𝑦𝜑    &   𝑥𝜓    &   (𝑥 = 𝑦 → (𝜑𝜓))       (∃!𝑥𝜑 ↔ ∃!𝑦𝜓)
 
Theoremeu1 2039* An alternate way to express uniqueness used by some authors. Exercise 2(b) of [Margaris] p. 110. (Contributed by NM, 20-Aug-1993.)
(𝜑 → ∀𝑦𝜑)       (∃!𝑥𝜑 ↔ ∃𝑥(𝜑 ∧ ∀𝑦([𝑦 / 𝑥]𝜑𝑥 = 𝑦)))
 
Theoremeuor 2040 Introduce a disjunct into a unique existential quantifier. (Contributed by NM, 21-Oct-2005.)
(𝜑 → ∀𝑥𝜑)       ((¬ 𝜑 ∧ ∃!𝑥𝜓) → ∃!𝑥(𝜑𝜓))
 
Theoremeuorv 2041* Introduce a disjunct into a unique existential quantifier. (Contributed by NM, 23-Mar-1995.)
((¬ 𝜑 ∧ ∃!𝑥𝜓) → ∃!𝑥(𝜑𝜓))
 
Theoremmo2n 2042* There is at most one of something which does not exist. (Contributed by Jim Kingdon, 2-Jul-2018.)
𝑦𝜑       (¬ ∃𝑥𝜑 → ∃𝑦𝑥(𝜑𝑥 = 𝑦))
 
Theoremmon 2043 There is at most one of something which does not exist. (Contributed by Jim Kingdon, 5-Jul-2018.)
(¬ ∃𝑥𝜑 → ∃*𝑥𝜑)
 
Theoremeuex 2044 Existential uniqueness implies existence. (Contributed by NM, 15-Sep-1993.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
(∃!𝑥𝜑 → ∃𝑥𝜑)
 
Theoremeumo0 2045* Existential uniqueness implies "at most one". (Contributed by NM, 8-Jul-1994.)
(𝜑 → ∀𝑦𝜑)       (∃!𝑥𝜑 → ∃𝑦𝑥(𝜑𝑥 = 𝑦))
 
Theoremeumo 2046 Existential uniqueness implies "at most one". (Contributed by NM, 23-Mar-1995.) (Proof rewritten by Jim Kingdon, 27-May-2018.)
(∃!𝑥𝜑 → ∃*𝑥𝜑)
 
Theoremeumoi 2047 "At most one" inferred from existential uniqueness. (Contributed by NM, 5-Apr-1995.)
∃!𝑥𝜑       ∃*𝑥𝜑
 
Theoremmobidh 2048 Formula-building rule for "at most one" quantifier (deduction form). (Contributed by NM, 8-Mar-1995.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃*𝑥𝜓 ↔ ∃*𝑥𝜒))
 
Theoremmobid 2049 Formula-building rule for "at most one" quantifier (deduction form). (Contributed by NM, 8-Mar-1995.)
𝑥𝜑    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃*𝑥𝜓 ↔ ∃*𝑥𝜒))
 
Theoremmobidv 2050* Formula-building rule for "at most one" quantifier (deduction form). (Contributed by Mario Carneiro, 7-Oct-2016.)
(𝜑 → (𝜓𝜒))       (𝜑 → (∃*𝑥𝜓 ↔ ∃*𝑥𝜒))
 
Theoremmobii 2051 Formula-building rule for "at most one" quantifier (inference form). (Contributed by NM, 9-Mar-1995.) (Revised by Mario Carneiro, 17-Oct-2016.)
(𝜓𝜒)       (∃*𝑥𝜓 ↔ ∃*𝑥𝜒)
 
Theoremhbmo1 2052 Bound-variable hypothesis builder for "at most one". (Contributed by NM, 8-Mar-1995.)
(∃*𝑥𝜑 → ∀𝑥∃*𝑥𝜑)
 
Theoremhbmo 2053 Bound-variable hypothesis builder for "at most one". (Contributed by NM, 9-Mar-1995.)
(𝜑 → ∀𝑥𝜑)       (∃*𝑦𝜑 → ∀𝑥∃*𝑦𝜑)
 
Theoremcbvmo 2054 Rule used to change bound variables, using implicit substitution. (Contributed by NM, 9-Mar-1995.) (Revised by Andrew Salmon, 8-Jun-2011.)
𝑦𝜑    &   𝑥𝜓    &   (𝑥 = 𝑦 → (𝜑𝜓))       (∃*𝑥𝜑 ↔ ∃*𝑦𝜓)
 
Theoremmo23 2055* An implication between two definitions of "there exists at most one." (Contributed by Jim Kingdon, 25-Jun-2018.)
𝑦𝜑       (∃𝑦𝑥(𝜑𝑥 = 𝑦) → ∀𝑥𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦))
 
Theoremmor 2056* Converse of mo23 2055 with an additional 𝑥𝜑 condition. (Contributed by Jim Kingdon, 25-Jun-2018.)
𝑦𝜑       (∃𝑥𝜑 → (∀𝑥𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦) → ∃𝑦𝑥(𝜑𝑥 = 𝑦)))
 
Theoremmodc 2057* Equivalent definitions of "there exists at most one," given decidable existence. (Contributed by Jim Kingdon, 1-Jul-2018.)
𝑦𝜑       (DECID𝑥𝜑 → (∃𝑦𝑥(𝜑𝑥 = 𝑦) ↔ ∀𝑥𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦)))
 
Theoremeu2 2058* An alternate way of defining existential uniqueness. Definition 6.10 of [TakeutiZaring] p. 26. (Contributed by NM, 8-Jul-1994.)
𝑦𝜑       (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∀𝑥𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦)))
 
Theoremeu3h 2059* An alternate way to express existential uniqueness. (Contributed by NM, 8-Jul-1994.) (New usage is discouraged.)
(𝜑 → ∀𝑦𝜑)       (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∃𝑦𝑥(𝜑𝑥 = 𝑦)))
 
Theoremeu3 2060* An alternate way to express existential uniqueness. (Contributed by NM, 8-Jul-1994.)
𝑦𝜑       (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∃𝑦𝑥(𝜑𝑥 = 𝑦)))
 
Theoremeu5 2061 Uniqueness in terms of "at most one". (Contributed by NM, 23-Mar-1995.) (Proof rewritten by Jim Kingdon, 27-May-2018.)
(∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∃*𝑥𝜑))
 
Theoremexmoeu2 2062 Existence implies "at most one" is equivalent to uniqueness. (Contributed by NM, 5-Apr-2004.)
(∃𝑥𝜑 → (∃*𝑥𝜑 ↔ ∃!𝑥𝜑))
 
Theoremmoabs 2063 Absorption of existence condition by "at most one". (Contributed by NM, 4-Nov-2002.)
(∃*𝑥𝜑 ↔ (∃𝑥𝜑 → ∃*𝑥𝜑))
 
Theoremexmodc 2064 If existence is decidable, something exists or at most one exists. (Contributed by Jim Kingdon, 30-Jun-2018.)
(DECID𝑥𝜑 → (∃𝑥𝜑 ∨ ∃*𝑥𝜑))
 
Theoremexmonim 2065 There is at most one of something which does not exist. Unlike exmodc 2064 there is no decidability condition. (Contributed by Jim Kingdon, 22-Sep-2018.)
(¬ ∃𝑥𝜑 → ∃*𝑥𝜑)
 
Theoremmo2r 2066* A condition which implies "at most one". (Contributed by Jim Kingdon, 2-Jul-2018.)
𝑦𝜑       (∃𝑦𝑥(𝜑𝑥 = 𝑦) → ∃*𝑥𝜑)
 
Theoremmo3h 2067* Alternate definition of "at most one". Definition of [BellMachover] p. 460, except that definition has the side condition that 𝑦 not occur in 𝜑 in place of our hypothesis. (Contributed by NM, 8-Mar-1995.) (New usage is discouraged.)
(𝜑 → ∀𝑦𝜑)       (∃*𝑥𝜑 ↔ ∀𝑥𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦))
 
Theoremmo3 2068* Alternate definition of "at most one". Definition of [BellMachover] p. 460, except that definition has the side condition that 𝑦 not occur in 𝜑 in place of our hypothesis. (Contributed by NM, 8-Mar-1995.)
𝑦𝜑       (∃*𝑥𝜑 ↔ ∀𝑥𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦))
 
Theoremmo2dc 2069* Alternate definition of "at most one" where existence is decidable. (Contributed by Jim Kingdon, 2-Jul-2018.)
𝑦𝜑       (DECID𝑥𝜑 → (∃*𝑥𝜑 ↔ ∃𝑦𝑥(𝜑𝑥 = 𝑦)))
 
Theoremeuan 2070 Introduction of a conjunct into unique existential quantifier. (Contributed by NM, 19-Feb-2005.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
(𝜑 → ∀𝑥𝜑)       (∃!𝑥(𝜑𝜓) ↔ (𝜑 ∧ ∃!𝑥𝜓))
 
Theoremeuanv 2071* Introduction of a conjunct into unique existential quantifier. (Contributed by NM, 23-Mar-1995.)
(∃!𝑥(𝜑𝜓) ↔ (𝜑 ∧ ∃!𝑥𝜓))
 
Theoremeuor2 2072 Introduce or eliminate a disjunct in a unique existential quantifier. (Contributed by NM, 21-Oct-2005.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
(¬ ∃𝑥𝜑 → (∃!𝑥(𝜑𝜓) ↔ ∃!𝑥𝜓))
 
Theoremsbmo 2073* Substitution into "at most one". (Contributed by Jeff Madsen, 2-Sep-2009.)
([𝑦 / 𝑥]∃*𝑧𝜑 ↔ ∃*𝑧[𝑦 / 𝑥]𝜑)
 
Theoremmo4f 2074* "At most one" expressed using implicit substitution. (Contributed by NM, 10-Apr-2004.)
𝑥𝜓    &   (𝑥 = 𝑦 → (𝜑𝜓))       (∃*𝑥𝜑 ↔ ∀𝑥𝑦((𝜑𝜓) → 𝑥 = 𝑦))
 
Theoremmo4 2075* "At most one" expressed using implicit substitution. (Contributed by NM, 26-Jul-1995.)
(𝑥 = 𝑦 → (𝜑𝜓))       (∃*𝑥𝜑 ↔ ∀𝑥𝑦((𝜑𝜓) → 𝑥 = 𝑦))
 
Theoremeu4 2076* Uniqueness using implicit substitution. (Contributed by NM, 26-Jul-1995.)
(𝑥 = 𝑦 → (𝜑𝜓))       (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∀𝑥𝑦((𝜑𝜓) → 𝑥 = 𝑦)))
 
Theoremexmoeudc 2077 Existence in terms of "at most one" and uniqueness. (Contributed by Jim Kingdon, 3-Jul-2018.)
(DECID𝑥𝜑 → (∃𝑥𝜑 ↔ (∃*𝑥𝜑 → ∃!𝑥𝜑)))
 
Theoremmoim 2078 "At most one" is preserved through implication (notice wff reversal). (Contributed by NM, 22-Apr-1995.)
(∀𝑥(𝜑𝜓) → (∃*𝑥𝜓 → ∃*𝑥𝜑))
 
Theoremmoimi 2079 "At most one" is preserved through implication (notice wff reversal). (Contributed by NM, 15-Feb-2006.)
(𝜑𝜓)       (∃*𝑥𝜓 → ∃*𝑥𝜑)
 
Theoremmoimv 2080* Move antecedent outside of "at most one". (Contributed by NM, 28-Jul-1995.)
(∃*𝑥(𝜑𝜓) → (𝜑 → ∃*𝑥𝜓))
 
Theoremeuimmo 2081 Uniqueness implies "at most one" through implication. (Contributed by NM, 22-Apr-1995.)
(∀𝑥(𝜑𝜓) → (∃!𝑥𝜓 → ∃*𝑥𝜑))
 
Theoremeuim 2082 Add existential unique existential quantifiers to an implication. Note the reversed implication in the antecedent. (Contributed by NM, 19-Oct-2005.) (Proof shortened by Andrew Salmon, 14-Jun-2011.)
((∃𝑥𝜑 ∧ ∀𝑥(𝜑𝜓)) → (∃!𝑥𝜓 → ∃!𝑥𝜑))
 
Theoremmoan 2083 "At most one" is still the case when a conjunct is added. (Contributed by NM, 22-Apr-1995.)
(∃*𝑥𝜑 → ∃*𝑥(𝜓𝜑))
 
Theoremmoani 2084 "At most one" is still true when a conjunct is added. (Contributed by NM, 9-Mar-1995.)
∃*𝑥𝜑       ∃*𝑥(𝜓𝜑)
 
Theoremmoor 2085 "At most one" is still the case when a disjunct is removed. (Contributed by NM, 5-Apr-2004.)
(∃*𝑥(𝜑𝜓) → ∃*𝑥𝜑)
 
Theoremmooran1 2086 "At most one" imports disjunction to conjunction. (Contributed by NM, 5-Apr-2004.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
((∃*𝑥𝜑 ∨ ∃*𝑥𝜓) → ∃*𝑥(𝜑𝜓))
 
Theoremmooran2 2087 "At most one" exports disjunction to conjunction. (Contributed by NM, 5-Apr-2004.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
(∃*𝑥(𝜑𝜓) → (∃*𝑥𝜑 ∧ ∃*𝑥𝜓))
 
Theoremmoanim 2088 Introduction of a conjunct into at-most-one quantifier. (Contributed by NM, 3-Dec-2001.)
𝑥𝜑       (∃*𝑥(𝜑𝜓) ↔ (𝜑 → ∃*𝑥𝜓))
 
Theoremmoanimv 2089* Introduction of a conjunct into at-most-one quantifier. (Contributed by NM, 23-Mar-1995.)
(∃*𝑥(𝜑𝜓) ↔ (𝜑 → ∃*𝑥𝜓))
 
Theoremmoaneu 2090 Nested at-most-one and unique existential quantifiers. (Contributed by NM, 25-Jan-2006.)
∃*𝑥(𝜑 ∧ ∃!𝑥𝜑)
 
Theoremmoanmo 2091 Nested at-most-one quantifiers. (Contributed by NM, 25-Jan-2006.)
∃*𝑥(𝜑 ∧ ∃*𝑥𝜑)
 
Theoremmopick 2092 "At most one" picks a variable value, eliminating an existential quantifier. (Contributed by NM, 27-Jan-1997.)
((∃*𝑥𝜑 ∧ ∃𝑥(𝜑𝜓)) → (𝜑𝜓))
 
Theoremeupick 2093 Existential uniqueness "picks" a variable value for which another wff is true. If there is only one thing 𝑥 such that 𝜑 is true, and there is also an 𝑥 (actually the same one) such that 𝜑 and 𝜓 are both true, then 𝜑 implies 𝜓 regardless of 𝑥. This theorem can be useful for eliminating existential quantifiers in a hypothesis. Compare Theorem *14.26 in [WhiteheadRussell] p. 192. (Contributed by NM, 10-Jul-1994.)
((∃!𝑥𝜑 ∧ ∃𝑥(𝜑𝜓)) → (𝜑𝜓))
 
Theoremeupicka 2094 Version of eupick 2093 with closed formulas. (Contributed by NM, 6-Sep-2008.)
((∃!𝑥𝜑 ∧ ∃𝑥(𝜑𝜓)) → ∀𝑥(𝜑𝜓))
 
Theoremeupickb 2095 Existential uniqueness "pick" showing wff equivalence. (Contributed by NM, 25-Nov-1994.)
((∃!𝑥𝜑 ∧ ∃!𝑥𝜓 ∧ ∃𝑥(𝜑𝜓)) → (𝜑𝜓))
 
Theoremeupickbi 2096 Theorem *14.26 in [WhiteheadRussell] p. 192. (Contributed by Andrew Salmon, 11-Jul-2011.)
(∃!𝑥𝜑 → (∃𝑥(𝜑𝜓) ↔ ∀𝑥(𝜑𝜓)))
 
Theoremmopick2 2097 "At most one" can show the existence of a common value. In this case we can infer existence of conjunction from a conjunction of existence, and it is one way to achieve the converse of 19.40 1619. (Contributed by NM, 5-Apr-2004.) (Proof shortened by Andrew Salmon, 9-Jul-2011.)
((∃*𝑥𝜑 ∧ ∃𝑥(𝜑𝜓) ∧ ∃𝑥(𝜑𝜒)) → ∃𝑥(𝜑𝜓𝜒))
 
Theoremmoexexdc 2098 "At most one" double quantification. (Contributed by Jim Kingdon, 5-Jul-2018.)
𝑦𝜑       (DECID𝑥𝜑 → ((∃*𝑥𝜑 ∧ ∀𝑥∃*𝑦𝜓) → ∃*𝑦𝑥(𝜑𝜓)))
 
Theoremeuexex 2099 Existential uniqueness and "at most one" double quantification. (Contributed by Jim Kingdon, 28-Dec-2018.)
𝑦𝜑       ((∃!𝑥𝜑 ∧ ∀𝑥∃*𝑦𝜓) → ∃*𝑦𝑥(𝜑𝜓))
 
Theorem2moex 2100 Double quantification with "at most one". (Contributed by NM, 3-Dec-2001.)
(∃*𝑥𝑦𝜑 → ∀𝑦∃*𝑥𝜑)
    < 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-13960
  Copyright terms: Public domain < Previous  Next >