HomeHome Intuitionistic Logic Explorer
Theorem List (p. 9 of 133)
< 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 - 801-900   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theorempm2.82 801 Theorem *2.82 of [WhiteheadRussell] p. 108. (Contributed by NM, 3-Jan-2005.)
(((𝜑𝜓) ∨ 𝜒) → (((𝜑 ∨ ¬ 𝜒) ∨ 𝜃) → ((𝜑𝜓) ∨ 𝜃)))
 
Theorempm3.2ni 802 Infer negated disjunction of negated premises. (Contributed by NM, 4-Apr-1995.)
¬ 𝜑    &    ¬ 𝜓        ¬ (𝜑𝜓)
 
Theoremorabs 803 Absorption of redundant internal disjunct. Compare Theorem *4.45 of [WhiteheadRussell] p. 119. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 28-Feb-2014.)
(𝜑 ↔ ((𝜑𝜓) ∧ 𝜑))
 
Theoremoranabs 804 Absorb a disjunct into a conjunct. (Contributed by Roy F. Longton, 23-Jun-2005.) (Proof shortened by Wolf Lammen, 10-Nov-2013.)
(((𝜑 ∨ ¬ 𝜓) ∧ 𝜓) ↔ (𝜑𝜓))
 
Theoremordi 805 Distributive law for disjunction. Theorem *4.41 of [WhiteheadRussell] p. 119. (Contributed by NM, 5-Aug-1993.) (Revised by Mario Carneiro, 31-Jan-2015.)
((𝜑 ∨ (𝜓𝜒)) ↔ ((𝜑𝜓) ∧ (𝜑𝜒)))
 
Theoremordir 806 Distributive law for disjunction. (Contributed by NM, 12-Aug-1994.)
(((𝜑𝜓) ∨ 𝜒) ↔ ((𝜑𝜒) ∧ (𝜓𝜒)))
 
Theoremandi 807 Distributive law for conjunction. Theorem *4.4 of [WhiteheadRussell] p. 118. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 5-Jan-2013.)
((𝜑 ∧ (𝜓𝜒)) ↔ ((𝜑𝜓) ∨ (𝜑𝜒)))
 
Theoremandir 808 Distributive law for conjunction. (Contributed by NM, 12-Aug-1994.)
(((𝜑𝜓) ∧ 𝜒) ↔ ((𝜑𝜒) ∨ (𝜓𝜒)))
 
Theoremorddi 809 Double distributive law for disjunction. (Contributed by NM, 12-Aug-1994.)
(((𝜑𝜓) ∨ (𝜒𝜃)) ↔ (((𝜑𝜒) ∧ (𝜑𝜃)) ∧ ((𝜓𝜒) ∧ (𝜓𝜃))))
 
Theoremanddi 810 Double distributive law for conjunction. (Contributed by NM, 12-Aug-1994.)
(((𝜑𝜓) ∧ (𝜒𝜃)) ↔ (((𝜑𝜒) ∨ (𝜑𝜃)) ∨ ((𝜓𝜒) ∨ (𝜓𝜃))))
 
Theorempm4.39 811 Theorem *4.39 of [WhiteheadRussell] p. 118. (Contributed by NM, 3-Jan-2005.)
(((𝜑𝜒) ∧ (𝜓𝜃)) → ((𝜑𝜓) ↔ (𝜒𝜃)))
 
Theorempm4.72 812 Implication in terms of biconditional and disjunction. Theorem *4.72 of [WhiteheadRussell] p. 121. (Contributed by NM, 30-Aug-1993.) (Proof shortened by Wolf Lammen, 30-Jan-2013.)
((𝜑𝜓) ↔ (𝜓 ↔ (𝜑𝜓)))
 
Theorempm5.16 813 Theorem *5.16 of [WhiteheadRussell] p. 124. (Contributed by NM, 3-Jan-2005.) (Revised by Mario Carneiro, 31-Jan-2015.)
¬ ((𝜑𝜓) ∧ (𝜑 ↔ ¬ 𝜓))
 
Theorembiort 814 A wff is disjoined with truth is true. (Contributed by NM, 23-May-1999.)
(𝜑 → (𝜑 ↔ (𝜑𝜓)))
 
1.2.7  Stable propositions
 
Syntaxwstab 815 Extend wff definition to include stability.
wff STAB 𝜑
 
Definitiondf-stab 816 Propositions where a double-negative can be removed are called stable. See Chapter 2 [Moschovakis] p. 2.

