Home | 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 |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | hbsb4t 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.) |
⊢ (∀𝑥∀𝑧(𝜑 → ∀𝑧𝜑) → (¬ ∀𝑧 𝑧 = 𝑦 → ([𝑦 / 𝑥]𝜑 → ∀𝑧[𝑦 / 𝑥]𝜑))) | ||
Theorem | nfsb4t 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.) |
⊢ (∀𝑥Ⅎ𝑧𝜑 → (¬ ∀𝑧 𝑧 = 𝑦 → Ⅎ𝑧[𝑦 / 𝑥]𝜑)) | ||
Theorem | dvelimf 2003 | Version of dvelim 2005 without any variable restrictions. (Contributed by NM, 1-Oct-2002.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜓 → ∀𝑧𝜓) & ⊢ (𝑧 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (¬ ∀𝑥 𝑥 = 𝑦 → (𝜓 → ∀𝑥𝜓)) | ||
Theorem | dvelimdf 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.) |
⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑧𝜑 & ⊢ (𝜑 → Ⅎ𝑥𝜓) & ⊢ (𝜑 → Ⅎ𝑧𝜒) & ⊢ (𝜑 → (𝑧 = 𝑦 → (𝜓 ↔ 𝜒))) ⇒ ⊢ (𝜑 → (¬ ∀𝑥 𝑥 = 𝑦 → Ⅎ𝑥𝜒)) | ||
Theorem | dvelim 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.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝑧 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (¬ ∀𝑥 𝑥 = 𝑦 → (𝜓 → ∀𝑥𝜓)) | ||
Theorem | dvelimor 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.) |
⊢ Ⅎ𝑥𝜑 & ⊢ (𝑧 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∀𝑥 𝑥 = 𝑦 ∨ Ⅎ𝑥𝜓) | ||
Theorem | dveeq1 2007* | Quantifier introduction when one pair of variables is distinct. (Contributed by NM, 2-Jan-2002.) (Proof rewritten by Jim Kingdon, 19-Feb-2018.) |
⊢ (¬ ∀𝑥 𝑥 = 𝑦 → (𝑦 = 𝑧 → ∀𝑥 𝑦 = 𝑧)) | ||
Theorem | sbal2 2008* | Move quantifier in and out of substitution. (Contributed by NM, 2-Jan-2002.) |
⊢ (¬ ∀𝑥 𝑥 = 𝑦 → ([𝑧 / 𝑦]∀𝑥𝜑 ↔ ∀𝑥[𝑧 / 𝑦]𝜑)) | ||
Theorem | nfsb4or 2009 | A variable not free remains so after substitution with a distinct variable. (Contributed by Jim Kingdon, 11-May-2018.) |
⊢ Ⅎ𝑧𝜑 ⇒ ⊢ (∀𝑧 𝑧 = 𝑦 ∨ Ⅎ𝑧[𝑦 / 𝑥]𝜑) | ||
Theorem | nfd2 2010 | Deduce that 𝑥 is not free in 𝜓 in a context. (Contributed by Wolf Lammen, 16-Sep-2021.) |
⊢ (𝜑 → (∃𝑥𝜓 → ∀𝑥𝜓)) ⇒ ⊢ (𝜑 → Ⅎ𝑥𝜓) | ||
Theorem | hbe1a 2011 | Dual statement of hbe1 1483. (Contributed by Wolf Lammen, 15-Sep-2021.) |
⊢ (∃𝑥∀𝑥𝜑 → ∀𝑥𝜑) | ||
Theorem | nf5-1 2012 | One direction of nf5 . (Contributed by Wolf Lammen, 16-Sep-2021.) |
⊢ (∀𝑥(𝜑 → ∀𝑥𝜑) → Ⅎ𝑥𝜑) | ||
Theorem | nf5d 2013 | Deduce that 𝑥 is not free in 𝜓 in a context. (Contributed by Mario Carneiro, 24-Sep-2016.) |
⊢ Ⅎ𝑥𝜑 & ⊢ (𝜑 → (𝜓 → ∀𝑥𝜓)) ⇒ ⊢ (𝜑 → Ⅎ𝑥𝜓) | ||
Syntax | weu 2014 | Extend wff definition to include existential uniqueness ("there exists a unique 𝑥 such that 𝜑"). |
wff ∃!𝑥𝜑 | ||
Syntax | wmo 2015 | Extend wff definition to include uniqueness ("there exists at most one 𝑥 such that 𝜑"). |
wff ∃*𝑥𝜑 | ||
Theorem | eujust 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.) |
⊢ (∃𝑦∀𝑥(𝜑 ↔ 𝑥 = 𝑦) ↔ ∃𝑧∀𝑥(𝜑 ↔ 𝑥 = 𝑧)) | ||
Definition | df-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.) |
⊢ (∃!𝑥𝜑 ↔ ∃𝑦∀𝑥(𝜑 ↔ 𝑥 = 𝑦)) | ||
Definition | df-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.) |
⊢ (∃*𝑥𝜑 ↔ (∃𝑥𝜑 → ∃!𝑥𝜑)) | ||
Theorem | euf 2019* | A version of the existential uniqueness definition with a hypothesis instead of a distinct variable condition. (Contributed by NM, 12-Aug-1993.) |
⊢ (𝜑 → ∀𝑦𝜑) ⇒ ⊢ (∃!𝑥𝜑 ↔ ∃𝑦∀𝑥(𝜑 ↔ 𝑥 = 𝑦)) | ||
Theorem | eubidh 2020 | Formula-building rule for unique existential quantifier (deduction form). (Contributed by NM, 9-Jul-1994.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃!𝑥𝜓 ↔ ∃!𝑥𝜒)) | ||
Theorem | eubid 2021 | Formula-building rule for unique existential quantifier (deduction form). (Contributed by NM, 9-Jul-1994.) |
⊢ Ⅎ𝑥𝜑 & ⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃!𝑥𝜓 ↔ ∃!𝑥𝜒)) | ||
Theorem | eubidv 2022* | Formula-building rule for unique existential quantifier (deduction form). (Contributed by NM, 9-Jul-1994.) |
⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃!𝑥𝜓 ↔ ∃!𝑥𝜒)) | ||
Theorem | eubii 2023 | Introduce unique existential quantifier to both sides of an equivalence. (Contributed by NM, 9-Jul-1994.) (Revised by Mario Carneiro, 6-Oct-2016.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (∃!𝑥𝜑 ↔ ∃!𝑥𝜓) | ||
Theorem | hbeu1 2024 | Bound-variable hypothesis builder for uniqueness. (Contributed by NM, 9-Jul-1994.) |
⊢ (∃!𝑥𝜑 → ∀𝑥∃!𝑥𝜑) | ||
Theorem | nfeu1 2025 | Bound-variable hypothesis builder for uniqueness. (Contributed by NM, 9-Jul-1994.) (Revised by Mario Carneiro, 7-Oct-2016.) |
⊢ Ⅎ𝑥∃!𝑥𝜑 | ||
Theorem | nfmo1 2026 | Bound-variable hypothesis builder for "at most one". (Contributed by NM, 8-Mar-1995.) (Revised by Mario Carneiro, 7-Oct-2016.) |
⊢ Ⅎ𝑥∃*𝑥𝜑 | ||
Theorem | sb8eu 2027 | Variable substitution in unique existential quantifier. (Contributed by NM, 7-Aug-1994.) (Revised by Mario Carneiro, 7-Oct-2016.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃!𝑥𝜑 ↔ ∃!𝑦[𝑦 / 𝑥]𝜑) | ||
Theorem | sb8mo 2028 | Variable substitution for "at most one". (Contributed by Alexander van der Vekens, 17-Jun-2017.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃*𝑥𝜑 ↔ ∃*𝑦[𝑦 / 𝑥]𝜑) | ||
Theorem | nfeudv 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.) |
⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜑 → Ⅎ𝑥∃!𝑦𝜓) | ||
Theorem | nfeud 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.) |
⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜑 → Ⅎ𝑥∃!𝑦𝜓) | ||
Theorem | nfmod 2031 | Bound-variable hypothesis builder for "at most one". (Contributed by Mario Carneiro, 14-Nov-2016.) |
⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜑 → Ⅎ𝑥∃*𝑦𝜓) | ||
Theorem | nfeuv 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.) |
⊢ Ⅎ𝑥𝜑 ⇒ ⊢ Ⅎ𝑥∃!𝑦𝜑 | ||
Theorem | nfeu 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.) |
⊢ Ⅎ𝑥𝜑 ⇒ ⊢ Ⅎ𝑥∃!𝑦𝜑 | ||
Theorem | nfmo 2034 | Bound-variable hypothesis builder for "at most one". (Contributed by NM, 9-Mar-1995.) |
⊢ Ⅎ𝑥𝜑 ⇒ ⊢ Ⅎ𝑥∃*𝑦𝜑 | ||
Theorem | hbeu 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.) |
⊢ (𝜑 → ∀𝑥𝜑) ⇒ ⊢ (∃!𝑦𝜑 → ∀𝑥∃!𝑦𝜑) | ||
Theorem | hbeud 2036 | Deduction version of hbeu 2035. (Contributed by NM, 15-Feb-2013.) (Proof rewritten by Jim Kingdon, 25-May-2018.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → ∀𝑦𝜑) & ⊢ (𝜑 → (𝜓 → ∀𝑥𝜓)) ⇒ ⊢ (𝜑 → (∃!𝑦𝜓 → ∀𝑥∃!𝑦𝜓)) | ||
Theorem | sb8euh 2037 | Variable substitution in unique existential quantifier. (Contributed by NM, 7-Aug-1994.) (Revised by Andrew Salmon, 9-Jul-2011.) |
⊢ (𝜑 → ∀𝑦𝜑) ⇒ ⊢ (∃!𝑥𝜑 ↔ ∃!𝑦[𝑦 / 𝑥]𝜑) | ||
Theorem | cbveu 2038 | Rule used to change bound variables, using implicit substitution. (Contributed by NM, 25-Nov-1994.) (Revised by Mario Carneiro, 7-Oct-2016.) |
⊢ Ⅎ𝑦𝜑 & ⊢ Ⅎ𝑥𝜓 & ⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∃!𝑥𝜑 ↔ ∃!𝑦𝜓) | ||
Theorem | eu1 2039* | An alternate way to express uniqueness used by some authors. Exercise 2(b) of [Margaris] p. 110. (Contributed by NM, 20-Aug-1993.) |
⊢ (𝜑 → ∀𝑦𝜑) ⇒ ⊢ (∃!𝑥𝜑 ↔ ∃𝑥(𝜑 ∧ ∀𝑦([𝑦 / 𝑥]𝜑 → 𝑥 = 𝑦))) | ||
Theorem | euor 2040 | Introduce a disjunct into a unique existential quantifier. (Contributed by NM, 21-Oct-2005.) |
⊢ (𝜑 → ∀𝑥𝜑) ⇒ ⊢ ((¬ 𝜑 ∧ ∃!𝑥𝜓) → ∃!𝑥(𝜑 ∨ 𝜓)) | ||
Theorem | euorv 2041* | Introduce a disjunct into a unique existential quantifier. (Contributed by NM, 23-Mar-1995.) |
⊢ ((¬ 𝜑 ∧ ∃!𝑥𝜓) → ∃!𝑥(𝜑 ∨ 𝜓)) | ||
Theorem | mo2n 2042* | There is at most one of something which does not exist. (Contributed by Jim Kingdon, 2-Jul-2018.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (¬ ∃𝑥𝜑 → ∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦)) | ||
Theorem | mon 2043 | There is at most one of something which does not exist. (Contributed by Jim Kingdon, 5-Jul-2018.) |
⊢ (¬ ∃𝑥𝜑 → ∃*𝑥𝜑) | ||
Theorem | euex 2044 | Existential uniqueness implies existence. (Contributed by NM, 15-Sep-1993.) (Proof shortened by Andrew Salmon, 9-Jul-2011.) |
⊢ (∃!𝑥𝜑 → ∃𝑥𝜑) | ||
Theorem | eumo0 2045* | Existential uniqueness implies "at most one". (Contributed by NM, 8-Jul-1994.) |
⊢ (𝜑 → ∀𝑦𝜑) ⇒ ⊢ (∃!𝑥𝜑 → ∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦)) | ||
Theorem | eumo 2046 | Existential uniqueness implies "at most one". (Contributed by NM, 23-Mar-1995.) (Proof rewritten by Jim Kingdon, 27-May-2018.) |
⊢ (∃!𝑥𝜑 → ∃*𝑥𝜑) | ||
Theorem | eumoi 2047 | "At most one" inferred from existential uniqueness. (Contributed by NM, 5-Apr-1995.) |
⊢ ∃!𝑥𝜑 ⇒ ⊢ ∃*𝑥𝜑 | ||
Theorem | mobidh 2048 | Formula-building rule for "at most one" quantifier (deduction form). (Contributed by NM, 8-Mar-1995.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃*𝑥𝜓 ↔ ∃*𝑥𝜒)) | ||
Theorem | mobid 2049 | Formula-building rule for "at most one" quantifier (deduction form). (Contributed by NM, 8-Mar-1995.) |
⊢ Ⅎ𝑥𝜑 & ⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃*𝑥𝜓 ↔ ∃*𝑥𝜒)) | ||
Theorem | mobidv 2050* | Formula-building rule for "at most one" quantifier (deduction form). (Contributed by Mario Carneiro, 7-Oct-2016.) |
⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃*𝑥𝜓 ↔ ∃*𝑥𝜒)) | ||
Theorem | mobii 2051 | Formula-building rule for "at most one" quantifier (inference form). (Contributed by NM, 9-Mar-1995.) (Revised by Mario Carneiro, 17-Oct-2016.) |
⊢ (𝜓 ↔ 𝜒) ⇒ ⊢ (∃*𝑥𝜓 ↔ ∃*𝑥𝜒) | ||
Theorem | hbmo1 2052 | Bound-variable hypothesis builder for "at most one". (Contributed by NM, 8-Mar-1995.) |
⊢ (∃*𝑥𝜑 → ∀𝑥∃*𝑥𝜑) | ||
Theorem | hbmo 2053 | Bound-variable hypothesis builder for "at most one". (Contributed by NM, 9-Mar-1995.) |
⊢ (𝜑 → ∀𝑥𝜑) ⇒ ⊢ (∃*𝑦𝜑 → ∀𝑥∃*𝑦𝜑) | ||
Theorem | cbvmo 2054 | Rule used to change bound variables, using implicit substitution. (Contributed by NM, 9-Mar-1995.) (Revised by Andrew Salmon, 8-Jun-2011.) |
⊢ Ⅎ𝑦𝜑 & ⊢ Ⅎ𝑥𝜓 & ⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∃*𝑥𝜑 ↔ ∃*𝑦𝜓) | ||
Theorem | mo23 2055* | An implication between two definitions of "there exists at most one." (Contributed by Jim Kingdon, 25-Jun-2018.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦) → ∀𝑥∀𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦)) | ||
Theorem | mor 2056* | Converse of mo23 2055 with an additional ∃𝑥𝜑 condition. (Contributed by Jim Kingdon, 25-Jun-2018.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃𝑥𝜑 → (∀𝑥∀𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦) → ∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦))) | ||
Theorem | modc 2057* | Equivalent definitions of "there exists at most one," given decidable existence. (Contributed by Jim Kingdon, 1-Jul-2018.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (DECID ∃𝑥𝜑 → (∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦) ↔ ∀𝑥∀𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦))) | ||
Theorem | eu2 2058* | An alternate way of defining existential uniqueness. Definition 6.10 of [TakeutiZaring] p. 26. (Contributed by NM, 8-Jul-1994.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∀𝑥∀𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦))) | ||
Theorem | eu3h 2059* | An alternate way to express existential uniqueness. (Contributed by NM, 8-Jul-1994.) (New usage is discouraged.) |
⊢ (𝜑 → ∀𝑦𝜑) ⇒ ⊢ (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦))) | ||
Theorem | eu3 2060* | An alternate way to express existential uniqueness. (Contributed by NM, 8-Jul-1994.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦))) | ||
Theorem | eu5 2061 | Uniqueness in terms of "at most one". (Contributed by NM, 23-Mar-1995.) (Proof rewritten by Jim Kingdon, 27-May-2018.) |
⊢ (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∃*𝑥𝜑)) | ||
Theorem | exmoeu2 2062 | Existence implies "at most one" is equivalent to uniqueness. (Contributed by NM, 5-Apr-2004.) |
⊢ (∃𝑥𝜑 → (∃*𝑥𝜑 ↔ ∃!𝑥𝜑)) | ||
Theorem | moabs 2063 | Absorption of existence condition by "at most one". (Contributed by NM, 4-Nov-2002.) |
⊢ (∃*𝑥𝜑 ↔ (∃𝑥𝜑 → ∃*𝑥𝜑)) | ||
Theorem | exmodc 2064 | If existence is decidable, something exists or at most one exists. (Contributed by Jim Kingdon, 30-Jun-2018.) |
⊢ (DECID ∃𝑥𝜑 → (∃𝑥𝜑 ∨ ∃*𝑥𝜑)) | ||
Theorem | exmonim 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.) |
⊢ (¬ ∃𝑥𝜑 → ∃*𝑥𝜑) | ||
Theorem | mo2r 2066* | A condition which implies "at most one". (Contributed by Jim Kingdon, 2-Jul-2018.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦) → ∃*𝑥𝜑) | ||
Theorem | mo3h 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.) |
⊢ (𝜑 → ∀𝑦𝜑) ⇒ ⊢ (∃*𝑥𝜑 ↔ ∀𝑥∀𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦)) | ||
Theorem | mo3 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.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃*𝑥𝜑 ↔ ∀𝑥∀𝑦((𝜑 ∧ [𝑦 / 𝑥]𝜑) → 𝑥 = 𝑦)) | ||
Theorem | mo2dc 2069* | Alternate definition of "at most one" where existence is decidable. (Contributed by Jim Kingdon, 2-Jul-2018.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (DECID ∃𝑥𝜑 → (∃*𝑥𝜑 ↔ ∃𝑦∀𝑥(𝜑 → 𝑥 = 𝑦))) | ||
Theorem | euan 2070 | Introduction of a conjunct into unique existential quantifier. (Contributed by NM, 19-Feb-2005.) (Proof shortened by Andrew Salmon, 9-Jul-2011.) |
⊢ (𝜑 → ∀𝑥𝜑) ⇒ ⊢ (∃!𝑥(𝜑 ∧ 𝜓) ↔ (𝜑 ∧ ∃!𝑥𝜓)) | ||
Theorem | euanv 2071* | Introduction of a conjunct into unique existential quantifier. (Contributed by NM, 23-Mar-1995.) |
⊢ (∃!𝑥(𝜑 ∧ 𝜓) ↔ (𝜑 ∧ ∃!𝑥𝜓)) | ||
Theorem | euor2 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.) |
⊢ (¬ ∃𝑥𝜑 → (∃!𝑥(𝜑 ∨ 𝜓) ↔ ∃!𝑥𝜓)) | ||
Theorem | sbmo 2073* | Substitution into "at most one". (Contributed by Jeff Madsen, 2-Sep-2009.) |
⊢ ([𝑦 / 𝑥]∃*𝑧𝜑 ↔ ∃*𝑧[𝑦 / 𝑥]𝜑) | ||
Theorem | mo4f 2074* | "At most one" expressed using implicit substitution. (Contributed by NM, 10-Apr-2004.) |
⊢ Ⅎ𝑥𝜓 & ⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∃*𝑥𝜑 ↔ ∀𝑥∀𝑦((𝜑 ∧ 𝜓) → 𝑥 = 𝑦)) | ||
Theorem | mo4 2075* | "At most one" expressed using implicit substitution. (Contributed by NM, 26-Jul-1995.) |
⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∃*𝑥𝜑 ↔ ∀𝑥∀𝑦((𝜑 ∧ 𝜓) → 𝑥 = 𝑦)) | ||
Theorem | eu4 2076* | Uniqueness using implicit substitution. (Contributed by NM, 26-Jul-1995.) |
⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∃!𝑥𝜑 ↔ (∃𝑥𝜑 ∧ ∀𝑥∀𝑦((𝜑 ∧ 𝜓) → 𝑥 = 𝑦))) | ||
Theorem | exmoeudc 2077 | Existence in terms of "at most one" and uniqueness. (Contributed by Jim Kingdon, 3-Jul-2018.) |
⊢ (DECID ∃𝑥𝜑 → (∃𝑥𝜑 ↔ (∃*𝑥𝜑 → ∃!𝑥𝜑))) | ||
Theorem | moim 2078 | "At most one" is preserved through implication (notice wff reversal). (Contributed by NM, 22-Apr-1995.) |
⊢ (∀𝑥(𝜑 → 𝜓) → (∃*𝑥𝜓 → ∃*𝑥𝜑)) | ||
Theorem | moimi 2079 | "At most one" is preserved through implication (notice wff reversal). (Contributed by NM, 15-Feb-2006.) |
⊢ (𝜑 → 𝜓) ⇒ ⊢ (∃*𝑥𝜓 → ∃*𝑥𝜑) | ||
Theorem | moimv 2080* | Move antecedent outside of "at most one". (Contributed by NM, 28-Jul-1995.) |
⊢ (∃*𝑥(𝜑 → 𝜓) → (𝜑 → ∃*𝑥𝜓)) | ||
Theorem | euimmo 2081 | Uniqueness implies "at most one" through implication. (Contributed by NM, 22-Apr-1995.) |
⊢ (∀𝑥(𝜑 → 𝜓) → (∃!𝑥𝜓 → ∃*𝑥𝜑)) | ||
Theorem | euim 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.) |
⊢ ((∃𝑥𝜑 ∧ ∀𝑥(𝜑 → 𝜓)) → (∃!𝑥𝜓 → ∃!𝑥𝜑)) | ||
Theorem | moan 2083 | "At most one" is still the case when a conjunct is added. (Contributed by NM, 22-Apr-1995.) |
⊢ (∃*𝑥𝜑 → ∃*𝑥(𝜓 ∧ 𝜑)) | ||
Theorem | moani 2084 | "At most one" is still true when a conjunct is added. (Contributed by NM, 9-Mar-1995.) |
⊢ ∃*𝑥𝜑 ⇒ ⊢ ∃*𝑥(𝜓 ∧ 𝜑) | ||
Theorem | moor 2085 | "At most one" is still the case when a disjunct is removed. (Contributed by NM, 5-Apr-2004.) |
⊢ (∃*𝑥(𝜑 ∨ 𝜓) → ∃*𝑥𝜑) | ||
Theorem | mooran1 2086 | "At most one" imports disjunction to conjunction. (Contributed by NM, 5-Apr-2004.) (Proof shortened by Andrew Salmon, 9-Jul-2011.) |
⊢ ((∃*𝑥𝜑 ∨ ∃*𝑥𝜓) → ∃*𝑥(𝜑 ∧ 𝜓)) | ||
Theorem | mooran2 2087 | "At most one" exports disjunction to conjunction. (Contributed by NM, 5-Apr-2004.) (Proof shortened by Andrew Salmon, 9-Jul-2011.) |
⊢ (∃*𝑥(𝜑 ∨ 𝜓) → (∃*𝑥𝜑 ∧ ∃*𝑥𝜓)) | ||
Theorem | moanim 2088 | Introduction of a conjunct into at-most-one quantifier. (Contributed by NM, 3-Dec-2001.) |
⊢ Ⅎ𝑥𝜑 ⇒ ⊢ (∃*𝑥(𝜑 ∧ 𝜓) ↔ (𝜑 → ∃*𝑥𝜓)) | ||
Theorem | moanimv 2089* | Introduction of a conjunct into at-most-one quantifier. (Contributed by NM, 23-Mar-1995.) |
⊢ (∃*𝑥(𝜑 ∧ 𝜓) ↔ (𝜑 → ∃*𝑥𝜓)) | ||
Theorem | moaneu 2090 | Nested at-most-one and unique existential quantifiers. (Contributed by NM, 25-Jan-2006.) |
⊢ ∃*𝑥(𝜑 ∧ ∃!𝑥𝜑) | ||
Theorem | moanmo 2091 | Nested at-most-one quantifiers. (Contributed by NM, 25-Jan-2006.) |
⊢ ∃*𝑥(𝜑 ∧ ∃*𝑥𝜑) | ||
Theorem | mopick 2092 | "At most one" picks a variable value, eliminating an existential quantifier. (Contributed by NM, 27-Jan-1997.) |
⊢ ((∃*𝑥𝜑 ∧ ∃𝑥(𝜑 ∧ 𝜓)) → (𝜑 → 𝜓)) | ||
Theorem | eupick 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.) |
⊢ ((∃!𝑥𝜑 ∧ ∃𝑥(𝜑 ∧ 𝜓)) → (𝜑 → 𝜓)) | ||
Theorem | eupicka 2094 | Version of eupick 2093 with closed formulas. (Contributed by NM, 6-Sep-2008.) |
⊢ ((∃!𝑥𝜑 ∧ ∃𝑥(𝜑 ∧ 𝜓)) → ∀𝑥(𝜑 → 𝜓)) | ||
Theorem | eupickb 2095 | Existential uniqueness "pick" showing wff equivalence. (Contributed by NM, 25-Nov-1994.) |
⊢ ((∃!𝑥𝜑 ∧ ∃!𝑥𝜓 ∧ ∃𝑥(𝜑 ∧ 𝜓)) → (𝜑 ↔ 𝜓)) | ||
Theorem | eupickbi 2096 | Theorem *14.26 in [WhiteheadRussell] p. 192. (Contributed by Andrew Salmon, 11-Jul-2011.) |
⊢ (∃!𝑥𝜑 → (∃𝑥(𝜑 ∧ 𝜓) ↔ ∀𝑥(𝜑 → 𝜓))) | ||
Theorem | mopick2 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.) |
⊢ ((∃*𝑥𝜑 ∧ ∃𝑥(𝜑 ∧ 𝜓) ∧ ∃𝑥(𝜑 ∧ 𝜒)) → ∃𝑥(𝜑 ∧ 𝜓 ∧ 𝜒)) | ||
Theorem | moexexdc 2098 | "At most one" double quantification. (Contributed by Jim Kingdon, 5-Jul-2018.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (DECID ∃𝑥𝜑 → ((∃*𝑥𝜑 ∧ ∀𝑥∃*𝑦𝜓) → ∃*𝑦∃𝑥(𝜑 ∧ 𝜓))) | ||
Theorem | euexex 2099 | Existential uniqueness and "at most one" double quantification. (Contributed by Jim Kingdon, 28-Dec-2018.) |
⊢ Ⅎ𝑦𝜑 ⇒ ⊢ ((∃!𝑥𝜑 ∧ ∀𝑥∃*𝑦𝜓) → ∃*𝑦∃𝑥(𝜑 ∧ 𝜓)) | ||
Theorem | 2moex 2100 | Double quantification with "at most one". (Contributed by NM, 3-Dec-2001.) |
⊢ (∃*𝑥∃𝑦𝜑 → ∀𝑦∃*𝑥𝜑) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |