MPE Home Metamath Proof Explorer < Previous   Next >
Nearby theorems
Mirrors  >  Home  >  MPE Home  >  Th. List  >  df-an Structured version   Visualization version   GIF version

Definition df-an 399
Description: Define conjunction (logical "and"). Definition of [Margaris] p. 49. When both the left and right operand are true, the result is true; when either is false, the result is false. For example, it is true that (2 = 2 ∧ 3 = 3). After we define the constant true (df-tru 1540) and the constant false (df-fal 1550), we will be able to prove these truth table values: ((⊤ ∧ ⊤) ↔ ⊤) (truantru 1570), ((⊤ ∧ ⊥) ↔ ⊥) (truanfal 1571), ((⊥ ∧ ⊤) ↔ ⊥) (falantru 1572), and ((⊥ ∧ ⊥) ↔ ⊥) (falanfal 1573).

This is our first use of the biconditional connective in a definition; we use the biconditional connective in place of the traditional "<=def=>", which means the same thing, except that we can manipulate the biconditional connective directly in proofs rather than having to rely on an informal definition substitution rule. Note that if we mechanically substitute ¬ (𝜑 → ¬ 𝜓) for (𝜑𝜓), we end up with an instance of previously proved theorem biid 263. This is the justification for the definition, along with the fact that it introduces a new symbol . Contrast with (df-or 844), (wi 4), (df-nan 1482), and (df-xor 1502). (Contributed by NM, 5-Jan-1993.)

Assertion
Ref Expression
df-an ((𝜑𝜓) ↔ ¬ (𝜑 → ¬ 𝜓))

Detailed syntax breakdown of Definition df-an
StepHypRef Expression
1 wph . . 3 wff 𝜑
2 wps . . 3 wff 𝜓
31, 2wa 398 . 2 wff (𝜑𝜓)
42wn 3 . . . 4 wff ¬ 𝜓
51, 4wi 4 . . 3 wff (𝜑 → ¬ 𝜓)
65wn 3 . 2 wff ¬ (𝜑 → ¬ 𝜓)
73, 6wb 208 1 wff ((𝜑𝜓) ↔ ¬ (𝜑 → ¬ 𝜓))
Colors of variables: wff setvar class
This definition is referenced by:  pm4.63  400  imnan  402  imp  409  ex  415  dfbi2  477  pm5.32  576  pm4.54  983  nfand  1898  nfan1  2200  sbanOLD  2312  sbanvOLD  2326  sbanALT  2610  dfac5lem4  9552  kmlem3  9578  axrepprim  32928  axunprim  32929  axregprim  32931  axinfprim  32932  axacprim  32933  nolt02o  33199  dfxor4  40131  df3an2  40134  expandan  40644  ismnuprim  40650  pm11.52  40739
  Copyright terms: Public domain W3C validator