Our notation for stability is a connective STAB which we place before the formula in question. For example, STAB 𝑥 = 𝑦 corresponds to "𝑥 = 𝑦 is stable".

(Contributed by David A. Wheeler, 13-Aug-2018.)

(STAB 𝜑 ↔ (¬ ¬ 𝜑𝜑))
 
Theoremstbid 817 The equivalent of a stable proposition is stable. (Contributed by Jim Kingdon, 12-Aug-2022.)
(𝜑 → (𝜓𝜒))       (𝜑 → (STAB 𝜓STAB 𝜒))
 
Theoremstabnot 818 Every negated formula is stable. (Contributed by David A. Wheeler, 13-Aug-2018.)
STAB ¬ 𝜑
 
1.2.8  Decidable propositions
 
Syntaxwdc 819 Extend wff definition to include decidability.
wff DECID 𝜑
 
Definitiondf-dc 820 Propositions which are known to be true or false are called decidable. The (classical) Law of the Excluded Middle corresponds to the principle that all propositions are decidable, but even given intuitionistic logic, particular kinds of propositions may be decidable (for example, the proposition that two natural numbers are equal will be decidable under most sets of axioms).

Our notation for decidability is a connective DECID which we place before the formula in question. For example, DECID 𝑥 = 𝑦 corresponds to "𝑥 = 𝑦 is decidable".

We could transform intuitionistic logic to classical logic by adding unconditional forms of condc 838, exmiddc 821, peircedc 899, or notnotrdc 828, any of which would correspond to the assertion that all propositions are decidable.

(Contributed by Jim Kingdon, 11-Mar-2018.)

(DECID 𝜑 ↔ (𝜑 ∨ ¬ 𝜑))
 
Theoremexmiddc 821 Law of excluded middle, for a decidable proposition. The law of the excluded middle is also called the principle of tertium non datur. Theorem *2.11 of [WhiteheadRussell] p. 101. It says that something is either true or not true; there are no in-between values of truth. The key way in which intuitionistic logic differs from classical logic is that intuitionistic logic says that excluded middle only holds for some propositions, and classical logic says that it holds for all propositions. (Contributed by Jim Kingdon, 12-May-2018.)
(DECID 𝜑 → (𝜑 ∨ ¬ 𝜑))
 
Theorempm2.1dc 822 Commuted law of the excluded middle for a decidable proposition. Based on theorem *2.1 of [WhiteheadRussell] p. 101. (Contributed by Jim Kingdon, 25-Mar-2018.)
(DECID 𝜑 → (¬ 𝜑𝜑))
 
Theoremdcbid 823 Equivalence property for decidability. Deduction form. (Contributed by Jim Kingdon, 7-Sep-2019.)
(𝜑 → (𝜓𝜒))       (𝜑 → (DECID 𝜓DECID 𝜒))
 
Theoremdcbiit 824 Equivalence property for decidability. Closed form. (Contributed by BJ, 27-Jan-2020.)
((𝜑𝜓) → (DECID 𝜑DECID 𝜓))
 
Theoremdcbii 825 Equivalence property for decidability. Inference form. (Contributed by Jim Kingdon, 28-Mar-2018.)
(𝜑𝜓)       (DECID 𝜑DECID 𝜓)
 
Theoremdcim 826 An implication between two decidable propositions is decidable. (Contributed by Jim Kingdon, 28-Mar-2018.)
(DECID 𝜑 → (DECID 𝜓DECID (𝜑𝜓)))
 
Theoremdcn 827 The negation of a decidable proposition is decidable. The converse need not hold, but does hold for negated propositions, see dcnn 833. (Contributed by Jim Kingdon, 25-Mar-2018.)
(DECID 𝜑DECID ¬ 𝜑)
 
Theoremnotnotrdc 828 Double negation elimination for a decidable proposition. The converse, notnot 618, holds for all propositions, not just decidable ones. This is Theorem *2.14 of [WhiteheadRussell] p. 102, but with a decidability condition added. (Contributed by Jim Kingdon, 11-Mar-2018.)
(DECID 𝜑 → (¬ ¬ 𝜑𝜑))
 
Theoremdcstab 829 Decidability implies stability. The converse need not hold. (Contributed by David A. Wheeler, 13-Aug-2018.)
(DECID 𝜑STAB 𝜑)
 
Theoremstdcndc 830 A formula is decidable if and only if its negation is decidable and it is stable (that is, it is testable and stable). (Contributed by David A. Wheeler, 13-Aug-2018.) (Proof shortened by BJ, 28-Oct-2023.)
((STAB 𝜑DECID ¬ 𝜑) ↔ DECID 𝜑)
 
TheoremstdcndcOLD 831 Obsolete version of stdcndc 830 as of 28-Oct-2023. (Contributed by David A. Wheeler, 13-Aug-2018.) (Proof modification is discouraged.) (New usage is discouraged.)
((STAB 𝜑DECID ¬ 𝜑) ↔ DECID 𝜑)
 
Theoremstdcn 832 A formula is stable if and only if the decidability of its negation implies its decidability. Note that the right-hand side of this biconditional is the converse of dcn 827. (Contributed by BJ, 18-Nov-2023.)
(STAB 𝜑 ↔ (DECID ¬ 𝜑DECID 𝜑))
 
Theoremdcnn 833 Decidability of the negation of a proposition is equivalent to decidability of its double negation. See also dcn 827. The relation between dcn 827 and dcnn 833 is analogous to that between notnot 618 and notnotnot 623 (and directly stems from it). Using the notion of "testable proposition" (proposition whose negation is decidable), dcnn 833 means that a proposition is testable if and only if its negation is testable, and dcn 827 means that decidability implies testability. (Contributed by David A. Wheeler, 6-Dec-2018.) (Proof shortened by BJ, 25-Nov-2023.)
(DECID ¬ 𝜑DECID ¬ ¬ 𝜑)
 
TheoremdcnnOLD 834 Obsolete proof of dcnnOLD 834 as of 25-Nov-2023. (Contributed by David A. Wheeler, 6-Dec-2018.) (Proof modification is discouraged.) (New usage is discouraged.)
(DECID ¬ 𝜑DECID ¬ ¬ 𝜑)
 
Theoremnnexmid 835 Double negation of excluded middle. Intuitionistic logic refutes the negation of excluded middle (but does not prove excluded middle) for any formula. Can also be proved quickly from bj-nnor 12935 as in bj-nndcALT 12952. (Contributed by BJ, 9-Oct-2019.)
¬ ¬ (𝜑 ∨ ¬ 𝜑)
 
Theoremnndc 836 Double negation of decidability of a formula. Intuitionistic logic refutes undecidability (but does not prove decidability) of any formula. (Contributed by BJ, 9-Oct-2019.)
¬ ¬ DECID 𝜑
 
1.2.9  Theorems of decidable propositions

Many theorems of logic hold in intuitionistic logic just as they do in classical (non-inuitionistic) logic, for all propositions. Other theorems only hold for decidable propositions, such as the law of the excluded middle (df-dc 820), double negation elimination (notnotrdc 828), or contraposition (condc 838). Our goal is to prove all well-known or important classical theorems, but with suitable decidability conditions so that the proofs follow from intuitionistic axioms. This section is focused on such proofs, given decidability conditions.

Many theorems of this section actually hold for stable propositions (see df-stab 816). Decidable propositions are stable (dcstab 829), but the converse need not hold.

 
Theoremconst 837 Contraposition of a stable proposition. See comment of condc 838. (Contributed by BJ, 18-Nov-2023.)
(STAB 𝜑 → ((¬ 𝜑 → ¬ 𝜓) → (𝜓𝜑)))
 
Theoremcondc 838 Contraposition of a decidable proposition.

This theorem swaps or "transposes" the order of the consequents when negation is removed. An informal example is that the statement "if there are no clouds in the sky, it is not raining" implies the statement "if it is raining, there are clouds in the sky." This theorem (without the decidability condition, of course) is called Transp or "the principle of transposition" in Principia Mathematica (Theorem *2.17 of [WhiteheadRussell] p. 103) and is Axiom A3 of [Margaris] p. 49. We will also use the term "contraposition" for this principle, although the reader is advised that in the field of philosophical logic, "contraposition" has a different technical meaning.

(Contributed by Jim Kingdon, 13-Mar-2018.) (Proof shortened by BJ, 18-Nov-2023.)

(DECID 𝜑 → ((¬ 𝜑 → ¬ 𝜓) → (𝜓𝜑)))
 
TheoremcondcOLD 839 Obsolete proof of condc 838 as of 18-Nov-2023. (Contributed by Jim Kingdon, 13-Mar-2018.) (Proof modification is discouraged.) (New usage is discouraged.)
(DECID 𝜑 → ((¬ 𝜑 → ¬ 𝜓) → (𝜓𝜑)))
 
