Description: The following User's Proof is a Natural Deduction Sequent Calculus
transcription of the Fitch-style Natural Deduction proof of Theorem 5 of
Section 14 of [Margaris] p. 59 (which is notnotr 130). The same proof
may also be interpreted as a Virtual Deduction Hilbert-style
axiomatic proof. It was completed automatically by the tools program
completeusersproof.cmd, which invokes Mel L. O'Cat's mmj2 and Norm
Megill's Metamath Proof Assistant. notnotrALT 42102 is notnotrALTVD 42488
without virtual deductions and was automatically derived
from notnotrALTVD 42488. Step i of the User's Proof corresponds to
step i of the Fitch-style proof.
1:: | ⊢ ( ¬ ¬ 𝜑 ▶ ¬ ¬ 𝜑 )
| 2:: | ⊢ (¬ ¬ 𝜑 → (¬ 𝜑 → ¬ ¬ ¬ 𝜑))
| 3:1: | ⊢ ( ¬ ¬ 𝜑 ▶ (¬ 𝜑 → ¬ ¬ ¬ 𝜑) )
| 4:: | ⊢ ((¬ 𝜑 → ¬ ¬ ¬ 𝜑) → (¬ ¬ 𝜑 →
𝜑))
| 5:3: | ⊢ ( ¬ ¬ 𝜑 ▶ (¬ ¬ 𝜑 → 𝜑) )
| 6:5,1: | ⊢ ( ¬ ¬ 𝜑 ▶ 𝜑 )
| qed:6: | ⊢ (¬ ¬ 𝜑 → 𝜑)
|
(Contributed by Alan Sare, 21-Apr-2013.) (Proof modification is
discouraged.) (New usage is discouraged.) |