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

Theorem nnne0 12241
Description: A positive integer is nonzero. See nnne0ALT 12245 for a shorter proof using ax-pre-mulgt0 11182. This proof avoids 0lt1 11731, and thus ax-pre-mulgt0 11182, by splitting ax-1ne0 11174 into the two separate cases 0 < 1 and 1 < 0. (Contributed by NM, 27-Sep-1999.) Remove dependency on ax-pre-mulgt0 11182. (Revised by Steven Nguyen, 30-Jan-2023.)
Assertion
Ref Expression
nnne0 (𝐴 ∈ ℕ → 𝐴 ≠ 0)

Proof of Theorem nnne0
Dummy variables 𝑥 𝑦 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 ax-1ne0 11174 . . 3 1 ≠ 0
2 1re 11209 . . . 4 1 ∈ ℝ
3 0re 11211 . . . 4 0 ∈ ℝ
42, 3lttri2i 11323 . . 3 (1 ≠ 0 ↔ (1 < 0 ∨ 0 < 1))
51, 4mpbi 229 . 2 (1 < 0 ∨ 0 < 1)
6 breq1 5149 . . . . . . 7 (𝑥 = 1 → (𝑥 < 0 ↔ 1 < 0))
76imbi2d 341 . . . . . 6 (𝑥 = 1 → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → 1 < 0)))
8 breq1 5149 . . . . . . 7 (𝑥 = 𝑦 → (𝑥 < 0 ↔ 𝑦 < 0))
98imbi2d 341 . . . . . 6 (𝑥 = 𝑦 → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → 𝑦 < 0)))
10 breq1 5149 . . . . . . 7 (𝑥 = (𝑦 + 1) → (𝑥 < 0 ↔ (𝑦 + 1) < 0))
1110imbi2d 341 . . . . . 6 (𝑥 = (𝑦 + 1) → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → (𝑦 + 1) < 0)))
12 breq1 5149 . . . . . . 7 (𝑥 = 𝐴 → (𝑥 < 0 ↔ 𝐴 < 0))
1312imbi2d 341 . . . . . 6 (𝑥 = 𝐴 → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → 𝐴 < 0)))
14 id 22 . . . . . 6 (1 < 0 → 1 < 0)
15 simp1 1137 . . . . . . . . . . 11 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 𝑦 ∈ ℕ)
1615nnred 12222 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 𝑦 ∈ ℝ)
17 1red 11210 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 1 ∈ ℝ)
1816, 17readdcld 11238 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (𝑦 + 1) ∈ ℝ)
193, 2readdcli 11224 . . . . . . . . . 10 (0 + 1) ∈ ℝ
2019a1i 11 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (0 + 1) ∈ ℝ)
21 0red 11212 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 0 ∈ ℝ)
22 simp3 1139 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 𝑦 < 0)
2316, 21, 17, 22ltadd1dd 11820 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (𝑦 + 1) < (0 + 1))
24 ax-1cn 11163 . . . . . . . . . . 11 1 ∈ ℂ
2524addlidi 11397 . . . . . . . . . 10 (0 + 1) = 1
26 simp2 1138 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 1 < 0)
2725, 26eqbrtrid 5181 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (0 + 1) < 0)
2818, 20, 21, 23, 27lttrd 11370 . . . . . . . 8 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (𝑦 + 1) < 0)
29283exp 1120 . . . . . . 7 (𝑦 ∈ ℕ → (1 < 0 → (𝑦 < 0 → (𝑦 + 1) < 0)))
3029a2d 29 . . . . . 6 (𝑦 ∈ ℕ → ((1 < 0 → 𝑦 < 0) → (1 < 0 → (𝑦 + 1) < 0)))
317, 9, 11, 13, 14, 30nnind 12225 . . . . 5 (𝐴 ∈ ℕ → (1 < 0 → 𝐴 < 0))
3231imp 408 . . . 4 ((𝐴 ∈ ℕ ∧ 1 < 0) → 𝐴 < 0)
3332lt0ne0d 11774 . . 3 ((𝐴 ∈ ℕ ∧ 1 < 0) → 𝐴 ≠ 0)
34 breq2 5150 . . . . . . 7 (𝑥 = 1 → (0 < 𝑥 ↔ 0 < 1))
3534imbi2d 341 . . . . . 6 (𝑥 = 1 → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < 1)))
36 breq2 5150 . . . . . . 7 (𝑥 = 𝑦 → (0 < 𝑥 ↔ 0 < 𝑦))
3736imbi2d 341 . . . . . 6 (𝑥 = 𝑦 → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < 𝑦)))
38 breq2 5150 . . . . . . 7 (𝑥 = (𝑦 + 1) → (0 < 𝑥 ↔ 0 < (𝑦 + 1)))
3938imbi2d 341 . . . . . 6 (𝑥 = (𝑦 + 1) → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < (𝑦 + 1))))
40 breq2 5150 . . . . . . 7 (𝑥 = 𝐴 → (0 < 𝑥 ↔ 0 < 𝐴))
4140imbi2d 341 . . . . . 6 (𝑥 = 𝐴 → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < 𝐴)))
42 id 22 . . . . . 6 (0 < 1 → 0 < 1)
43 simp1 1137 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 𝑦 ∈ ℕ)
4443nnred 12222 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 𝑦 ∈ ℝ)
45 1red 11210 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 1 ∈ ℝ)
46 simp3 1139 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 0 < 𝑦)
47 simp2 1138 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 0 < 1)
4844, 45, 46, 47addgt0d 11784 . . . . . . . 8 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 0 < (𝑦 + 1))
49483exp 1120 . . . . . . 7 (𝑦 ∈ ℕ → (0 < 1 → (0 < 𝑦 → 0 < (𝑦 + 1))))
5049a2d 29 . . . . . 6 (𝑦 ∈ ℕ → ((0 < 1 → 0 < 𝑦) → (0 < 1 → 0 < (𝑦 + 1))))
5135, 37, 39, 41, 42, 50nnind 12225 . . . . 5 (𝐴 ∈ ℕ → (0 < 1 → 0 < 𝐴))
5251imp 408 . . . 4 ((𝐴 ∈ ℕ ∧ 0 < 1) → 0 < 𝐴)
5352gt0ne0d 11773 . . 3 ((𝐴 ∈ ℕ ∧ 0 < 1) → 𝐴 ≠ 0)
5433, 53jaodan 957 . 2 ((𝐴 ∈ ℕ ∧ (1 < 0 ∨ 0 < 1)) → 𝐴 ≠ 0)
555, 54mpan2 690 1 (𝐴 ∈ ℕ → 𝐴 ≠ 0)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 397  wo 846  w3a 1088   = wceq 1542  wcel 2107  wne 2941   class class class wbr 5146  (class class class)co 7403  cr 11104  0cc0 11105  1c1 11106   + caddc 11108   < clt 11243  cn 12207
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1798  ax-4 1812  ax-5 1914  ax-6 1972  ax-7 2012  ax-8 2109  ax-9 2117  ax-10 2138  ax-11 2155  ax-12 2172  ax-ext 2704  ax-sep 5297  ax-nul 5304  ax-pow 5361  ax-pr 5425  ax-un 7719  ax-resscn 11162  ax-1cn 11163  ax-icn 11164  ax-addcl 11165  ax-addrcl 11166  ax-mulcl 11167  ax-mulrcl 11168  ax-mulcom 11169  ax-addass 11170  ax-mulass 11171  ax-distr 11172  ax-i2m1 11173  ax-1ne0 11174  ax-1rid 11175  ax-rnegex 11176  ax-rrecex 11177  ax-cnre 11178  ax-pre-lttri 11179  ax-pre-lttrn 11180  ax-pre-ltadd 11181
This theorem depends on definitions:  df-bi 206  df-an 398  df-or 847  df-3or 1089  df-3an 1090  df-tru 1545  df-fal 1555  df-ex 1783  df-nf 1787  df-sb 2069  df-mo 2535  df-eu 2564  df-clab 2711  df-cleq 2725  df-clel 2811  df-nfc 2886  df-ne 2942  df-nel 3048  df-ral 3063  df-rex 3072  df-reu 3378  df-rab 3434  df-v 3477  df-sbc 3776  df-csb 3892  df-dif 3949  df-un 3951  df-in 3953  df-ss 3963  df-pss 3965  df-nul 4321  df-if 4527  df-pw 4602  df-sn 4627  df-pr 4629  df-op 4633  df-uni 4907  df-iun 4997  df-br 5147  df-opab 5209  df-mpt 5230  df-tr 5264  df-id 5572  df-eprel 5578  df-po 5586  df-so 5587  df-fr 5629  df-we 5631  df-xp 5680  df-rel 5681  df-cnv 5682  df-co 5683  df-dm 5684  df-rn 5685  df-res 5686  df-ima 5687  df-pred 6296  df-ord 6363  df-on 6364  df-lim 6365  df-suc 6366  df-iota 6491  df-fun 6541  df-fn 6542  df-f 6543  df-f1 6544  df-fo 6545  df-f1o 6546  df-fv 6547  df-ov 7406  df-om 7850  df-2nd 7970  df-frecs 8260  df-wrecs 8291  df-recs 8365  df-rdg 8404  df-er 8698  df-en 8935  df-dom 8936  df-sdom 8937  df-pnf 11245  df-mnf 11246  df-xr 11247  df-ltxr 11248  df-le 11249  df-nn 12208
This theorem is referenced by:  nnneneg  12242  0nnn  12243  nndivre  12248  nndiv  12253  nndivtr  12254  nnne0d  12257  zdiv  12627  zdivadd  12628  zdivmul  12629  elq  12929  qmulz  12930  qre  12932  qaddcl  12944  qnegcl  12945  qmulcl  12946  qreccl  12948  rpnnen1lem5  12960  nn0ledivnn  13082  fzo1fzo0n0  13678  quoremz  13815  quoremnn0ALT  13817  intfracq  13819  fldiv  13820  fldiv2  13821  modmulnn  13849  modsumfzodifsn  13904  expnnval  14025  expneg  14030  digit2  14194  facdiv  14242  facndiv  14243  bcm1k  14270  bcp1n  14271  bcval5  14273  hashnncl  14321  cshwidxmod  14748  relexpsucnnr  14967  divcnv  15794  harmonic  15800  expcnv  15805  ef0lem  16017  ruclem6  16173  sqrt2irr  16187  dvdsval3  16196  nndivdvds  16201  modmulconst  16226  dvdsdivcl  16254  dvdsflip  16255  divalg2  16343  divalgmod  16344  ndvdssub  16347  nndvdslegcd  16441  divgcdz  16447  divgcdnn  16451  modgcd  16469  gcddiv  16488  gcdzeq  16489  eucalgf  16515  eucalginv  16516  lcmgcdlem  16538  lcmftp  16568  qredeq  16589  qredeu  16590  cncongr1  16599  cncongr2  16600  isprm6  16646  divnumden  16679  divdenle  16680  phimullem  16707  hashgcdlem  16716  phisum  16718  prm23lt5  16742  pythagtriplem10  16748  pythagtriplem8  16751  pythagtriplem9  16752  pccl  16777  pcdiv  16780  pcqcl  16784  pcdvds  16792  pcndvds  16794  pcndvds2  16796  pceq0  16799  pcneg  16802  pcz  16809  pcmpt  16820  fldivp1  16825  pcfac  16827  oddprmdvds  16831  infpnlem2  16839  cshwshashlem1  17024  smndex1n0mnd  18788  mulgnn  18951  mulgnegnn  18957  mulgmodid  18986  oddvdsnn0  19404  odmulgeq  19417  gexnnod  19448  qsssubdrg  20988  prmirredlem  21025  znf1o  21090  znhash  21097  znidomb  21100  znunithash  21103  znrrg  21104  cply1coe0  21804  cply1coe0bi  21805  m2cpm  22224  m2cpminvid2lem  22237  fvmptnn04ifc  22335  vitali  25111  mbfi1fseqlem3  25216  dvexp2  25452  plyeq0lem  25705  abelthlem9  25933  logtayllem  26148  logtayl  26149  logtaylsum  26150  logtayl2  26151  cxpexp  26157  cxproot  26179  root1id  26241  root1eq1  26242  cxpeq  26244  logbgcd1irr  26278  atantayl  26421  atantayl2  26422  leibpilem2  26425  leibpi  26426  birthdaylem2  26436  birthdaylem3  26437  dfef2  26454  emcllem2  26480  emcllem3  26481  zetacvg  26498  lgam1  26547  basellem4  26567  basellem8  26571  basellem9  26572  mumullem2  26663  fsumdvdscom  26668  chtublem  26693  dchrelbas4  26725  bclbnd  26762  lgsval4a  26801  lgsabs1  26818  lgssq2  26820  dchrmusumlema  26975  dchrmusum2  26976  dchrvmasumiflem1  26983  dchrvmaeq0  26986  dchrisum0flblem1  26990  dchrisum0flblem2  26991  dchrisum0re  26995  ostthlem1  27109  ostth1  27115  pthdlem2lem  29003  wspthsnonn0vne  29150  clwwisshclwwslem  29246  ipasslem4  30064  ipasslem5  30065  divnumden2  32001  1fldgenq  32380  qqhval2  32899  qqhnm  32907  signstfveq0  33525  subfacp1lem6  34113  circum  34596  fz0n  34637  divcnvlin  34639  iprodgam  34649  faclim  34653  nndivsub  35279  poimirlem29  36454  poimirlem31  36456  poimirlem32  36457  heiborlem4  36619  heiborlem6  36621  nnproddivdvdsd  40803  pellexlem1  41499  congrep  41644  jm2.20nn  41668  proot1ex  41875  hashnzfzclim  43013  binomcxplemnotnn0  43047  nnne1ge2  43935  mccllem  44247  clim1fr1  44251  dvnxpaek  44592  dvnprodlem2  44597  wallispilem5  44719  wallispi2lem1  44721  stirlinglem1  44724  stirlinglem3  44726  stirlinglem4  44727  stirlinglem5  44728  stirlinglem7  44730  stirlinglem10  44733  stirlinglem12  44735  stirlinglem14  44737  stirlinglem15  44738  fouriersw  44881  vonioolem2  45331  vonicclem2  45334  iccpartiltu  46024  divgcdoddALTV  46284  fpprwppr  46341  nnsgrpnmnd  46522  eluz2cnn0n1  47093  mod0mul  47106  modn0mul  47107  blennn  47162  nnpw2blen  47167  digvalnn0  47186  nn0digval  47187  dignn0fr  47188  dignn0ldlem  47189  dig0  47193
  Copyright terms: Public domain W3C validator