Theorempm2.18dc 840 Proof by contradiction for a decidable proposition. Based on Theorem *2.18 of [WhiteheadRussell] p. 103 (also called Clavius law). Intuitionistically it requires a decidability assumption, but compare with pm2.01 605 which does not. (Contributed by Jim Kingdon, 24-Mar-2018.)
(DECID 𝜑 → ((¬ 𝜑𝜑) → 𝜑))
 
Theoremcon1dc 841 Contraposition for a decidable proposition. Based on theorem *2.15 of [WhiteheadRussell] p. 102. (Contributed by Jim Kingdon, 29-Mar-2018.)
(DECID 𝜑 → ((¬ 𝜑𝜓) → (¬ 𝜓𝜑)))
 
Theoremcon4biddc 842 A contraposition deduction. (Contributed by Jim Kingdon, 18-May-2018.)
(𝜑 → (DECID 𝜓 → (DECID 𝜒 → (¬ 𝜓 ↔ ¬ 𝜒))))       (𝜑 → (DECID 𝜓 → (DECID 𝜒 → (𝜓𝜒))))
 
Theoremimpidc 843 An importation inference for a decidable consequent. (Contributed by Jim Kingdon, 30-Apr-2018.)
(DECID 𝜒 → (𝜑 → (𝜓𝜒)))       (DECID 𝜒 → (¬ (𝜑 → ¬ 𝜓) → 𝜒))
 
Theoremsimprimdc 844 Simplification given a decidable proposition. Similar to Theorem *3.27 (Simp) of [WhiteheadRussell] p. 112. (Contributed by Jim Kingdon, 30-Apr-2018.)
(DECID 𝜓 → (¬ (𝜑 → ¬ 𝜓) → 𝜓))
 
Theoremsimplimdc 845 Simplification for a decidable proposition. Similar to Theorem *3.26 (Simp) of [WhiteheadRussell] p. 112. (Contributed by Jim Kingdon, 29-Mar-2018.)
(DECID 𝜑 → (¬ (𝜑𝜓) → 𝜑))
 
Theorempm2.61ddc 846 Deduction eliminating a decidable antecedent. (Contributed by Jim Kingdon, 4-May-2018.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (¬ 𝜓𝜒))       (DECID 𝜓 → (𝜑𝜒))
 
Theorempm2.6dc 847 Case elimination for a decidable proposition. Based on theorem *2.6 of [WhiteheadRussell] p. 107. (Contributed by Jim Kingdon, 25-Mar-2018.)
(DECID 𝜑 → ((¬ 𝜑𝜓) → ((𝜑𝜓) → 𝜓)))
 
Theoremjadc 848 Inference forming an implication from the antecedents of two premises, where a decidable antecedent is negated. (Contributed by Jim Kingdon, 25-Mar-2018.)
(DECID 𝜑 → (¬ 𝜑𝜒))    &   (𝜓𝜒)       (DECID 𝜑 → ((𝜑𝜓) → 𝜒))
 
Theoremjaddc 849 Deduction forming an implication from the antecedents of two premises, where a decidable antecedent is negated. (Contributed by Jim Kingdon, 26-Mar-2018.)
(𝜑 → (DECID 𝜓 → (¬ 𝜓𝜃)))    &   (𝜑 → (𝜒𝜃))       (𝜑 → (DECID 𝜓 → ((𝜓𝜒) → 𝜃)))
 
Theorempm2.61dc 850 Case elimination for a decidable proposition. Theorem *2.61 of [WhiteheadRussell] p. 107 under a decidability condition. (Contributed by Jim Kingdon, 29-Mar-2018.)
(DECID 𝜑 → ((𝜑𝜓) → ((¬ 𝜑𝜓) → 𝜓)))
 
Theorempm2.5gdc 851 Negating an implication for a decidable antecedent. General instance of Theorem *2.5 of [WhiteheadRussell] p. 107 under a decidability condition. (Contributed by Jim Kingdon, 29-Mar-2018.)
(DECID 𝜑 → (¬ (𝜑𝜓) → (¬ 𝜑𝜒)))
 
Theorempm2.5dc 852 Negating an implication for a decidable antecedent. Theorem *2.5 of [WhiteheadRussell] p. 107 under a decidability condition. (Contributed by Jim Kingdon, 29-Mar-2018.)
(DECID 𝜑 → (¬ (𝜑𝜓) → (¬ 𝜑𝜓)))
 
Theorempm2.521gdc 853 A general instance of Theorem *2.521 of [WhiteheadRussell] p. 107, under a decidability condition. (Contributed by BJ, 28-Oct-2023.)
(DECID 𝜑 → (¬ (𝜑𝜓) → (𝜒𝜑)))
 
Theorempm2.521dc 854 Theorem *2.521 of [WhiteheadRussell] p. 107, but with an additional decidability condition. Note that by replacing in proof pm2.52 645 with conax1k 643, we obtain a proof of the more general instance where the last occurrence of 𝜑 is replaced with any 𝜒. (Contributed by Jim Kingdon, 5-May-2018.)
(DECID 𝜑 → (¬ (𝜑𝜓) → (𝜓𝜑)))
 
Theorempm2.521dcALT 855 Alternate proof of pm2.521dc 854. (Contributed by Jim Kingdon, 5-May-2018.) (Proof modification is discouraged.) (New usage is discouraged.)
(DECID 𝜑 → (¬ (𝜑𝜓) → (𝜓𝜑)))
 
Theoremcon34bdc 856 Contraposition. Theorem *4.1 of [WhiteheadRussell] p. 116, but for a decidable proposition. (Contributed by Jim Kingdon, 24-Apr-2018.)
(DECID 𝜓 → ((𝜑𝜓) ↔ (¬ 𝜓 → ¬ 𝜑)))
 
Theoremnotnotbdc 857 Double negation equivalence for a decidable proposition. Like Theorem *4.13 of [WhiteheadRussell] p. 117, but with a decidability antecendent. The forward direction, notnot 618, holds for all propositions, not just decidable ones. (Contributed by Jim Kingdon, 13-Mar-2018.)
(DECID 𝜑 → (𝜑 ↔ ¬ ¬ 𝜑))
 
Theoremcon1biimdc 858 Contraposition. (Contributed by Jim Kingdon, 4-Apr-2018.)
(DECID 𝜑 → ((¬ 𝜑𝜓) → (¬ 𝜓𝜑)))
 
Theoremcon1bidc 859 Contraposition. (Contributed by Jim Kingdon, 17-Apr-2018.)
(DECID 𝜑 → (DECID 𝜓 → ((¬ 𝜑𝜓) ↔ (¬ 𝜓𝜑))))
 
Theoremcon2bidc 860 Contraposition. (Contributed by Jim Kingdon, 17-Apr-2018.)
(DECID 𝜑 → (DECID 𝜓 → ((𝜑 ↔ ¬ 𝜓) ↔ (𝜓 ↔ ¬ 𝜑))))
 
Theoremcon1biddc 861 A contraposition deduction. (Contributed by Jim Kingdon, 4-Apr-2018.)
(𝜑 → (DECID 𝜓 → (¬ 𝜓𝜒)))       (𝜑 → (DECID 𝜓 → (¬ 𝜒𝜓)))
 
Theoremcon1biidc 862 A contraposition inference. (Contributed by Jim Kingdon, 15-Mar-2018.)
(DECID 𝜑 → (¬ 𝜑𝜓))       (DECID 𝜑 → (¬ 𝜓𝜑))
 
Theoremcon1bdc 863 Contraposition. Bidirectional version of con1dc 841. (Contributed by NM, 5-Aug-1993.)
(DECID 𝜑 → (DECID 𝜓 → ((¬ 𝜑𝜓) ↔ (¬ 𝜓𝜑))))
 
Theoremcon2biidc 864 A contraposition inference. (Contributed by Jim Kingdon, 15-Mar-2018.)
(DECID 𝜓 → (𝜑 ↔ ¬ 𝜓))       (DECID 𝜓 → (𝜓 ↔ ¬ 𝜑))
 
Theoremcon2biddc 865 A contraposition deduction. (Contributed by Jim Kingdon, 11-Apr-2018.)
(𝜑 → (DECID 𝜒 → (𝜓 ↔ ¬ 𝜒)))       (𝜑 → (DECID 𝜒 → (𝜒 ↔ ¬ 𝜓)))
 
Theoremcondandc 866 Proof by contradiction. This only holds for decidable propositions, as it is part of the family of theorems which assume ¬ 𝜓, derive a contradiction, and therefore conclude 𝜓. By contrast, assuming 𝜓, deriving a contradiction, and therefore concluding ¬ 𝜓, as in pm2.65 648, is valid for all propositions. (Contributed by Jim Kingdon, 13-May-2018.)
((𝜑 ∧ ¬ 𝜓) → 𝜒)    &   ((𝜑 ∧ ¬ 𝜓) → ¬ 𝜒)       (DECID 𝜓 → (𝜑𝜓))
 
Theorembijadc 867 Combine antecedents into a single biconditional. This inference is reminiscent of jadc 848. (Contributed by Jim Kingdon, 4-May-2018.)
(𝜑 → (𝜓𝜒))    &   𝜑 → (¬ 𝜓𝜒))       (DECID 𝜓 → ((𝜑𝜓) → 𝜒))
 
Theorempm5.18dc 868 Relationship between an equivalence and an equivalence with some negation, for decidable propositions. Based on theorem *5.18 of [WhiteheadRussell] p. 124. Given decidability, we can consider ¬ (𝜑 ↔ ¬ 𝜓) to represent "negated exclusive-or". (Contributed by Jim Kingdon, 4-Apr-2018.)
(DECID 𝜑 → (DECID 𝜓 → ((𝜑𝜓) ↔ ¬ (𝜑 ↔ ¬ 𝜓))))
 
Theoremdfandc 869 Definition of 'and' in terms of negation and implication, for decidable propositions. The forward direction holds for all propositions, and can (basically) be found at pm3.2im 626. (Contributed by Jim Kingdon, 30-Apr-2018.)
(DECID 𝜑 → (DECID 𝜓 → ((𝜑𝜓) ↔ ¬ (𝜑 → ¬ 𝜓))))
 
Theorempm2.13dc 870 A decidable proposition or its triple negation is true. Theorem *2.13 of [WhiteheadRussell] p. 101 with decidability condition added. (Contributed by Jim Kingdon, 13-May-2018.)
(DECID 𝜑 → (𝜑 ∨ ¬ ¬ ¬ 𝜑))
 
Theorempm4.63dc 871 Theorem *4.63 of [WhiteheadRussell] p. 120, for decidable propositions. (Contributed by Jim Kingdon, 1-May-2018.)
(DECID 𝜑 → (DECID 𝜓 → (¬ (𝜑 → ¬ 𝜓) ↔ (𝜑𝜓))))
 
Theorempm4.67dc 872 Theorem *4.67 of [WhiteheadRussell] p. 120, for decidable propositions. (Contributed by Jim Kingdon, 1-May-2018.)
(DECID 𝜑 → (DECID 𝜓 → (¬ (¬ 𝜑 → ¬ 𝜓) ↔ (¬ 𝜑𝜓))))
 
Theoremimanst 873 Express implication in terms of conjunction. Theorem 3.4(27) of [Stoll] p. 176. (Contributed by NM, 12-Mar-1993.) (Proof shortened by Wolf Lammen, 30-Oct-2012.)
(STAB 𝜓 → ((𝜑𝜓) ↔ ¬ (𝜑 ∧ ¬ 𝜓)))
 
Theoremimandc 874 Express implication in terms of conjunction. Theorem 3.4(27) of [Stoll] p. 176, with an added decidability condition. The forward direction, imanim 677, holds for all propositions, not just decidable ones. (Contributed by Jim Kingdon, 25-Apr-2018.)
(DECID 𝜓 → ((𝜑𝜓) ↔ ¬ (𝜑 ∧ ¬ 𝜓)))
 
Theorempm4.14dc 875 Theorem *4.14 of [WhiteheadRussell] p. 117, given a decidability condition. (Contributed by Jim Kingdon, 24-Apr-2018.)
(DECID 𝜒 → (((𝜑𝜓) → 𝜒) ↔ ((𝜑 ∧ ¬ 𝜒) → ¬ 𝜓)))
 
Theorempm2.54dc 876 Deriving disjunction from implication for a decidable proposition. Based on theorem *2.54 of [WhiteheadRussell] p. 107. The converse, pm2.53 711, holds whether the proposition is decidable or not. (Contributed by Jim Kingdon, 26-Mar-2018.)
(DECID 𝜑 → ((¬ 𝜑𝜓) → (𝜑𝜓)))
 
Theoremdfordc 877 Definition of disjunction in terms of negation and implication for a decidable proposition. Based on definition of [Margaris] p. 49. One direction, pm2.53 711, holds for all propositions, not just decidable ones. (Contributed by Jim Kingdon, 26-Mar-2018.)
(DECID 𝜑 → ((𝜑𝜓) ↔ (¬ 𝜑𝜓)))
 
Theorempm2.25dc 878 Elimination of disjunction based on a disjunction, for a decidable proposition. Based on theorem *2.25 of [WhiteheadRussell] p. 104. (Contributed by NM, 3-Jan-2005.)
(DECID 𝜑 → (𝜑 ∨ ((𝜑𝜓) → 𝜓)))
 
Theorempm2.68dc 879 Concluding disjunction from implication for a decidable proposition. Based on theorem *2.68 of [WhiteheadRussell] p. 108. Converse of pm2.62 737 and one half of dfor2dc 880. (Contributed by Jim Kingdon, 27-Mar-2018.)
(DECID 𝜑 → (((𝜑𝜓) → 𝜓) → (𝜑𝜓)))
 
Theoremdfor2dc 880 Disjunction expressed in terms of implication only, for a decidable proposition. Based on theorem *5.25 of [WhiteheadRussell] p. 124. (Contributed by Jim Kingdon, 27-Mar-2018.)
(DECID 𝜑 → ((𝜑𝜓) ↔ ((𝜑𝜓) → 𝜓)))
 
Theoremimimorbdc 881 Simplify an implication between implications, for a decidable proposition. (Contributed by Jim Kingdon, 18-Mar-2018.)
(DECID 𝜓 → (((𝜓𝜒) → (𝜑𝜒)) ↔ (𝜑 → (𝜓𝜒))))
 
Theoremimordc 882 Implication in terms of disjunction for a decidable proposition. Based on theorem *4.6 of [WhiteheadRussell] p. 120. The reverse direction, imorr 710, holds for all propositions. (Contributed by Jim Kingdon, 20-Apr-2018.)
(DECID 𝜑 → ((𝜑𝜓) ↔ (¬ 𝜑𝜓)))
 
Theorempm4.62dc 883 Implication in terms of disjunction. Like Theorem *4.62 of [WhiteheadRussell] p. 120, but for a decidable antecedent. (Contributed by Jim Kingdon, 21-Apr-2018.)
(DECID 𝜑 → ((𝜑 → ¬ 𝜓) ↔ (¬ 𝜑 ∨ ¬ 𝜓)))
 
