Home | Intuitionistic Logic Explorer Theorem List (p. 9 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 | pm2.81 801 | Theorem *2.81 of [WhiteheadRussell] p. 108. (Contributed by NM, 3-Jan-2005.) |
⊢ ((𝜓 → (𝜒 → 𝜃)) → ((𝜑 ∨ 𝜓) → ((𝜑 ∨ 𝜒) → (𝜑 ∨ 𝜃)))) | ||
Theorem | pm2.82 802 | Theorem *2.82 of [WhiteheadRussell] p. 108. (Contributed by NM, 3-Jan-2005.) |
⊢ (((𝜑 ∨ 𝜓) ∨ 𝜒) → (((𝜑 ∨ ¬ 𝜒) ∨ 𝜃) → ((𝜑 ∨ 𝜓) ∨ 𝜃))) | ||
Theorem | pm3.2ni 803 | Infer negated disjunction of negated premises. (Contributed by NM, 4-Apr-1995.) |
⊢ ¬ 𝜑 & ⊢ ¬ 𝜓 ⇒ ⊢ ¬ (𝜑 ∨ 𝜓) | ||
Theorem | orabs 804 | 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.) |
⊢ (𝜑 ↔ ((𝜑 ∨ 𝜓) ∧ 𝜑)) | ||
Theorem | oranabs 805 | Absorb a disjunct into a conjunct. (Contributed by Roy F. Longton, 23-Jun-2005.) (Proof shortened by Wolf Lammen, 10-Nov-2013.) |
⊢ (((𝜑 ∨ ¬ 𝜓) ∧ 𝜓) ↔ (𝜑 ∧ 𝜓)) | ||
Theorem | ordi 806 | Distributive law for disjunction. Theorem *4.41 of [WhiteheadRussell] p. 119. (Contributed by NM, 5-Aug-1993.) (Revised by Mario Carneiro, 31-Jan-2015.) |
⊢ ((𝜑 ∨ (𝜓 ∧ 𝜒)) ↔ ((𝜑 ∨ 𝜓) ∧ (𝜑 ∨ 𝜒))) | ||
Theorem | ordir 807 | Distributive law for disjunction. (Contributed by NM, 12-Aug-1994.) |
⊢ (((𝜑 ∧ 𝜓) ∨ 𝜒) ↔ ((𝜑 ∨ 𝜒) ∧ (𝜓 ∨ 𝜒))) | ||
Theorem | andi 808 | 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.) |
⊢ ((𝜑 ∧ (𝜓 ∨ 𝜒)) ↔ ((𝜑 ∧ 𝜓) ∨ (𝜑 ∧ 𝜒))) | ||
Theorem | andir 809 | Distributive law for conjunction. (Contributed by NM, 12-Aug-1994.) |
⊢ (((𝜑 ∨ 𝜓) ∧ 𝜒) ↔ ((𝜑 ∧ 𝜒) ∨ (𝜓 ∧ 𝜒))) | ||
Theorem | orddi 810 | Double distributive law for disjunction. (Contributed by NM, 12-Aug-1994.) |
⊢ (((𝜑 ∧ 𝜓) ∨ (𝜒 ∧ 𝜃)) ↔ (((𝜑 ∨ 𝜒) ∧ (𝜑 ∨ 𝜃)) ∧ ((𝜓 ∨ 𝜒) ∧ (𝜓 ∨ 𝜃)))) | ||
Theorem | anddi 811 | Double distributive law for conjunction. (Contributed by NM, 12-Aug-1994.) |
⊢ (((𝜑 ∨ 𝜓) ∧ (𝜒 ∨ 𝜃)) ↔ (((𝜑 ∧ 𝜒) ∨ (𝜑 ∧ 𝜃)) ∨ ((𝜓 ∧ 𝜒) ∨ (𝜓 ∧ 𝜃)))) | ||
Theorem | pm4.39 812 | Theorem *4.39 of [WhiteheadRussell] p. 118. (Contributed by NM, 3-Jan-2005.) |
⊢ (((𝜑 ↔ 𝜒) ∧ (𝜓 ↔ 𝜃)) → ((𝜑 ∨ 𝜓) ↔ (𝜒 ∨ 𝜃))) | ||
Theorem | animorl 813 | Conjunction implies disjunction with one common formula (1/4). (Contributed by BJ, 4-Oct-2019.) |
⊢ ((𝜑 ∧ 𝜓) → (𝜑 ∨ 𝜒)) | ||
Theorem | animorr 814 | Conjunction implies disjunction with one common formula (2/4). (Contributed by BJ, 4-Oct-2019.) |
⊢ ((𝜑 ∧ 𝜓) → (𝜒 ∨ 𝜓)) | ||
Theorem | animorlr 815 | Conjunction implies disjunction with one common formula (3/4). (Contributed by BJ, 4-Oct-2019.) |
⊢ ((𝜑 ∧ 𝜓) → (𝜒 ∨ 𝜑)) | ||
Theorem | animorrl 816 | Conjunction implies disjunction with one common formula (4/4). (Contributed by BJ, 4-Oct-2019.) |
⊢ ((𝜑 ∧ 𝜓) → (𝜓 ∨ 𝜒)) | ||
Theorem | pm4.72 817 | 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.) |
⊢ ((𝜑 → 𝜓) ↔ (𝜓 ↔ (𝜑 ∨ 𝜓))) | ||
Theorem | pm5.16 818 | Theorem *5.16 of [WhiteheadRussell] p. 124. (Contributed by NM, 3-Jan-2005.) (Revised by Mario Carneiro, 31-Jan-2015.) |
⊢ ¬ ((𝜑 ↔ 𝜓) ∧ (𝜑 ↔ ¬ 𝜓)) | ||
Theorem | biort 819 | A disjunction with a true formula is equivalent to that true formula. (Contributed by NM, 23-May-1999.) |
⊢ (𝜑 → (𝜑 ↔ (𝜑 ∨ 𝜓))) | ||
Syntax | wstab 820 | Extend wff definition to include stability. |
wff STAB 𝜑 | ||
Definition | df-stab 821 |
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 𝜑 ↔ (¬ ¬ 𝜑 → 𝜑)) | ||
Theorem | stbid 822 | The equivalent of a stable proposition is stable. (Contributed by Jim Kingdon, 12-Aug-2022.) |
⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (STAB 𝜓 ↔ STAB 𝜒)) | ||
Theorem | stabnot 823 | Every negated formula is stable. (Contributed by David A. Wheeler, 13-Aug-2018.) |
⊢ STAB ¬ 𝜑 | ||
Syntax | wdc 824 | Extend wff definition to include decidability. |
wff DECID 𝜑 | ||
Definition | df-dc 825 |
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 843, exmiddc 826, peircedc 904, or notnotrdc 833, any of which would correspond to the assertion that all propositions are decidable. (Contributed by Jim Kingdon, 11-Mar-2018.) |
⊢ (DECID 𝜑 ↔ (𝜑 ∨ ¬ 𝜑)) | ||
Theorem | exmiddc 826 | 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 𝜑 → (𝜑 ∨ ¬ 𝜑)) | ||
Theorem | pm2.1dc 827 | 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 𝜑 → (¬ 𝜑 ∨ 𝜑)) | ||
Theorem | dcbid 828 | Equivalence property for decidability. Deduction form. (Contributed by Jim Kingdon, 7-Sep-2019.) |
⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (DECID 𝜓 ↔ DECID 𝜒)) | ||
Theorem | dcbiit 829 | Equivalence property for decidability. Closed form. (Contributed by BJ, 27-Jan-2020.) |
⊢ ((𝜑 ↔ 𝜓) → (DECID 𝜑 ↔ DECID 𝜓)) | ||
Theorem | dcbii 830 | Equivalence property for decidability. Inference form. (Contributed by Jim Kingdon, 28-Mar-2018.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (DECID 𝜑 ↔ DECID 𝜓) | ||
Theorem | dcim 831 | An implication between two decidable propositions is decidable. (Contributed by Jim Kingdon, 28-Mar-2018.) |
⊢ (DECID 𝜑 → (DECID 𝜓 → DECID (𝜑 → 𝜓))) | ||
Theorem | dcn 832 | The negation of a decidable proposition is decidable. The converse need not hold, but does hold for negated propositions, see dcnn 838. (Contributed by Jim Kingdon, 25-Mar-2018.) |
⊢ (DECID 𝜑 → DECID ¬ 𝜑) | ||
Theorem | notnotrdc 833 | Double negation elimination for a decidable proposition. The converse, notnot 619, 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 𝜑 → (¬ ¬ 𝜑 → 𝜑)) | ||
Theorem | dcstab 834 | Decidability implies stability. The converse need not hold. (Contributed by David A. Wheeler, 13-Aug-2018.) |
⊢ (DECID 𝜑 → STAB 𝜑) | ||
Theorem | stdcndc 835 | 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 𝜑) | ||
Theorem | stdcndcOLD 836 | Obsolete version of stdcndc 835 as of 28-Oct-2023. (Contributed by David A. Wheeler, 13-Aug-2018.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ ((STAB 𝜑 ∧ DECID ¬ 𝜑) ↔ DECID 𝜑) | ||
Theorem | stdcn 837 | 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 832. (Contributed by BJ, 18-Nov-2023.) |
⊢ (STAB 𝜑 ↔ (DECID ¬ 𝜑 → DECID 𝜑)) | ||
Theorem | dcnn 838 | Decidability of the negation of a proposition is equivalent to decidability of its double negation. See also dcn 832. The relation between dcn 832 and dcnn 838 is analogous to that between notnot 619 and notnotnot 624 (and directly stems from it). Using the notion of "testable proposition" (proposition whose negation is decidable), dcnn 838 means that a proposition is testable if and only if its negation is testable, and dcn 832 means that decidability implies testability. (Contributed by David A. Wheeler, 6-Dec-2018.) (Proof shortened by BJ, 25-Nov-2023.) |
⊢ (DECID ¬ 𝜑 ↔ DECID ¬ ¬ 𝜑) | ||
Theorem | dcnnOLD 839 | Obsolete proof of dcnnOLD 839 as of 25-Nov-2023. (Contributed by David A. Wheeler, 6-Dec-2018.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (DECID ¬ 𝜑 ↔ DECID ¬ ¬ 𝜑) | ||
Theorem | nnexmid 840 | Double negation of decidability of a formula. See also comment of nndc 841 to avoid a pitfall that could come from the label "nnexmid". This theorem can also be proved from bj-nnor 13615 as in bj-nndcALT 13639. (Contributed by BJ, 9-Oct-2019.) |
⊢ ¬ ¬ (𝜑 ∨ ¬ 𝜑) | ||
Theorem | nndc 841 |
Double negation of decidability of a formula. Intuitionistic logic
refutes the negation of decidability (but does not prove decidability) of
any formula.
This should not trick the reader into thinking that ¬ ¬ EXMID is provable in intuitionistic logic. Indeed, if we could quantify over formula metavariables, then generalizing nnexmid 840 over 𝜑 would give "⊢ ∀𝜑¬ ¬ DECID 𝜑", but EXMID is "∀𝜑DECID 𝜑", so proving ¬ ¬ EXMID would amount to proving "¬ ¬ ∀𝜑DECID 𝜑", which is not implied by the above theorem. Indeed, the converse of nnal 1637 does not hold. Since our system does not allow quantification over formula metavariables, we can reproduce this argument by representing formulas as subsets of 𝒫 1o, like we do in our definition of EXMID (df-exmid 4174): then, we can prove ∀𝑥 ∈ 𝒫 1o¬ ¬ DECID 𝑥 = 1o but we cannot prove ¬ ¬ ∀𝑥 ∈ 𝒫 1oDECID 𝑥 = 1o because the converse of nnral 2456 does not hold. Actually, ¬ ¬ EXMID is not provable in intuitionistic logic since intuitionistic logic has models satisfying ¬ EXMID and noncontradiction holds (pm3.24 683). (Contributed by BJ, 9-Oct-2019.) Add explanation on non-provability of ¬ ¬ EXMID. (Revised by BJ, 11-Aug-2024.) |
⊢ ¬ ¬ DECID 𝜑 | ||
Many theorems of logic hold in intuitionistic logic just as they do in classical (non-intuitionistic) logic, for all propositions. Other theorems only hold for decidable propositions, such as the law of the excluded middle (df-dc 825), double negation elimination (notnotrdc 833), or contraposition (condc 843). 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 821). Decidable propositions are stable (dcstab 834), but the converse need not hold. | ||
Theorem | const 842 | Contraposition when the antecedent is a negated stable proposition. See comment of condc 843. (Contributed by BJ, 18-Nov-2023.) (Proof shortened by BJ, 11-Nov-2024.) |
⊢ (STAB 𝜑 → ((¬ 𝜑 → ¬ 𝜓) → (𝜓 → 𝜑))) | ||
Theorem | condc 843 |
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 𝜑 → ((¬ 𝜑 → ¬ 𝜓) → (𝜓 → 𝜑))) | ||
Theorem | condcOLD 844 | Obsolete proof of condc 843 as of 18-Nov-2023. (Contributed by Jim Kingdon, 13-Mar-2018.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 → ¬ 𝜓) → (𝜓 → 𝜑))) | ||
Theorem | pm2.18dc 845 | 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 606 which does not. (Contributed by Jim Kingdon, 24-Mar-2018.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 → 𝜑) → 𝜑)) | ||
Theorem | con1dc 846 | Contraposition for a decidable proposition. Based on theorem *2.15 of [WhiteheadRussell] p. 102. (Contributed by Jim Kingdon, 29-Mar-2018.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 → 𝜓) → (¬ 𝜓 → 𝜑))) | ||
Theorem | con4biddc 847 | A contraposition deduction. (Contributed by Jim Kingdon, 18-May-2018.) |
⊢ (𝜑 → (DECID 𝜓 → (DECID 𝜒 → (¬ 𝜓 ↔ ¬ 𝜒)))) ⇒ ⊢ (𝜑 → (DECID 𝜓 → (DECID 𝜒 → (𝜓 ↔ 𝜒)))) | ||
Theorem | impidc 848 | An importation inference for a decidable consequent. (Contributed by Jim Kingdon, 30-Apr-2018.) |
⊢ (DECID 𝜒 → (𝜑 → (𝜓 → 𝜒))) ⇒ ⊢ (DECID 𝜒 → (¬ (𝜑 → ¬ 𝜓) → 𝜒)) | ||
Theorem | simprimdc 849 | Simplification given a decidable proposition. Similar to Theorem *3.27 (Simp) of [WhiteheadRussell] p. 112. (Contributed by Jim Kingdon, 30-Apr-2018.) |
⊢ (DECID 𝜓 → (¬ (𝜑 → ¬ 𝜓) → 𝜓)) | ||
Theorem | simplimdc 850 | Simplification for a decidable proposition. Similar to Theorem *3.26 (Simp) of [WhiteheadRussell] p. 112. (Contributed by Jim Kingdon, 29-Mar-2018.) |
⊢ (DECID 𝜑 → (¬ (𝜑 → 𝜓) → 𝜑)) | ||
Theorem | pm2.61ddc 851 | Deduction eliminating a decidable antecedent. (Contributed by Jim Kingdon, 4-May-2018.) |
⊢ (𝜑 → (𝜓 → 𝜒)) & ⊢ (𝜑 → (¬ 𝜓 → 𝜒)) ⇒ ⊢ (DECID 𝜓 → (𝜑 → 𝜒)) | ||
Theorem | pm2.6dc 852 | Case elimination for a decidable proposition. Based on theorem *2.6 of [WhiteheadRussell] p. 107. (Contributed by Jim Kingdon, 25-Mar-2018.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 → 𝜓) → ((𝜑 → 𝜓) → 𝜓))) | ||
Theorem | jadc 853 | 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 𝜑 → ((𝜑 → 𝜓) → 𝜒)) | ||
Theorem | jaddc 854 | 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 𝜓 → ((𝜓 → 𝜒) → 𝜃))) | ||
Theorem | pm2.61dc 855 | 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 𝜑 → ((𝜑 → 𝜓) → ((¬ 𝜑 → 𝜓) → 𝜓))) | ||
Theorem | pm2.5gdc 856 | 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 𝜑 → (¬ (𝜑 → 𝜓) → (¬ 𝜑 → 𝜒))) | ||
Theorem | pm2.5dc 857 | 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 𝜑 → (¬ (𝜑 → 𝜓) → (¬ 𝜑 → 𝜓))) | ||
Theorem | pm2.521gdc 858 | A general instance of Theorem *2.521 of [WhiteheadRussell] p. 107, under a decidability condition. (Contributed by BJ, 28-Oct-2023.) |
⊢ (DECID 𝜑 → (¬ (𝜑 → 𝜓) → (𝜒 → 𝜑))) | ||
Theorem | pm2.521dc 859 | Theorem *2.521 of [WhiteheadRussell] p. 107, but with an additional decidability condition. Note that by replacing in proof pm2.52 646 with conax1k 644, 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 𝜑 → (¬ (𝜑 → 𝜓) → (𝜓 → 𝜑))) | ||
Theorem | pm2.521dcALT 860 | Alternate proof of pm2.521dc 859. (Contributed by Jim Kingdon, 5-May-2018.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (DECID 𝜑 → (¬ (𝜑 → 𝜓) → (𝜓 → 𝜑))) | ||
Theorem | con34bdc 861 | Contraposition. Theorem *4.1 of [WhiteheadRussell] p. 116, but for a decidable proposition. (Contributed by Jim Kingdon, 24-Apr-2018.) |
⊢ (DECID 𝜓 → ((𝜑 → 𝜓) ↔ (¬ 𝜓 → ¬ 𝜑))) | ||
Theorem | notnotbdc 862 | Double negation equivalence for a decidable proposition. Like Theorem *4.13 of [WhiteheadRussell] p. 117, but with a decidability antecendent. The forward direction, notnot 619, holds for all propositions, not just decidable ones. (Contributed by Jim Kingdon, 13-Mar-2018.) |
⊢ (DECID 𝜑 → (𝜑 ↔ ¬ ¬ 𝜑)) | ||
Theorem | con1biimdc 863 | Contraposition. (Contributed by Jim Kingdon, 4-Apr-2018.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 ↔ 𝜓) → (¬ 𝜓 ↔ 𝜑))) | ||
Theorem | con1bidc 864 | Contraposition. (Contributed by Jim Kingdon, 17-Apr-2018.) |
⊢ (DECID 𝜑 → (DECID 𝜓 → ((¬ 𝜑 ↔ 𝜓) ↔ (¬ 𝜓 ↔ 𝜑)))) | ||
Theorem | con2bidc 865 | Contraposition. (Contributed by Jim Kingdon, 17-Apr-2018.) |
⊢ (DECID 𝜑 → (DECID 𝜓 → ((𝜑 ↔ ¬ 𝜓) ↔ (𝜓 ↔ ¬ 𝜑)))) | ||
Theorem | con1biddc 866 | A contraposition deduction. (Contributed by Jim Kingdon, 4-Apr-2018.) |
⊢ (𝜑 → (DECID 𝜓 → (¬ 𝜓 ↔ 𝜒))) ⇒ ⊢ (𝜑 → (DECID 𝜓 → (¬ 𝜒 ↔ 𝜓))) | ||
Theorem | con1biidc 867 | A contraposition inference. (Contributed by Jim Kingdon, 15-Mar-2018.) |
⊢ (DECID 𝜑 → (¬ 𝜑 ↔ 𝜓)) ⇒ ⊢ (DECID 𝜑 → (¬ 𝜓 ↔ 𝜑)) | ||
Theorem | con1bdc 868 | Contraposition. Bidirectional version of con1dc 846. (Contributed by NM, 5-Aug-1993.) |
⊢ (DECID 𝜑 → (DECID 𝜓 → ((¬ 𝜑 → 𝜓) ↔ (¬ 𝜓 → 𝜑)))) | ||
Theorem | con2biidc 869 | A contraposition inference. (Contributed by Jim Kingdon, 15-Mar-2018.) |
⊢ (DECID 𝜓 → (𝜑 ↔ ¬ 𝜓)) ⇒ ⊢ (DECID 𝜓 → (𝜓 ↔ ¬ 𝜑)) | ||
Theorem | con2biddc 870 | A contraposition deduction. (Contributed by Jim Kingdon, 11-Apr-2018.) |
⊢ (𝜑 → (DECID 𝜒 → (𝜓 ↔ ¬ 𝜒))) ⇒ ⊢ (𝜑 → (DECID 𝜒 → (𝜒 ↔ ¬ 𝜓))) | ||
Theorem | condandc 871 | 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 649, is valid for all propositions. (Contributed by Jim Kingdon, 13-May-2018.) |
⊢ ((𝜑 ∧ ¬ 𝜓) → 𝜒) & ⊢ ((𝜑 ∧ ¬ 𝜓) → ¬ 𝜒) ⇒ ⊢ (DECID 𝜓 → (𝜑 → 𝜓)) | ||
Theorem | bijadc 872 | Combine antecedents into a single biconditional. This inference is reminiscent of jadc 853. (Contributed by Jim Kingdon, 4-May-2018.) |
⊢ (𝜑 → (𝜓 → 𝜒)) & ⊢ (¬ 𝜑 → (¬ 𝜓 → 𝜒)) ⇒ ⊢ (DECID 𝜓 → ((𝜑 ↔ 𝜓) → 𝜒)) | ||
Theorem | pm5.18dc 873 | 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 𝜓 → ((𝜑 ↔ 𝜓) ↔ ¬ (𝜑 ↔ ¬ 𝜓)))) | ||
Theorem | dfandc 874 | 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 627. (Contributed by Jim Kingdon, 30-Apr-2018.) |
⊢ (DECID 𝜑 → (DECID 𝜓 → ((𝜑 ∧ 𝜓) ↔ ¬ (𝜑 → ¬ 𝜓)))) | ||
Theorem | pm2.13dc 875 | 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 𝜑 → (𝜑 ∨ ¬ ¬ ¬ 𝜑)) | ||
Theorem | pm4.63dc 876 | Theorem *4.63 of [WhiteheadRussell] p. 120, for decidable propositions. (Contributed by Jim Kingdon, 1-May-2018.) |
⊢ (DECID 𝜑 → (DECID 𝜓 → (¬ (𝜑 → ¬ 𝜓) ↔ (𝜑 ∧ 𝜓)))) | ||
Theorem | pm4.67dc 877 | Theorem *4.67 of [WhiteheadRussell] p. 120, for decidable propositions. (Contributed by Jim Kingdon, 1-May-2018.) |
⊢ (DECID 𝜑 → (DECID 𝜓 → (¬ (¬ 𝜑 → ¬ 𝜓) ↔ (¬ 𝜑 ∧ 𝜓)))) | ||
Theorem | imanst 878 | 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 𝜓 → ((𝜑 → 𝜓) ↔ ¬ (𝜑 ∧ ¬ 𝜓))) | ||
Theorem | imandc 879 | Express implication in terms of conjunction. Theorem 3.4(27) of [Stoll] p. 176, with an added decidability condition. The forward direction, imanim 678, holds for all propositions, not just decidable ones. (Contributed by Jim Kingdon, 25-Apr-2018.) |
⊢ (DECID 𝜓 → ((𝜑 → 𝜓) ↔ ¬ (𝜑 ∧ ¬ 𝜓))) | ||
Theorem | pm4.14dc 880 | Theorem *4.14 of [WhiteheadRussell] p. 117, given a decidability condition. (Contributed by Jim Kingdon, 24-Apr-2018.) |
⊢ (DECID 𝜒 → (((𝜑 ∧ 𝜓) → 𝜒) ↔ ((𝜑 ∧ ¬ 𝜒) → ¬ 𝜓))) | ||
Theorem | pm2.54dc 881 | Deriving disjunction from implication for a decidable proposition. Based on theorem *2.54 of [WhiteheadRussell] p. 107. The converse, pm2.53 712, holds whether the proposition is decidable or not. (Contributed by Jim Kingdon, 26-Mar-2018.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 → 𝜓) → (𝜑 ∨ 𝜓))) | ||
Theorem | dfordc 882 | Definition of disjunction in terms of negation and implication for a decidable proposition. Based on definition of [Margaris] p. 49. One direction, pm2.53 712, holds for all propositions, not just decidable ones. (Contributed by Jim Kingdon, 26-Mar-2018.) |
⊢ (DECID 𝜑 → ((𝜑 ∨ 𝜓) ↔ (¬ 𝜑 → 𝜓))) | ||
Theorem | pm2.25dc 883 | 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 𝜑 → (𝜑 ∨ ((𝜑 ∨ 𝜓) → 𝜓))) | ||
Theorem | pm2.68dc 884 | Concluding disjunction from implication for a decidable proposition. Based on theorem *2.68 of [WhiteheadRussell] p. 108. Converse of pm2.62 738 and one half of dfor2dc 885. (Contributed by Jim Kingdon, 27-Mar-2018.) |
⊢ (DECID 𝜑 → (((𝜑 → 𝜓) → 𝜓) → (𝜑 ∨ 𝜓))) | ||
Theorem | dfor2dc 885 | 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 𝜑 → ((𝜑 ∨ 𝜓) ↔ ((𝜑 → 𝜓) → 𝜓))) | ||
Theorem | imimorbdc 886 | Simplify an implication between implications, for a decidable proposition. (Contributed by Jim Kingdon, 18-Mar-2018.) |
⊢ (DECID 𝜓 → (((𝜓 → 𝜒) → (𝜑 → 𝜒)) ↔ (𝜑 → (𝜓 ∨ 𝜒)))) | ||
Theorem | imordc 887 | Implication in terms of disjunction for a decidable proposition. Based on theorem *4.6 of [WhiteheadRussell] p. 120. The reverse direction, imorr 711, holds for all propositions. (Contributed by Jim Kingdon, 20-Apr-2018.) |
⊢ (DECID 𝜑 → ((𝜑 → 𝜓) ↔ (¬ 𝜑 ∨ 𝜓))) | ||
Theorem | pm4.62dc 888 | 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 𝜑 → ((𝜑 → ¬ 𝜓) ↔ (¬ 𝜑 ∨ ¬ 𝜓))) | ||
Theorem | ianordc 889 | 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 743, holds for all propositions, but the equivalence only holds where one proposition is decidable. (Contributed by Jim Kingdon, 21-Apr-2018.) |
⊢ (DECID 𝜑 → (¬ (𝜑 ∧ 𝜓) ↔ (¬ 𝜑 ∨ ¬ 𝜓))) | ||
Theorem | pm4.64dc 890 | Theorem *4.64 of [WhiteheadRussell] p. 120, given a decidability condition. The reverse direction, pm2.53 712, holds for all propositions. (Contributed by Jim Kingdon, 2-May-2018.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 → 𝜓) ↔ (𝜑 ∨ 𝜓))) | ||
Theorem | pm4.66dc 891 | Theorem *4.66 of [WhiteheadRussell] p. 120, given a decidability condition. (Contributed by Jim Kingdon, 2-May-2018.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 → ¬ 𝜓) ↔ (𝜑 ∨ ¬ 𝜓))) | ||
Theorem | pm4.54dc 892 | 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 𝜓 → ((¬ 𝜑 ∧ 𝜓) ↔ ¬ (𝜑 ∨ ¬ 𝜓)))) | ||
Theorem | pm4.79dc 893 | 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 𝜓 → (((𝜓 → 𝜑) ∨ (𝜒 → 𝜑)) ↔ ((𝜓 ∧ 𝜒) → 𝜑)))) | ||
Theorem | pm5.17dc 894 | 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 𝜓 → (((𝜑 ∨ 𝜓) ∧ ¬ (𝜑 ∧ 𝜓)) ↔ (𝜑 ↔ ¬ 𝜓))) | ||
Theorem | pm2.85dc 895 | 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 𝜑 → (((𝜑 ∨ 𝜓) → (𝜑 ∨ 𝜒)) → (𝜑 ∨ (𝜓 → 𝜒)))) | ||
Theorem | orimdidc 896 | Disjunction distributes over implication. The forward direction, pm2.76 798, is valid intuitionistically. The reverse direction holds if 𝜑 is decidable, as can be seen at pm2.85dc 895. (Contributed by Jim Kingdon, 1-Apr-2018.) |
⊢ (DECID 𝜑 → ((𝜑 ∨ (𝜓 → 𝜒)) ↔ ((𝜑 ∨ 𝜓) → (𝜑 ∨ 𝜒)))) | ||
Theorem | pm2.26dc 897 | Decidable proposition version of theorem *2.26 of [WhiteheadRussell] p. 104. (Contributed by Jim Kingdon, 20-Apr-2018.) |
⊢ (DECID 𝜑 → (¬ 𝜑 ∨ ((𝜑 → 𝜓) → 𝜓))) | ||
Theorem | pm4.81dc 898 | Theorem *4.81 of [WhiteheadRussell] p. 122, for decidable propositions. This one needs a decidability condition, but compare with pm4.8 697 which holds for all propositions. (Contributed by Jim Kingdon, 4-Jul-2018.) |
⊢ (DECID 𝜑 → ((¬ 𝜑 → 𝜑) ↔ 𝜑)) | ||
Theorem | pm5.11dc 899 | 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 𝜓 → ((𝜑 → 𝜓) ∨ (¬ 𝜑 → 𝜓)))) | ||
Theorem | pm5.12dc 900 | 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 𝜓 → ((𝜑 → 𝜓) ∨ (𝜑 → ¬ 𝜓))) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |