![]() |
Metamath
Proof Explorer Theorem List (p. 30 of 486) | < Previous Next > |
Bad symbols? Try the
GIF version. |
||
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Color key: | ![]() (1-30851) |
![]() (30852-32374) |
![]() (32375-48553) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | nfaba1OLD 2901* | Obsolete version of nfaba1 2900 as of 14-May-2025. (Contributed by Mario Carneiro, 14-Oct-2016.) (Revised by GG, 20-Jan-2024.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ Ⅎ𝑥{𝑦 ∣ ∀𝑥𝜑} | ||
Theorem | nfaba1g 2902 | Bound-variable hypothesis builder for a class abstraction. Usage of this theorem is discouraged because it depends on ax-13 2366. See nfaba1 2900 for a version with a disjoint variable condition, but not requiring ax-13 2366. (Contributed by Mario Carneiro, 14-Oct-2016.) (New usage is discouraged.) |
⊢ Ⅎ𝑥{𝑦 ∣ ∀𝑥𝜑} | ||
Theorem | nfeqd 2903 | Hypothesis builder for equality. (Contributed by Mario Carneiro, 7-Oct-2016.) |
⊢ (𝜑 → Ⅎ𝑥𝐴) & ⊢ (𝜑 → Ⅎ𝑥𝐵) ⇒ ⊢ (𝜑 → Ⅎ𝑥 𝐴 = 𝐵) | ||
Theorem | nfeld 2904 | Hypothesis builder for elementhood. (Contributed by Mario Carneiro, 7-Oct-2016.) |
⊢ (𝜑 → Ⅎ𝑥𝐴) & ⊢ (𝜑 → Ⅎ𝑥𝐵) ⇒ ⊢ (𝜑 → Ⅎ𝑥 𝐴 ∈ 𝐵) | ||
Theorem | nfnfc 2905 | Hypothesis builder for Ⅎ𝑦𝐴. (Contributed by Mario Carneiro, 11-Aug-2016.) Remove dependency on ax-13 2366. (Revised by Wolf Lammen, 10-Dec-2019.) |
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ Ⅎ𝑥Ⅎ𝑦𝐴 | ||
Theorem | nfeq 2906 | Hypothesis builder for equality. (Contributed by NM, 21-Jun-1993.) (Revised by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 16-Nov-2019.) |
⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥 𝐴 = 𝐵 | ||
Theorem | nfel 2907 | Hypothesis builder for elementhood. (Contributed by NM, 1-Aug-1993.) (Revised by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 16-Nov-2019.) |
⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥 𝐴 ∈ 𝐵 | ||
Theorem | nfeq1 2908* | Hypothesis builder for equality, special case. (Contributed by Mario Carneiro, 10-Oct-2016.) |
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ Ⅎ𝑥 𝐴 = 𝐵 | ||
Theorem | nfel1 2909* | Hypothesis builder for elementhood, special case. (Contributed by Mario Carneiro, 10-Oct-2016.) |
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ Ⅎ𝑥 𝐴 ∈ 𝐵 | ||
Theorem | nfeq2 2910* | Hypothesis builder for equality, special case. (Contributed by Mario Carneiro, 10-Oct-2016.) |
⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥 𝐴 = 𝐵 | ||
Theorem | nfel2 2911* | Hypothesis builder for elementhood, special case. (Contributed by Mario Carneiro, 10-Oct-2016.) |
⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥 𝐴 ∈ 𝐵 | ||
Theorem | drnfc1 2912 | Formula-building lemma for use with the Distinctor Reduction Theorem. Usage of this theorem is discouraged because it depends on ax-13 2366. (Contributed by Mario Carneiro, 8-Oct-2016.) Avoid ax-8 2101, ax-11 2147. (Revised by Wolf Lammen, 22-Sep-2024.) (New usage is discouraged.) |
⊢ (∀𝑥 𝑥 = 𝑦 → 𝐴 = 𝐵) ⇒ ⊢ (∀𝑥 𝑥 = 𝑦 → (Ⅎ𝑥𝐴 ↔ Ⅎ𝑦𝐵)) | ||
Theorem | drnfc1OLD 2913 | Obsolete version of drnfc1 2912 as of 22-Sep-2024. (Contributed by Mario Carneiro, 8-Oct-2016.) Avoid ax-11 2147. (Revised by Wolf Lammen, 10-May-2023.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ (∀𝑥 𝑥 = 𝑦 → 𝐴 = 𝐵) ⇒ ⊢ (∀𝑥 𝑥 = 𝑦 → (Ⅎ𝑥𝐴 ↔ Ⅎ𝑦𝐵)) | ||
Theorem | drnfc2 2914 | Formula-building lemma for use with the Distinctor Reduction Theorem. Proof revision is marked as discouraged because the minimizer replaces albidv 1916 with dral2 2432, leading to a one byte longer proof. However feel free to manually edit it according to conventions. (TODO: dral2 2432 depends on ax-13 2366, hence its usage during minimizing is discouraged. Check in the long run whether this is a permanent restriction). Usage of this theorem is discouraged because it depends on ax-13 2366. (Contributed by Mario Carneiro, 8-Oct-2016.) Avoid ax-8 2101. (Revised by Wolf Lammen, 22-Sep-2024.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (∀𝑥 𝑥 = 𝑦 → 𝐴 = 𝐵) ⇒ ⊢ (∀𝑥 𝑥 = 𝑦 → (Ⅎ𝑧𝐴 ↔ Ⅎ𝑧𝐵)) | ||
Theorem | drnfc2OLD 2915 | Obsolete version of drnfc2 2914 as of 22-Sep-2024. (Contributed by Mario Carneiro, 8-Oct-2016.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (∀𝑥 𝑥 = 𝑦 → 𝐴 = 𝐵) ⇒ ⊢ (∀𝑥 𝑥 = 𝑦 → (Ⅎ𝑧𝐴 ↔ Ⅎ𝑧𝐵)) | ||
Theorem | nfabdw 2916* | Bound-variable hypothesis builder for a class abstraction. Version of nfabd 2918 with a disjoint variable condition, which does not require ax-13 2366. (Contributed by Mario Carneiro, 8-Oct-2016.) Avoid ax-13 2366. (Revised by GG, 10-Jan-2024.) (Proof shortened by Wolf Lammen, 23-Sep-2024.) |
⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜑 → Ⅎ𝑥{𝑦 ∣ 𝜓}) | ||
Theorem | nfabdwOLD 2917* | Obsolete version of nfabdw 2916 as of 23-Sep-2024. (Contributed by Mario Carneiro, 8-Oct-2016.) (Revised by GG, 10-Jan-2024.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜑 → Ⅎ𝑥{𝑦 ∣ 𝜓}) | ||
Theorem | nfabd 2918 | Bound-variable hypothesis builder for a class abstraction. Usage of this theorem is discouraged because it depends on ax-13 2366. Use the weaker nfabdw 2916 when possible. (Contributed by Mario Carneiro, 8-Oct-2016.) Avoid ax-9 2109 and ax-ext 2697. (Revised by Wolf Lammen, 23-May-2023.) (New usage is discouraged.) |
⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜑 → Ⅎ𝑥{𝑦 ∣ 𝜓}) | ||
Theorem | nfabd2 2919 | Bound-variable hypothesis builder for a class abstraction. Usage of this theorem is discouraged because it depends on ax-13 2366. (Contributed by Mario Carneiro, 8-Oct-2016.) (Proof shortened by Wolf Lammen, 10-May-2023.) (New usage is discouraged.) |
⊢ Ⅎ𝑦𝜑 & ⊢ ((𝜑 ∧ ¬ ∀𝑥 𝑥 = 𝑦) → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜑 → Ⅎ𝑥{𝑦 ∣ 𝜓}) | ||
Theorem | dvelimdc 2920 | Deduction form of dvelimc 2921. Usage of this theorem is discouraged because it depends on ax-13 2366. (Contributed by Mario Carneiro, 8-Oct-2016.) (New usage is discouraged.) |
⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑧𝜑 & ⊢ (𝜑 → Ⅎ𝑥𝐴) & ⊢ (𝜑 → Ⅎ𝑧𝐵) & ⊢ (𝜑 → (𝑧 = 𝑦 → 𝐴 = 𝐵)) ⇒ ⊢ (𝜑 → (¬ ∀𝑥 𝑥 = 𝑦 → Ⅎ𝑥𝐵)) | ||
Theorem | dvelimc 2921 | Version of dvelim 2445 for classes. Usage of this theorem is discouraged because it depends on ax-13 2366. (Contributed by Mario Carneiro, 8-Oct-2016.) (New usage is discouraged.) |
⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑧𝐵 & ⊢ (𝑧 = 𝑦 → 𝐴 = 𝐵) ⇒ ⊢ (¬ ∀𝑥 𝑥 = 𝑦 → Ⅎ𝑥𝐵) | ||
Theorem | nfcvf 2922 | If 𝑥 and 𝑦 are distinct, then 𝑥 is not free in 𝑦. Usage of this theorem is discouraged because it depends on ax-13 2366. See nfcv 2892 for a version that replaces the distinctor with a disjoint variable condition, requiring fewer axioms. (Contributed by Mario Carneiro, 8-Oct-2016.) Avoid ax-ext 2697. (Revised by Wolf Lammen, 10-May-2023.) (New usage is discouraged.) |
⊢ (¬ ∀𝑥 𝑥 = 𝑦 → Ⅎ𝑥𝑦) | ||
Theorem | nfcvf2 2923 | If 𝑥 and 𝑦 are distinct, then 𝑦 is not free in 𝑥. Usage of this theorem is discouraged because it depends on ax-13 2366. See nfcv 2892 for a version that replaces the distinctor with a disjoint variable condition, requiring fewer axioms. (Contributed by Mario Carneiro, 5-Dec-2016.) (New usage is discouraged.) |
⊢ (¬ ∀𝑥 𝑥 = 𝑦 → Ⅎ𝑦𝑥) | ||
Theorem | cleqf 2924 | Establish equality between classes, using bound-variable hypotheses instead of distinct variable conditions as in dfcleq 2719. See also cleqh 2856. (Contributed by NM, 26-May-1993.) (Revised by Mario Carneiro, 7-Oct-2016.) (Proof shortened by Wolf Lammen, 17-Nov-2019.) Avoid ax-13 2366. (Revised by Wolf Lammen, 10-May-2023.) Avoid ax-10 2130. (Revised by GG, 20-Aug-2023.) |
⊢ Ⅎ𝑥𝐴 & ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ (𝐴 = 𝐵 ↔ ∀𝑥(𝑥 ∈ 𝐴 ↔ 𝑥 ∈ 𝐵)) | ||
Theorem | eqabf 2925 | Equality of a class variable and a class abstraction. In this version, the fact that 𝑥 is a nonfree variable in 𝐴 is explicitly stated as a hypothesis. (Contributed by Thierry Arnoux, 11-May-2017.) Avoid ax-13 2366. (Revised by Wolf Lammen, 13-May-2023.) |
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ (𝐴 = {𝑥 ∣ 𝜑} ↔ ∀𝑥(𝑥 ∈ 𝐴 ↔ 𝜑)) | ||
Theorem | abid2f 2926 | A simplification of class abstraction. Theorem 5.2 of [Quine] p. 35. (Contributed by NM, 5-Sep-2011.) (Revised by Mario Carneiro, 7-Oct-2016.) (Proof shortened by Wolf Lammen, 26-Feb-2025.) |
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ {𝑥 ∣ 𝑥 ∈ 𝐴} = 𝐴 | ||
Theorem | abid2fOLD 2927 | Obsolete version of abid2f 2926 as of 26-Feb-2025. (Contributed by NM, 5-Sep-2011.) (Revised by Mario Carneiro, 7-Oct-2016.) (Proof shortened by Wolf Lammen, 17-Nov-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ {𝑥 ∣ 𝑥 ∈ 𝐴} = 𝐴 | ||
Theorem | sbabel 2928* | Theorem to move a substitution in and out of a class abstraction. (Contributed by NM, 27-Sep-2003.) (Revised by Mario Carneiro, 7-Oct-2016.) (Proof shortened by Wolf Lammen, 28-Oct-2024.) |
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ ([𝑦 / 𝑥]{𝑧 ∣ 𝜑} ∈ 𝐴 ↔ {𝑧 ∣ [𝑦 / 𝑥]𝜑} ∈ 𝐴) | ||
Theorem | sbabelOLD 2929* | Obsolete version of sbabel 2928 as of 28-Oct-2024. (Contributed by NM, 27-Sep-2003.) (Revised by Mario Carneiro, 7-Oct-2016.) (Proof shortened by Wolf Lammen, 26-Dec-2019.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ Ⅎ𝑥𝐴 ⇒ ⊢ ([𝑦 / 𝑥]{𝑧 ∣ 𝜑} ∈ 𝐴 ↔ {𝑧 ∣ [𝑦 / 𝑥]𝜑} ∈ 𝐴) | ||
Syntax | wne 2930 | Extend wff notation to include inequality. |
wff 𝐴 ≠ 𝐵 | ||
Definition | df-ne 2931 | Define inequality. (Contributed by NM, 26-May-1993.) |
⊢ (𝐴 ≠ 𝐵 ↔ ¬ 𝐴 = 𝐵) | ||
Theorem | neii 2932 | Inference associated with df-ne 2931. (Contributed by BJ, 7-Jul-2018.) |
⊢ 𝐴 ≠ 𝐵 ⇒ ⊢ ¬ 𝐴 = 𝐵 | ||
Theorem | neir 2933 | Inference associated with df-ne 2931. (Contributed by BJ, 7-Jul-2018.) |
⊢ ¬ 𝐴 = 𝐵 ⇒ ⊢ 𝐴 ≠ 𝐵 | ||
Theorem | nne 2934 | Negation of inequality. (Contributed by NM, 9-Jun-2006.) |
⊢ (¬ 𝐴 ≠ 𝐵 ↔ 𝐴 = 𝐵) | ||
Theorem | neneqd 2935 | Deduction eliminating inequality definition. (Contributed by Jonathan Ben-Naim, 3-Jun-2011.) |
⊢ (𝜑 → 𝐴 ≠ 𝐵) ⇒ ⊢ (𝜑 → ¬ 𝐴 = 𝐵) | ||
Theorem | neneq 2936 | From inequality to non-equality. (Contributed by Glauco Siliprandi, 11-Dec-2019.) |
⊢ (𝐴 ≠ 𝐵 → ¬ 𝐴 = 𝐵) | ||
Theorem | neqned 2937 | If it is not the case that two classes are equal, then they are unequal. Converse of neneqd 2935. One-way deduction form of df-ne 2931. (Contributed by David Moews, 28-Feb-2017.) Allow a shortening of necon3bi 2957. (Revised by Wolf Lammen, 22-Nov-2019.) |
⊢ (𝜑 → ¬ 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → 𝐴 ≠ 𝐵) | ||
Theorem | neqne 2938 | From non-equality to inequality. (Contributed by Glauco Siliprandi, 11-Dec-2019.) |
⊢ (¬ 𝐴 = 𝐵 → 𝐴 ≠ 𝐵) | ||
Theorem | neirr 2939 | No class is unequal to itself. Inequality is irreflexive. (Contributed by Stefan O'Rear, 1-Jan-2015.) |
⊢ ¬ 𝐴 ≠ 𝐴 | ||
Theorem | exmidne 2940 | Excluded middle with equality and inequality. (Contributed by NM, 3-Feb-2012.) (Proof shortened by Wolf Lammen, 17-Nov-2019.) |
⊢ (𝐴 = 𝐵 ∨ 𝐴 ≠ 𝐵) | ||
Theorem | eqneqall 2941 | A contradiction concerning equality implies anything. (Contributed by Alexander van der Vekens, 25-Jan-2018.) |
⊢ (𝐴 = 𝐵 → (𝐴 ≠ 𝐵 → 𝜑)) | ||
Theorem | nonconne 2942 | Law of noncontradiction with equality and inequality. (Contributed by NM, 3-Feb-2012.) (Proof shortened by Wolf Lammen, 21-Dec-2019.) |
⊢ ¬ (𝐴 = 𝐵 ∧ 𝐴 ≠ 𝐵) | ||
Theorem | necon3ad 2943 | Contrapositive law deduction for inequality. (Contributed by NM, 2-Apr-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 23-Nov-2019.) |
⊢ (𝜑 → (𝜓 → 𝐴 = 𝐵)) ⇒ ⊢ (𝜑 → (𝐴 ≠ 𝐵 → ¬ 𝜓)) | ||
Theorem | necon3bd 2944 | Contrapositive law deduction for inequality. (Contributed by NM, 2-Apr-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) |
⊢ (𝜑 → (𝐴 = 𝐵 → 𝜓)) ⇒ ⊢ (𝜑 → (¬ 𝜓 → 𝐴 ≠ 𝐵)) | ||
Theorem | necon2ad 2945 | Contrapositive inference for inequality. (Contributed by NM, 19-Apr-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 23-Nov-2019.) |
⊢ (𝜑 → (𝐴 = 𝐵 → ¬ 𝜓)) ⇒ ⊢ (𝜑 → (𝜓 → 𝐴 ≠ 𝐵)) | ||
Theorem | necon2bd 2946 | Contrapositive inference for inequality. (Contributed by NM, 13-Apr-2007.) |
⊢ (𝜑 → (𝜓 → 𝐴 ≠ 𝐵)) ⇒ ⊢ (𝜑 → (𝐴 = 𝐵 → ¬ 𝜓)) | ||
Theorem | necon1ad 2947 | Contrapositive deduction for inequality. (Contributed by NM, 2-Apr-2007.) (Proof shortened by Wolf Lammen, 23-Nov-2019.) |
⊢ (𝜑 → (¬ 𝜓 → 𝐴 = 𝐵)) ⇒ ⊢ (𝜑 → (𝐴 ≠ 𝐵 → 𝜓)) | ||
Theorem | necon1bd 2948 | Contrapositive deduction for inequality. (Contributed by NM, 21-Mar-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 23-Nov-2019.) |
⊢ (𝜑 → (𝐴 ≠ 𝐵 → 𝜓)) ⇒ ⊢ (𝜑 → (¬ 𝜓 → 𝐴 = 𝐵)) | ||
Theorem | necon4ad 2949 | Contrapositive inference for inequality. (Contributed by NM, 2-Apr-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 23-Nov-2019.) |
⊢ (𝜑 → (𝐴 ≠ 𝐵 → ¬ 𝜓)) ⇒ ⊢ (𝜑 → (𝜓 → 𝐴 = 𝐵)) | ||
Theorem | necon4bd 2950 | Contrapositive inference for inequality. (Contributed by NM, 1-Jun-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 23-Nov-2019.) |
⊢ (𝜑 → (¬ 𝜓 → 𝐴 ≠ 𝐵)) ⇒ ⊢ (𝜑 → (𝐴 = 𝐵 → 𝜓)) | ||
Theorem | necon3d 2951 | Contrapositive law deduction for inequality. (Contributed by NM, 10-Jun-2006.) |
⊢ (𝜑 → (𝐴 = 𝐵 → 𝐶 = 𝐷)) ⇒ ⊢ (𝜑 → (𝐶 ≠ 𝐷 → 𝐴 ≠ 𝐵)) | ||
Theorem | necon1d 2952 | Contrapositive law deduction for inequality. (Contributed by NM, 28-Dec-2008.) (Proof shortened by Andrew Salmon, 25-May-2011.) |
⊢ (𝜑 → (𝐴 ≠ 𝐵 → 𝐶 = 𝐷)) ⇒ ⊢ (𝜑 → (𝐶 ≠ 𝐷 → 𝐴 = 𝐵)) | ||
Theorem | necon2d 2953 | Contrapositive inference for inequality. (Contributed by NM, 28-Dec-2008.) |
⊢ (𝜑 → (𝐴 = 𝐵 → 𝐶 ≠ 𝐷)) ⇒ ⊢ (𝜑 → (𝐶 = 𝐷 → 𝐴 ≠ 𝐵)) | ||
Theorem | necon4d 2954 | Contrapositive inference for inequality. (Contributed by NM, 2-Apr-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) |
⊢ (𝜑 → (𝐴 ≠ 𝐵 → 𝐶 ≠ 𝐷)) ⇒ ⊢ (𝜑 → (𝐶 = 𝐷 → 𝐴 = 𝐵)) | ||
Theorem | necon3ai 2955 | Contrapositive inference for inequality. (Contributed by NM, 23-May-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 28-Oct-2024.) |
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝐴 ≠ 𝐵 → ¬ 𝜑) | ||
Theorem | necon3aiOLD 2956 | Obsolete version of necon3ai 2955 as of 28-Oct-2024. (Contributed by NM, 23-May-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝐴 ≠ 𝐵 → ¬ 𝜑) | ||
Theorem | necon3bi 2957 | Contrapositive inference for inequality. (Contributed by NM, 1-Jun-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 22-Nov-2019.) |
⊢ (𝐴 = 𝐵 → 𝜑) ⇒ ⊢ (¬ 𝜑 → 𝐴 ≠ 𝐵) | ||
Theorem | necon1ai 2958 | Contrapositive inference for inequality. (Contributed by NM, 12-Feb-2007.) (Proof shortened by Wolf Lammen, 22-Nov-2019.) |
⊢ (¬ 𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝐴 ≠ 𝐵 → 𝜑) | ||
Theorem | necon1bi 2959 | Contrapositive inference for inequality. (Contributed by NM, 18-Mar-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 22-Nov-2019.) |
⊢ (𝐴 ≠ 𝐵 → 𝜑) ⇒ ⊢ (¬ 𝜑 → 𝐴 = 𝐵) | ||
Theorem | necon2ai 2960 | Contrapositive inference for inequality. (Contributed by NM, 16-Jan-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 22-Nov-2019.) |
⊢ (𝐴 = 𝐵 → ¬ 𝜑) ⇒ ⊢ (𝜑 → 𝐴 ≠ 𝐵) | ||
Theorem | necon2bi 2961 | Contrapositive inference for inequality. (Contributed by NM, 1-Apr-2007.) |
⊢ (𝜑 → 𝐴 ≠ 𝐵) ⇒ ⊢ (𝐴 = 𝐵 → ¬ 𝜑) | ||
Theorem | necon4ai 2962 | Contrapositive inference for inequality. (Contributed by NM, 16-Jan-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 22-Nov-2019.) |
⊢ (𝐴 ≠ 𝐵 → ¬ 𝜑) ⇒ ⊢ (𝜑 → 𝐴 = 𝐵) | ||
Theorem | necon3i 2963 | Contrapositive inference for inequality. (Contributed by NM, 9-Aug-2006.) (Proof shortened by Wolf Lammen, 22-Nov-2019.) |
⊢ (𝐴 = 𝐵 → 𝐶 = 𝐷) ⇒ ⊢ (𝐶 ≠ 𝐷 → 𝐴 ≠ 𝐵) | ||
Theorem | necon1i 2964 | Contrapositive inference for inequality. (Contributed by NM, 18-Mar-2007.) |
⊢ (𝐴 ≠ 𝐵 → 𝐶 = 𝐷) ⇒ ⊢ (𝐶 ≠ 𝐷 → 𝐴 = 𝐵) | ||
Theorem | necon2i 2965 | Contrapositive inference for inequality. (Contributed by NM, 18-Mar-2007.) |
⊢ (𝐴 = 𝐵 → 𝐶 ≠ 𝐷) ⇒ ⊢ (𝐶 = 𝐷 → 𝐴 ≠ 𝐵) | ||
Theorem | necon4i 2966 | Contrapositive inference for inequality. (Contributed by NM, 17-Mar-2007.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 24-Nov-2019.) |
⊢ (𝐴 ≠ 𝐵 → 𝐶 ≠ 𝐷) ⇒ ⊢ (𝐶 = 𝐷 → 𝐴 = 𝐵) | ||
Theorem | necon3abid 2967 | Deduction from equality to inequality. (Contributed by NM, 21-Mar-2007.) |
⊢ (𝜑 → (𝐴 = 𝐵 ↔ 𝜓)) ⇒ ⊢ (𝜑 → (𝐴 ≠ 𝐵 ↔ ¬ 𝜓)) | ||
Theorem | necon3bbid 2968 | Deduction from equality to inequality. (Contributed by NM, 2-Jun-2007.) |
⊢ (𝜑 → (𝜓 ↔ 𝐴 = 𝐵)) ⇒ ⊢ (𝜑 → (¬ 𝜓 ↔ 𝐴 ≠ 𝐵)) | ||
Theorem | necon1abid 2969 | Contrapositive deduction for inequality. (Contributed by NM, 21-Aug-2007.) (Proof shortened by Wolf Lammen, 24-Nov-2019.) |
⊢ (𝜑 → (¬ 𝜓 ↔ 𝐴 = 𝐵)) ⇒ ⊢ (𝜑 → (𝐴 ≠ 𝐵 ↔ 𝜓)) | ||
Theorem | necon1bbid 2970 | Contrapositive inference for inequality. (Contributed by NM, 31-Jan-2008.) |
⊢ (𝜑 → (𝐴 ≠ 𝐵 ↔ 𝜓)) ⇒ ⊢ (𝜑 → (¬ 𝜓 ↔ 𝐴 = 𝐵)) | ||
Theorem | necon4abid 2971 | Contrapositive law deduction for inequality. (Contributed by NM, 11-Jan-2008.) (Proof shortened by Wolf Lammen, 24-Nov-2019.) |
⊢ (𝜑 → (𝐴 ≠ 𝐵 ↔ ¬ 𝜓)) ⇒ ⊢ (𝜑 → (𝐴 = 𝐵 ↔ 𝜓)) | ||
Theorem | necon4bbid 2972 | Contrapositive law deduction for inequality. (Contributed by NM, 9-May-2012.) |
⊢ (𝜑 → (¬ 𝜓 ↔ 𝐴 ≠ 𝐵)) ⇒ ⊢ (𝜑 → (𝜓 ↔ 𝐴 = 𝐵)) | ||
Theorem | necon2abid 2973 | Contrapositive deduction for inequality. (Contributed by NM, 18-Jul-2007.) (Proof shortened by Wolf Lammen, 24-Nov-2019.) |
⊢ (𝜑 → (𝐴 = 𝐵 ↔ ¬ 𝜓)) ⇒ ⊢ (𝜑 → (𝜓 ↔ 𝐴 ≠ 𝐵)) | ||
Theorem | necon2bbid 2974 | Contrapositive deduction for inequality. (Contributed by NM, 13-Apr-2007.) (Proof shortened by Wolf Lammen, 24-Nov-2019.) |
⊢ (𝜑 → (𝜓 ↔ 𝐴 ≠ 𝐵)) ⇒ ⊢ (𝜑 → (𝐴 = 𝐵 ↔ ¬ 𝜓)) | ||
Theorem | necon3bid 2975 | Deduction from equality to inequality. (Contributed by NM, 23-Feb-2005.) (Proof shortened by Andrew Salmon, 25-May-2011.) |
⊢ (𝜑 → (𝐴 = 𝐵 ↔ 𝐶 = 𝐷)) ⇒ ⊢ (𝜑 → (𝐴 ≠ 𝐵 ↔ 𝐶 ≠ 𝐷)) | ||
Theorem | necon4bid 2976 | Contrapositive law deduction for inequality. (Contributed by NM, 29-Jun-2007.) |
⊢ (𝜑 → (𝐴 ≠ 𝐵 ↔ 𝐶 ≠ 𝐷)) ⇒ ⊢ (𝜑 → (𝐴 = 𝐵 ↔ 𝐶 = 𝐷)) | ||
Theorem | necon3abii 2977 | Deduction from equality to inequality. (Contributed by NM, 9-Nov-2007.) |
⊢ (𝐴 = 𝐵 ↔ 𝜑) ⇒ ⊢ (𝐴 ≠ 𝐵 ↔ ¬ 𝜑) | ||
Theorem | necon3bbii 2978 | Deduction from equality to inequality. (Contributed by NM, 13-Apr-2007.) |
⊢ (𝜑 ↔ 𝐴 = 𝐵) ⇒ ⊢ (¬ 𝜑 ↔ 𝐴 ≠ 𝐵) | ||
Theorem | necon1abii 2979 | Contrapositive inference for inequality. (Contributed by NM, 17-Mar-2007.) (Proof shortened by Wolf Lammen, 25-Nov-2019.) |
⊢ (¬ 𝜑 ↔ 𝐴 = 𝐵) ⇒ ⊢ (𝐴 ≠ 𝐵 ↔ 𝜑) | ||
Theorem | necon1bbii 2980 | Contrapositive inference for inequality. (Contributed by NM, 17-Mar-2007.) (Proof shortened by Wolf Lammen, 24-Nov-2019.) |
⊢ (𝐴 ≠ 𝐵 ↔ 𝜑) ⇒ ⊢ (¬ 𝜑 ↔ 𝐴 = 𝐵) | ||
Theorem | necon2abii 2981 | Contrapositive inference for inequality. (Contributed by NM, 2-Mar-2007.) |
⊢ (𝐴 = 𝐵 ↔ ¬ 𝜑) ⇒ ⊢ (𝜑 ↔ 𝐴 ≠ 𝐵) | ||
Theorem | necon2bbii 2982 | Contrapositive inference for inequality. (Contributed by NM, 13-Apr-2007.) |
⊢ (𝜑 ↔ 𝐴 ≠ 𝐵) ⇒ ⊢ (𝐴 = 𝐵 ↔ ¬ 𝜑) | ||
Theorem | necon3bii 2983 | Inference from equality to inequality. (Contributed by NM, 23-Feb-2005.) |
⊢ (𝐴 = 𝐵 ↔ 𝐶 = 𝐷) ⇒ ⊢ (𝐴 ≠ 𝐵 ↔ 𝐶 ≠ 𝐷) | ||
Theorem | necom 2984 | Commutation of inequality. (Contributed by NM, 14-May-1999.) |
⊢ (𝐴 ≠ 𝐵 ↔ 𝐵 ≠ 𝐴) | ||
Theorem | necomi 2985 | Inference from commutative law for inequality. (Contributed by NM, 17-Oct-2012.) |
⊢ 𝐴 ≠ 𝐵 ⇒ ⊢ 𝐵 ≠ 𝐴 | ||
Theorem | necomd 2986 | Deduction from commutative law for inequality. (Contributed by NM, 12-Feb-2008.) |
⊢ (𝜑 → 𝐴 ≠ 𝐵) ⇒ ⊢ (𝜑 → 𝐵 ≠ 𝐴) | ||
Theorem | nesym 2987 | Characterization of inequality in terms of reversed equality (see bicom 221). (Contributed by BJ, 7-Jul-2018.) |
⊢ (𝐴 ≠ 𝐵 ↔ ¬ 𝐵 = 𝐴) | ||
Theorem | nesymi 2988 | Inference associated with nesym 2987. (Contributed by BJ, 7-Jul-2018.) (Proof shortened by Wolf Lammen, 25-Nov-2019.) |
⊢ 𝐴 ≠ 𝐵 ⇒ ⊢ ¬ 𝐵 = 𝐴 | ||
Theorem | nesymir 2989 | Inference associated with nesym 2987. (Contributed by BJ, 7-Jul-2018.) (Proof shortened by Wolf Lammen, 25-Nov-2019.) |
⊢ ¬ 𝐴 = 𝐵 ⇒ ⊢ 𝐵 ≠ 𝐴 | ||
Theorem | neeq1d 2990 | Deduction for inequality. (Contributed by NM, 25-Oct-1999.) (Proof shortened by Wolf Lammen, 19-Nov-2019.) |
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐴 ≠ 𝐶 ↔ 𝐵 ≠ 𝐶)) | ||
Theorem | neeq2d 2991 | Deduction for inequality. (Contributed by NM, 25-Oct-1999.) (Proof shortened by Wolf Lammen, 19-Nov-2019.) |
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐶 ≠ 𝐴 ↔ 𝐶 ≠ 𝐵)) | ||
Theorem | neeq12d 2992 | Deduction for inequality. (Contributed by NM, 24-Jul-2012.) (Proof shortened by Wolf Lammen, 25-Nov-2019.) |
⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ≠ 𝐶 ↔ 𝐵 ≠ 𝐷)) | ||
Theorem | neeq1 2993 | Equality theorem for inequality. (Contributed by NM, 19-Nov-1994.) (Proof shortened by Wolf Lammen, 18-Nov-2019.) |
⊢ (𝐴 = 𝐵 → (𝐴 ≠ 𝐶 ↔ 𝐵 ≠ 𝐶)) | ||
Theorem | neeq2 2994 | Equality theorem for inequality. (Contributed by NM, 19-Nov-1994.) (Proof shortened by Wolf Lammen, 18-Nov-2019.) |
⊢ (𝐴 = 𝐵 → (𝐶 ≠ 𝐴 ↔ 𝐶 ≠ 𝐵)) | ||
Theorem | neeq1i 2995 | Inference for inequality. (Contributed by NM, 29-Apr-2005.) (Proof shortened by Wolf Lammen, 19-Nov-2019.) |
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐴 ≠ 𝐶 ↔ 𝐵 ≠ 𝐶) | ||
Theorem | neeq2i 2996 | Inference for inequality. (Contributed by NM, 29-Apr-2005.) (Proof shortened by Wolf Lammen, 19-Nov-2019.) |
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐶 ≠ 𝐴 ↔ 𝐶 ≠ 𝐵) | ||
Theorem | neeq12i 2997 | Inference for inequality. (Contributed by NM, 24-Jul-2012.) (Proof shortened by Wolf Lammen, 25-Nov-2019.) |
⊢ 𝐴 = 𝐵 & ⊢ 𝐶 = 𝐷 ⇒ ⊢ (𝐴 ≠ 𝐶 ↔ 𝐵 ≠ 𝐷) | ||
Theorem | eqnetrd 2998 | Substitution of equal classes into an inequality. (Contributed by NM, 4-Jul-2012.) |
⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ (𝜑 → 𝐵 ≠ 𝐶) ⇒ ⊢ (𝜑 → 𝐴 ≠ 𝐶) | ||
Theorem | eqnetrrd 2999 | Substitution of equal classes into an inequality. (Contributed by NM, 4-Jul-2012.) |
⊢ (𝜑 → 𝐴 = 𝐵) & ⊢ (𝜑 → 𝐴 ≠ 𝐶) ⇒ ⊢ (𝜑 → 𝐵 ≠ 𝐶) | ||
Theorem | neeqtrd 3000 | Substitution of equal classes into an inequality. (Contributed by NM, 4-Jul-2012.) |
⊢ (𝜑 → 𝐴 ≠ 𝐵) & ⊢ (𝜑 → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → 𝐴 ≠ 𝐶) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |