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

Theorem nnne0 12246
Description: A positive integer is nonzero. See nnne0ALT 12250 for a shorter proof using ax-pre-mulgt0 11187. This proof avoids 0lt1 11736, and thus ax-pre-mulgt0 11187, by splitting ax-1ne0 11179 into the two separate cases 0 < 1 and 1 < 0. (Contributed by NM, 27-Sep-1999.) Remove dependency on ax-pre-mulgt0 11187. (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 11179 . . 3 1 ≠ 0
2 1re 11214 . . . 4 1 ∈ ℝ
3 0re 11216 . . . 4 0 ∈ ℝ
42, 3lttri2i 11328 . . 3 (1 ≠ 0 ↔ (1 < 0 ∨ 0 < 1))
51, 4mpbi 229 . 2 (1 < 0 ∨ 0 < 1)
6 breq1 5152 . . . . . . 7 (𝑥 = 1 → (𝑥 < 0 ↔ 1 < 0))
76imbi2d 341 . . . . . 6 (𝑥 = 1 → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → 1 < 0)))
8 breq1 5152 . . . . . . 7 (𝑥 = 𝑦 → (𝑥 < 0 ↔ 𝑦 < 0))
98imbi2d 341 . . . . . 6 (𝑥 = 𝑦 → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → 𝑦 < 0)))
10 breq1 5152 . . . . . . 7 (𝑥 = (𝑦 + 1) → (𝑥 < 0 ↔ (𝑦 + 1) < 0))
1110imbi2d 341 . . . . . 6 (𝑥 = (𝑦 + 1) → ((1 < 0 → 𝑥 < 0) ↔ (1 < 0 → (𝑦 + 1) < 0)))
12 breq1 5152 . . . . . . 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 12227 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 𝑦 ∈ ℝ)
17 1red 11215 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 1 ∈ ℝ)
1816, 17readdcld 11243 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (𝑦 + 1) ∈ ℝ)
193, 2readdcli 11229 . . . . . . . . . 10 (0 + 1) ∈ ℝ
2019a1i 11 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (0 + 1) ∈ ℝ)
21 0red 11217 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 0 ∈ ℝ)
22 simp3 1139 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 𝑦 < 0)
2316, 21, 17, 22ltadd1dd 11825 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (𝑦 + 1) < (0 + 1))
24 ax-1cn 11168 . . . . . . . . . . 11 1 ∈ ℂ
2524addlidi 11402 . . . . . . . . . 10 (0 + 1) = 1
26 simp2 1138 . . . . . . . . . 10 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → 1 < 0)
2725, 26eqbrtrid 5184 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 1 < 0 ∧ 𝑦 < 0) → (0 + 1) < 0)
2818, 20, 21, 23, 27lttrd 11375 . . . . . . . 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 12230 . . . . 5 (𝐴 ∈ ℕ → (1 < 0 → 𝐴 < 0))
3231imp 408 . . . 4 ((𝐴 ∈ ℕ ∧ 1 < 0) → 𝐴 < 0)
3332lt0ne0d 11779 . . 3 ((𝐴 ∈ ℕ ∧ 1 < 0) → 𝐴 ≠ 0)
34 breq2 5153 . . . . . . 7 (𝑥 = 1 → (0 < 𝑥 ↔ 0 < 1))
3534imbi2d 341 . . . . . 6 (𝑥 = 1 → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < 1)))
36 breq2 5153 . . . . . . 7 (𝑥 = 𝑦 → (0 < 𝑥 ↔ 0 < 𝑦))
3736imbi2d 341 . . . . . 6 (𝑥 = 𝑦 → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < 𝑦)))
38 breq2 5153 . . . . . . 7 (𝑥 = (𝑦 + 1) → (0 < 𝑥 ↔ 0 < (𝑦 + 1)))
3938imbi2d 341 . . . . . 6 (𝑥 = (𝑦 + 1) → ((0 < 1 → 0 < 𝑥) ↔ (0 < 1 → 0 < (𝑦 + 1))))
40 breq2 5153 . . . . . . 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 12227 . . . . . . . . 9 ((𝑦 ∈ ℕ ∧ 0 < 1 ∧ 0 < 𝑦) → 𝑦 ∈ ℝ)
45 1red 11215 . . . . . . . . 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 11789 . . . . . . . 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 12230 . . . . 5 (𝐴 ∈ ℕ → (0 < 1 → 0 < 𝐴))
5251imp 408 . . . 4 ((𝐴 ∈ ℕ ∧ 0 < 1) → 0 < 𝐴)
5352gt0ne0d 11778 . . 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 5149  (class class class)co 7409  cr 11109  0cc0 11110  1c1 11111   + caddc 11113   < clt 11248  cn 12212
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 5300  ax-nul 5307  ax-pow 5364  ax-pr 5428  ax-un 7725  ax-resscn 11167  ax-1cn 11168  ax-icn 11169  ax-addcl 11170  ax-addrcl 11171  ax-mulcl 11172  ax-mulrcl 11173  ax-mulcom 11174  ax-addass 11175  ax-mulass 11176  ax-distr 11177  ax-i2m1 11178  ax-1ne0 11179  ax-1rid 11180  ax-rnegex 11181  ax-rrecex 11182  ax-cnre 11183  ax-pre-lttri 11184  ax-pre-lttrn 11185  ax-pre-ltadd 11186
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 3779  df-csb 3895  df-dif 3952  df-un 3954  df-in 3956  df-ss 3966  df-pss 3968  df-nul 4324  df-if 4530  df-pw 4605  df-sn 4630  df-pr 4632  df-op 4636  df-uni 4910  df-iun 5000  df-br 5150  df-opab 5212  df-mpt 5233  df-tr 5267  df-id 5575  df-eprel 5581  df-po 5589  df-so 5590  df-fr 5632  df-we 5634  df-xp 5683  df-rel 5684  df-cnv 5685  df-co 5686  df-dm 5687  df-rn 5688  df-res 5689  df-ima 5690  df-pred 6301  df-ord 6368  df-on 6369  df-lim 6370  df-suc 6371  df-iota 6496  df-fun 6546  df-fn 6547  df-f 6548  df-f1 6549  df-fo 6550  df-f1o 6551  df-fv 6552  df-ov 7412  df-om 7856  df-2nd 7976  df-frecs 8266  df-wrecs 8297  df-recs 8371  df-rdg 8410  df-er 8703  df-en 8940  df-dom 8941  df-sdom 8942  df-pnf 11250  df-mnf 11251  df-xr 11252  df-ltxr 11253  df-le 11254  df-nn 12213
This theorem is referenced by:  nnneneg  12247  0nnn  12248  nndivre  12253  nndiv  12258  nndivtr  12259  nnne0d  12262  zdiv  12632  zdivadd  12633  zdivmul  12634  elq  12934  qmulz  12935  qre  12937  qaddcl  12949  qnegcl  12950  qmulcl  12951  qreccl  12953  rpnnen1lem5  12965  nn0ledivnn  13087  fzo1fzo0n0  13683  quoremz  13820  quoremnn0ALT  13822  intfracq  13824  fldiv  13825  fldiv2  13826  modmulnn  13854  modsumfzodifsn  13909  expnnval  14030  expneg  14035  digit2  14199  facdiv  14247  facndiv  14248  bcm1k  14275  bcp1n  14276  bcval5  14278  hashnncl  14326  cshwidxmod  14753  relexpsucnnr  14972  divcnv  15799  harmonic  15805  expcnv  15810  ef0lem  16022  ruclem6  16178  sqrt2irr  16192  dvdsval3  16201  nndivdvds  16206  modmulconst  16231  dvdsdivcl  16259  dvdsflip  16260  divalg2  16348  divalgmod  16349  ndvdssub  16352  nndvdslegcd  16446  divgcdz  16452  divgcdnn  16456  modgcd  16474  gcddiv  16493  gcdzeq  16494  eucalgf  16520  eucalginv  16521  lcmgcdlem  16543  lcmftp  16573  qredeq  16594  qredeu  16595  cncongr1  16604  cncongr2  16605  isprm6  16651  divnumden  16684  divdenle  16685  phimullem  16712  hashgcdlem  16721  phisum  16723  prm23lt5  16747  pythagtriplem10  16753  pythagtriplem8  16756  pythagtriplem9  16757  pccl  16782  pcdiv  16785  pcqcl  16789  pcdvds  16797  pcndvds  16799  pcndvds2  16801  pceq0  16804  pcneg  16807  pcz  16814  pcmpt  16825  fldivp1  16830  pcfac  16832  oddprmdvds  16836  infpnlem2  16844  cshwshashlem1  17029  smndex1n0mnd  18793  mulgnn  18958  mulgnegnn  18964  mulgmodid  18993  oddvdsnn0  19412  odmulgeq  19425  gexnnod  19456  qsssubdrg  21004  prmirredlem  21042  znf1o  21107  znhash  21114  znidomb  21117  znunithash  21120  znrrg  21121  cply1coe0  21823  cply1coe0bi  21824  m2cpm  22243  m2cpminvid2lem  22256  fvmptnn04ifc  22354  vitali  25130  mbfi1fseqlem3  25235  dvexp2  25471  plyeq0lem  25724  abelthlem9  25952  logtayllem  26167  logtayl  26168  logtaylsum  26169  logtayl2  26170  cxpexp  26176  cxproot  26198  root1id  26262  root1eq1  26263  cxpeq  26265  logbgcd1irr  26299  atantayl  26442  atantayl2  26443  leibpilem2  26446  leibpi  26447  birthdaylem2  26457  birthdaylem3  26458  dfef2  26475  emcllem2  26501  emcllem3  26502  zetacvg  26519  lgam1  26568  basellem4  26588  basellem8  26592  basellem9  26593  mumullem2  26684  fsumdvdscom  26689  chtublem  26714  dchrelbas4  26746  bclbnd  26783  lgsval4a  26822  lgsabs1  26839  lgssq2  26841  dchrmusumlema  26996  dchrmusum2  26997  dchrvmasumiflem1  27004  dchrvmaeq0  27007  dchrisum0flblem1  27011  dchrisum0flblem2  27012  dchrisum0re  27016  ostthlem1  27130  ostth1  27136  pthdlem2lem  29024  wspthsnonn0vne  29171  clwwisshclwwslem  29267  ipasslem4  30087  ipasslem5  30088  divnumden2  32024  1fldgenq  32412  qqhval2  32962  qqhnm  32970  signstfveq0  33588  subfacp1lem6  34176  circum  34659  fz0n  34700  divcnvlin  34702  iprodgam  34712  faclim  34716  nndivsub  35342  poimirlem29  36517  poimirlem31  36519  poimirlem32  36520  heiborlem4  36682  heiborlem6  36684  nnproddivdvdsd  40866  pellexlem1  41567  congrep  41712  jm2.20nn  41736  proot1ex  41943  hashnzfzclim  43081  binomcxplemnotnn0  43115  nnne1ge2  44001  mccllem  44313  clim1fr1  44317  dvnxpaek  44658  dvnprodlem2  44663  wallispilem5  44785  wallispi2lem1  44787  stirlinglem1  44790  stirlinglem3  44792  stirlinglem4  44793  stirlinglem5  44794  stirlinglem7  44796  stirlinglem10  44799  stirlinglem12  44801  stirlinglem14  44803  stirlinglem15  44804  fouriersw  44947  vonioolem2  45397  vonicclem2  45400  iccpartiltu  46090  divgcdoddALTV  46350  fpprwppr  46407  nnsgrpnmnd  46588  eluz2cnn0n1  47192  mod0mul  47205  modn0mul  47206  blennn  47261  nnpw2blen  47266  digvalnn0  47285  nn0digval  47286  dignn0fr  47287  dignn0ldlem  47288  dig0  47292
  Copyright terms: Public domain W3C validator