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

Theorem nnne0 12291
Description: A positive integer is nonzero. See nnne0ALT 12295 for a shorter proof using ax-pre-mulgt0 11225. This proof avoids 0lt1 11776, and thus ax-pre-mulgt0 11225, by splitting ax-1ne0 11217 into the two separate cases 0 < 1 and 1 < 0. (Contributed by NM, 27-Sep-1999.) Remove dependency on ax-pre-mulgt0 11225. (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 11217 . . 3 1 ≠ 0
2 1re 11254 . . . 4 1 ∈ ℝ
3 0re 11256 . . . 4 0 ∈ ℝ
42, 3lttri2i 11368 . . 3 (1 ≠ 0 ↔ (1 < 0 ∨ 0 < 1))
51, 4mpbi 229 . 2 (1 < 0 ∨ 0 < 1)
6 breq1 5148 . . . . . . 7 (𝑥 = 1 → (𝑥 < 0 ↔ 1 < 0))
76imbi2d 339 . . . . . 6 (𝑥 = 1 → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → 1 < 0)))
8 breq1 5148 . . . . . . 7 (𝑥 = 𝑦 → (𝑥 < 0 ↔ 𝑦 < 0))
98imbi2d 339 . . . . . 6 (𝑥 = 𝑦 → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → 𝑦 < 0)))
10 breq1 5148 . . . . . . 7 (𝑥 = (𝑦 + 1) → (𝑥 < 0 ↔ (𝑦 + 1) < 0))
1110imbi2d 339 . . . . . 6 (𝑥 = (𝑦 + 1) → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → (𝑦 + 1) < 0)))
12 breq1 5148 . . . . . . 7 (𝑥 = 𝐴 → (𝑥 < 0 ↔ 𝐴 < 0))
1312imbi2d 339 . . . . . 6 (𝑥 = 𝐴 → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → 𝐴 < 0)))
14 id 22 . . . . . 6 (1 < 0 → 1 < 0)
15 simp1 1133 . . . . . . . . . . 11 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 𝑦 ∈ ℕ)
1615nnred 12272 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 𝑦 ∈ ℝ)
17 1red 11255 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 1 ∈ ℝ)
1816, 17readdcld 11283 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (𝑦 + 1) ∈ ℝ)
193, 2readdcli 11269 . . . . . . . . . 10 (0 + 1) ∈ ℝ
2019a1i 11 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (0 + 1) ∈ ℝ)
21 0red 11257 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 0 ∈ ℝ)
22 simp3 1135 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 𝑦 < 0)
2316, 21, 17, 22ltadd1dd 11865 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (𝑦 + 1) < (0 + 1))
24 ax-1cn 11206 . . . . . . . . . . 11 1 ∈ ℂ
2524addlidi 11442 . . . . . . . . . 10 (0 + 1) = 1
26 simp2 1134 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 1 < 0)
2725, 26eqbrtrid 5180 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (0 + 1) < 0)
2818, 20, 21, 23, 27lttrd 11415 . . . . . . . 8 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (𝑦 + 1) < 0)
29283exp 1116 . . . . . . 7 (𝑦 ∈ ℕ → (1 < 0 → (𝑦 < 0 → (𝑦 + 1) < 0)))
3029a2d 29 . . . . . 6 (𝑦 ∈ ℕ → ((1 < 0 → 𝑦 < 0) → (1 < 0 → (𝑦 + 1) < 0)))
317, 9, 11, 13, 14, 30nnind 12275 . . . . 5 (𝐴 ∈ ℕ → (1 < 0 → 𝐴 < 0))
3231imp 405 . . . 4 ((𝐴 ∈ ℕ ∧ 1 < 0) → 𝐴 < 0)
3332lt0ne0d 11819 . . 3 ((𝐴 ∈ ℕ ∧ 1 < 0) → 𝐴 ≠ 0)
34 breq2 5149 . . . . . . 7 (𝑥 = 1 → (0 < 𝑥 ↔ 0 < 1))
3534imbi2d 339 . . . . . 6 (𝑥 = 1 → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < 1)))
36 breq2 5149 . . . . . . 7 (𝑥 = 𝑦 → (0 < 𝑥 ↔ 0 < 𝑦))
3736imbi2d 339 . . . . . 6 (𝑥 = 𝑦 → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < 𝑦)))
38 breq2 5149 . . . . . . 7 (𝑥 = (𝑦 + 1) → (0 < 𝑥 ↔ 0 < (𝑦 + 1)))
3938imbi2d 339 . . . . . 6 (𝑥 = (𝑦 + 1) → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < (𝑦 + 1))))
40 breq2 5149 . . . . . . 7 (𝑥 = 𝐴 → (0 < 𝑥 ↔ 0 < 𝐴))
4140imbi2d 339 . . . . . 6 (𝑥 = 𝐴 → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < 𝐴)))
42 id 22 . . . . . 6 (0 < 1 → 0 < 1)
43 simp1 1133 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 𝑦 ∈ ℕ)
4443nnred 12272 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 𝑦 ∈ ℝ)
45 1red 11255 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 1 ∈ ℝ)
46 simp3 1135 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 0 < 𝑦)
47 simp2 1134 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 0 < 1)
4844, 45, 46, 47addgt0d 11829 . . . . . . . 8 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 0 < (𝑦 + 1))
49483exp 1116 . . . . . . 7 (𝑦 ∈ ℕ → (0 < 1 → (0 < 𝑦 → 0 < (𝑦 + 1))))
5049a2d 29 . . . . . 6 (𝑦 ∈ ℕ → ((0 < 1 → 0 < 𝑦) → (0 < 1 → 0 < (𝑦 + 1))))
5135, 37, 39, 41, 42, 50nnind 12275 . . . . 5 (𝐴 ∈ ℕ → (0 < 1 → 0 < 𝐴))
5251imp 405 . . . 4 ((𝐴 ∈ ℕ ∧ 0 < 1) → 0 < 𝐴)
5352gt0ne0d 11818 . . 3 ((𝐴 ∈ ℕ ∧ 0 < 1) → 𝐴 ≠ 0)
5433, 53jaodan 955 . 2 ((𝐴 ∈ ℕ ∧ (1 < 0 ∨ 0 < 1)) → 𝐴 ≠ 0)
555, 54mpan2 689 1 (𝐴 ∈ ℕ → 𝐴 ≠ 0)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 394  wo 845  w3a 1084   = wceq 1534  wcel 2099  wne 2930   class class class wbr 5145  (class class class)co 7415  cr 11147  0cc0 11148  1c1 11149   + caddc 11151   < clt 11288  cn 12257
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1790  ax-4 1804  ax-5 1906  ax-6 1964  ax-7 2004  ax-8 2101  ax-9 2109  ax-10 2130  ax-11 2147  ax-12 2167  ax-ext 2697  ax-sep 5296  ax-nul 5303  ax-pow 5361  ax-pr 5425  ax-un 7737  ax-resscn 11205  ax-1cn 11206  ax-icn 11207  ax-addcl 11208  ax-addrcl 11209  ax-mulcl 11210  ax-mulrcl 11211  ax-mulcom 11212  ax-addass 11213  ax-mulass 11214  ax-distr 11215  ax-i2m1 11216  ax-1ne0 11217  ax-1rid 11218  ax-rnegex 11219  ax-rrecex 11220  ax-cnre 11221  ax-pre-lttri 11222  ax-pre-lttrn 11223  ax-pre-ltadd 11224
This theorem depends on definitions:  df-bi 206  df-an 395  df-or 846  df-3or 1085  df-3an 1086  df-tru 1537  df-fal 1547  df-ex 1775  df-nf 1779  df-sb 2061  df-mo 2529  df-eu 2558  df-clab 2704  df-cleq 2718  df-clel 2803  df-nfc 2878  df-ne 2931  df-nel 3037  df-ral 3052  df-rex 3061  df-reu 3366  df-rab 3421  df-v 3466  df-sbc 3778  df-csb 3894  df-dif 3951  df-un 3953  df-in 3955  df-ss 3965  df-pss 3968  df-nul 4325  df-if 4526  df-pw 4601  df-sn 4626  df-pr 4628  df-op 4632  df-uni 4908  df-iun 4997  df-br 5146  df-opab 5208  df-mpt 5229  df-tr 5263  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 6304  df-ord 6370  df-on 6371  df-lim 6372  df-suc 6373  df-iota 6497  df-fun 6547  df-fn 6548  df-f 6549  df-f1 6550  df-fo 6551  df-f1o 6552  df-fv 6553  df-ov 7418  df-om 7868  df-2nd 7995  df-frecs 8287  df-wrecs 8318  df-recs 8392  df-rdg 8431  df-er 8725  df-en 8966  df-dom 8967  df-sdom 8968  df-pnf 11290  df-mnf 11291  df-xr 11292  df-ltxr 11293  df-le 11294  df-nn 12258
This theorem is referenced by:  nnneneg  12292  0nnn  12293  nndivre  12298  nndiv  12303  nndivtr  12304  nnne0d  12307  zdiv  12677  zdivadd  12678  zdivmul  12679  elq  12979  qmulz  12980  qre  12982  qaddcl  12994  qnegcl  12995  qmulcl  12996  qreccl  12998  rpnnen1lem5  13010  nn0ledivnn  13134  fzo1fzo0n0  13730  quoremz  13868  quoremnn0ALT  13870  intfracq  13872  fldiv  13873  fldiv2  13874  modmulnn  13902  modsumfzodifsn  13957  expnnval  14077  expneg  14082  digit2  14247  facdiv  14298  facndiv  14299  bcm1k  14326  bcp1n  14327  bcval5  14329  hashnncl  14377  cshwidxmod  14805  relexpsucnnr  15024  divcnv  15851  harmonic  15857  expcnv  15862  ef0lem  16074  ruclem6  16231  sqrt2irr  16245  dvdsval3  16254  nndivdvds  16259  modmulconst  16284  dvdsdivcl  16312  dvdsflip  16313  divalg2  16401  divalgmod  16402  ndvdssub  16405  nndvdslegcd  16499  divgcdz  16505  divgcdnn  16509  modgcd  16527  gcddiv  16546  gcdzeq  16547  eucalgf  16578  eucalginv  16579  lcmgcdlem  16601  lcmftp  16631  qredeq  16652  qredeu  16653  cncongr1  16662  cncongr2  16663  isprm6  16709  divnumden  16744  divdenle  16745  phimullem  16775  hashgcdlem  16784  phisum  16786  prm23lt5  16810  pythagtriplem10  16816  pythagtriplem8  16819  pythagtriplem9  16820  pccl  16845  pcdiv  16848  pcqcl  16852  pcdvds  16860  pcndvds  16862  pcndvds2  16864  pceq0  16867  pcneg  16870  pcz  16877  pcmpt  16888  fldivp1  16893  pcfac  16895  oddprmdvds  16899  infpnlem2  16907  cshwshashlem1  17092  smndex1n0mnd  18896  mulgnn  19064  mulgnegnn  19073  mulgmodid  19102  oddvdsnn0  19537  odmulgeq  19550  gexnnod  19581  qsssubdrg  21418  prmirredlem  21457  znf1o  21544  znhash  21551  znidomb  21554  znunithash  21557  znrrg  21558  cply1coe0  22288  cply1coe0bi  22289  m2cpm  22730  m2cpminvid2lem  22743  fvmptnn04ifc  22841  vitali  25629  mbfi1fseqlem3  25734  dvexp2  25973  plyeq0lem  26233  abelthlem9  26466  logtayllem  26682  logtayl  26683  logtaylsum  26684  logtayl2  26685  cxpexp  26691  cxproot  26713  root1id  26778  root1eq1  26779  cxpeq  26781  logbgcd1irr  26818  atantayl  26961  atantayl2  26962  leibpilem2  26965  leibpi  26966  birthdaylem2  26976  birthdaylem3  26977  dfef2  26995  emcllem2  27021  emcllem3  27022  zetacvg  27039  lgam1  27088  basellem4  27108  basellem8  27112  basellem9  27113  mumullem2  27204  fsumdvdscom  27209  chtublem  27236  dchrelbas4  27268  bclbnd  27305  lgsval4a  27344  lgsabs1  27361  lgssq2  27363  dchrmusumlema  27518  dchrmusum2  27519  dchrvmasumiflem1  27526  dchrvmaeq0  27529  dchrisum0flblem1  27533  dchrisum0flblem2  27534  dchrisum0re  27538  ostthlem1  27652  ostth1  27658  pthdlem2lem  29700  wspthsnonn0vne  29847  clwwisshclwwslem  29943  ipasslem4  30763  ipasslem5  30764  divnumden2  32718  1fldgenq  33176  qqhval2  33809  qqhnm  33817  signstfveq0  34435  subfacp1lem6  35025  circum  35514  fz0n  35565  divcnvlin  35567  iprodgam  35576  faclim  35580  nndivsub  36181  poimirlem29  37362  poimirlem31  37364  poimirlem32  37365  heiborlem4  37527  heiborlem6  37529  nnproddivdvdsd  41711  pellexlem1  42522  congrep  42667  jm2.20nn  42691  proot1ex  42897  hashnzfzclim  44032  binomcxplemnotnn0  44066  nnne1ge2  44941  mccllem  45253  clim1fr1  45257  dvnxpaek  45598  dvnprodlem2  45603  wallispilem5  45725  wallispi2lem1  45727  stirlinglem1  45730  stirlinglem3  45732  stirlinglem4  45733  stirlinglem5  45734  stirlinglem7  45736  stirlinglem10  45739  stirlinglem12  45741  stirlinglem14  45743  stirlinglem15  45744  fouriersw  45887  vonioolem2  46337  vonicclem2  46340  iccpartiltu  47029  divgcdoddALTV  47289  fpprwppr  47346  nnsgrpnmnd  47590  eluz2cnn0n1  47929  mod0mul  47942  modn0mul  47943  blennn  47998  nnpw2blen  48003  digvalnn0  48022  nn0digval  48023  dignn0fr  48024  dignn0ldlem  48025  dig0  48029
  Copyright terms: Public domain W3C validator