Theoremianordc 884 Negated conjunction in terms of disjunction (DeMorgan's law). Theorem *4.51 of [WhiteheadRussell] p. 120, but where one proposition is decidable. The reverse direction, pm3.14 742, holds for all propositions, but the equivalence only holds where one proposition is decidable. (Contributed by Jim Kingdon, 21-Apr-2018.)
(DECID 𝜑 → (¬ (𝜑𝜓) ↔ (¬ 𝜑 ∨ ¬ 𝜓)))
 
Theorempm4.64dc 885 Theorem *4.64 of [WhiteheadRussell] p. 120, given a decidability condition. The reverse direction, pm2.53 711, holds for all propositions. (Contributed by Jim Kingdon, 2-May-2018.)
(DECID 𝜑 → ((¬ 𝜑𝜓) ↔ (𝜑𝜓)))
 
Theorempm4.66dc 886 Theorem *4.66 of [WhiteheadRussell] p. 120, given a decidability condition. (Contributed by Jim Kingdon, 2-May-2018.)
(DECID 𝜑 → ((¬ 𝜑 → ¬ 𝜓) ↔ (𝜑 ∨ ¬ 𝜓)))
 
Theorempm4.54dc 887 Theorem *4.54 of [WhiteheadRussell] p. 120, for decidable propositions. One form of DeMorgan's law. (Contributed by Jim Kingdon, 2-May-2018.)
(DECID 𝜑 → (DECID 𝜓 → ((¬ 𝜑𝜓) ↔ ¬ (𝜑 ∨ ¬ 𝜓))))
 
Theorempm4.79dc 888 Equivalence between a disjunction of two implications, and a conjunction and an implication. Based on theorem *4.79 of [WhiteheadRussell] p. 121 but with additional decidability antecedents. (Contributed by Jim Kingdon, 28-Mar-2018.)
(DECID 𝜑 → (DECID 𝜓 → (((𝜓𝜑) ∨ (𝜒𝜑)) ↔ ((𝜓𝜒) → 𝜑))))
 
Theorempm5.17dc 889 Two ways of stating exclusive-or which are equivalent for a decidable proposition. Based on theorem *5.17 of [WhiteheadRussell] p. 124. (Contributed by Jim Kingdon, 16-Apr-2018.)
(DECID 𝜓 → (((𝜑𝜓) ∧ ¬ (𝜑𝜓)) ↔ (𝜑 ↔ ¬ 𝜓)))
 
Theorempm2.85dc 890 Reverse distribution of disjunction over implication, given decidability. Based on theorem *2.85 of [WhiteheadRussell] p. 108. (Contributed by Jim Kingdon, 1-Apr-2018.)
(DECID 𝜑 → (((𝜑𝜓) → (𝜑𝜒)) → (𝜑 ∨ (𝜓𝜒))))
 
Theoremorimdidc 891 Disjunction distributes over implication. The forward direction, pm2.76 797, is valid intuitionistically. The reverse direction holds if 𝜑 is decidable, as can be seen at pm2.85dc 890. (Contributed by Jim Kingdon, 1-Apr-2018.)
(DECID 𝜑 → ((𝜑 ∨ (𝜓𝜒)) ↔ ((𝜑𝜓) → (𝜑𝜒))))
 
Theorempm2.26dc 892 Decidable proposition version of theorem *2.26 of [WhiteheadRussell] p. 104. (Contributed by Jim Kingdon, 20-Apr-2018.)
(DECID 𝜑 → (¬ 𝜑 ∨ ((𝜑𝜓) → 𝜓)))
 
Theorempm4.81dc 893 Theorem *4.81 of [WhiteheadRussell] p. 122, for decidable propositions. This one needs a decidability condition, but compare with pm4.8 696 which holds for all propositions. (Contributed by Jim Kingdon, 4-Jul-2018.)
(DECID 𝜑 → ((¬ 𝜑𝜑) ↔ 𝜑))
 
Theorempm5.11dc 894 A decidable proposition or its negation implies a second proposition. Based on theorem *5.11 of [WhiteheadRussell] p. 123. (Contributed by Jim Kingdon, 29-Mar-2018.)
(DECID 𝜑 → (DECID 𝜓 → ((𝜑𝜓) ∨ (¬ 𝜑𝜓))))
 
Theorempm5.12dc 895 Excluded middle with antecedents for a decidable consequent. Based on theorem *5.12 of [WhiteheadRussell] p. 123. (Contributed by Jim Kingdon, 30-Mar-2018.)
(DECID 𝜓 → ((𝜑𝜓) ∨ (𝜑 → ¬ 𝜓)))
 
Theorempm5.14dc 896 A decidable proposition is implied by or implies other propositions. Based on theorem *5.14 of [WhiteheadRussell] p. 123. (Contributed by Jim Kingdon, 30-Mar-2018.)
(DECID 𝜓 → ((𝜑𝜓) ∨ (𝜓𝜒)))
 
Theorempm5.13dc 897 An implication holds in at least one direction, where one proposition is decidable. Based on theorem *5.13 of [WhiteheadRussell] p. 123. (Contributed by Jim Kingdon, 30-Mar-2018.)
(DECID 𝜓 → ((𝜑𝜓) ∨ (𝜓𝜑)))
 
Theorempm5.55dc 898 A disjunction is equivalent to one of its disjuncts, given a decidable disjunct. Based on theorem *5.55 of [WhiteheadRussell] p. 125. (Contributed by Jim Kingdon, 30-Mar-2018.)
(DECID 𝜑 → (((𝜑𝜓) ↔ 𝜑) ∨ ((𝜑𝜓) ↔ 𝜓)))
 
Theorempeircedc 899 Peirce's theorem for a decidable proposition. This odd-looking theorem can be seen as an alternative to exmiddc 821, condc 838, or notnotrdc 828 in the sense of expressing the "difference" between an intuitionistic system of propositional calculus and a classical system. In intuitionistic logic, it only holds for decidable propositions. (Contributed by Jim Kingdon, 3-Jul-2018.)
(DECID 𝜑 → (((𝜑𝜓) → 𝜑) → 𝜑))
 
Theoremlooinvdc 900 The Inversion Axiom of the infinite-valued sentential logic (L-infinity) of Lukasiewicz, but where one of the propositions is decidable. Using dfor2dc 880, we can see that this expresses "disjunction commutes." Theorem *2.69 of [WhiteheadRussell] p. 108 (plus the decidability condition). (Contributed by NM, 12-Aug-2004.)
(DECID 𝜑 → (((𝜑𝜓) → 𝜓) → ((𝜓𝜑) → 𝜑)))
    < 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-800801-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-13239
  Copyright terms: Public domain < Previous  Next >