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 398
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 1545) and the constant false (df-fal 1555), we will be able to prove these truth table values: ((⊤ ∧ ⊤) ↔ ⊤) (truantru 1575), ((⊤ ∧ ⊥) ↔ ⊥) (truanfal 1576), ((⊥ ∧ ⊤) ↔ ⊥) (falantru 1577), and ((⊥ ∧ ⊥) ↔ ⊥) (falanfal 1578).

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 261. This is the justification for the definition, along with the fact that it introduces a new symbol . Contrast with (df-or 847), (wi 4), (df-nan 1491), and (df-xor 1511). (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 397 . 2 wff (𝜑𝜓)
42wn 3 . . . 4 wff ¬ 𝜓
51, 4wi 4 . . 3 wff (𝜑 → ¬ 𝜓)
65wn 3 . 2 wff ¬ (𝜑 → ¬ 𝜓)
73, 6wb 205 1 wff ((𝜑𝜓) ↔ ¬ (𝜑 → ¬ 𝜓))
Colors of variables: wff setvar class
This definition is referenced by:  pm4.63  399  imnan  401  imp  408  ex  414  dfbi2  476  pm5.32  575  pm4.54  986  nfand  1901  nfan1  2194  dfac5lem4  10117  kmlem3  10143  nolt02o  27178  axrepprim  34609  axunprim  34610  axregprim  34612  axinfprim  34613  axacprim  34614  orddif0suc  41951  dfxor4  42450  df3an2  42453  expandan  42980  ismnuprim  42986  pm11.52  43079
  Copyright terms: Public domain W3C validator