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

Theorem finds 7589
Description: Principle of Finite Induction (inference schema), using implicit substitutions. The first four hypotheses establish the substitutions we need. The last two are the basis and the induction step. Theorem Schema 22 of [Suppes] p. 136. This is Metamath 100 proof #74. (Contributed by NM, 14-Apr-1995.)
Hypotheses
Ref Expression
finds.1 (𝑥 = ∅ → (𝜑𝜓))
finds.2 (𝑥 = 𝑦 → (𝜑𝜒))
finds.3 (𝑥 = suc 𝑦 → (𝜑𝜃))
finds.4 (𝑥 = 𝐴 → (𝜑𝜏))
finds.5 𝜓
finds.6 (𝑦 ∈ ω → (𝜒𝜃))
Assertion
Ref Expression
finds (𝐴 ∈ ω → 𝜏)
Distinct variable groups:   𝑥,𝑦   𝑥,𝐴   𝜓,𝑥   𝜒,𝑥   𝜃,𝑥   𝜏,𝑥   𝜑,𝑦
Allowed substitution hints:   𝜑(𝑥)   𝜓(𝑦)   𝜒(𝑦)   𝜃(𝑦)   𝜏(𝑦)   𝐴(𝑦)

Proof of Theorem finds
StepHypRef Expression
1 finds.5 . . . . 5 𝜓
2 0ex 5175 . . . . . 6 ∅ ∈ V
3 finds.1 . . . . . 6 (𝑥 = ∅ → (𝜑𝜓))
42, 3elab 3615 . . . . 5 (∅ ∈ {𝑥𝜑} ↔ 𝜓)
51, 4mpbir 234 . . . 4 ∅ ∈ {𝑥𝜑}
6 finds.6 . . . . . 6 (𝑦 ∈ ω → (𝜒𝜃))
7 vex 3444 . . . . . . 7 𝑦 ∈ V
8 finds.2 . . . . . . 7 (𝑥 = 𝑦 → (𝜑𝜒))
97, 8elab 3615 . . . . . 6 (𝑦 ∈ {𝑥𝜑} ↔ 𝜒)
107sucex 7506 . . . . . . 7 suc 𝑦 ∈ V
11 finds.3 . . . . . . 7 (𝑥 = suc 𝑦 → (𝜑𝜃))
1210, 11elab 3615 . . . . . 6 (suc 𝑦 ∈ {𝑥𝜑} ↔ 𝜃)
136, 9, 123imtr4g 299 . . . . 5 (𝑦 ∈ ω → (𝑦 ∈ {𝑥𝜑} → suc 𝑦 ∈ {𝑥𝜑}))
1413rgen 3116 . . . 4 𝑦 ∈ ω (𝑦 ∈ {𝑥𝜑} → suc 𝑦 ∈ {𝑥𝜑})
15 peano5 7585 . . . 4 ((∅ ∈ {𝑥𝜑} ∧ ∀𝑦 ∈ ω (𝑦 ∈ {𝑥𝜑} → suc 𝑦 ∈ {𝑥𝜑})) → ω ⊆ {𝑥𝜑})
165, 14, 15mp2an 691 . . 3 ω ⊆ {𝑥𝜑}
1716sseli 3911 . 2 (𝐴 ∈ ω → 𝐴 ∈ {𝑥𝜑})
18 finds.4 . . 3 (𝑥 = 𝐴 → (𝜑𝜏))
1918elabg 3614 . 2 (𝐴 ∈ ω → (𝐴 ∈ {𝑥𝜑} ↔ 𝜏))
2017, 19mpbid 235 1 (𝐴 ∈ ω → 𝜏)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 209   = wceq 1538  wcel 2111  {cab 2776  wral 3106  wss 3881  c0 4243  suc csuc 6161  ωcom 7560
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1797  ax-4 1811  ax-5 1911  ax-6 1970  ax-7 2015  ax-8 2113  ax-9 2121  ax-10 2142  ax-11 2158  ax-12 2175  ax-ext 2770  ax-sep 5167  ax-nul 5174  ax-pr 5295  ax-un 7441
This theorem depends on definitions:  df-bi 210  df-an 400  df-or 845  df-3or 1085  df-3an 1086  df-tru 1541  df-ex 1782  df-nf 1786  df-sb 2070  df-mo 2598  df-eu 2629  df-clab 2777  df-cleq 2791  df-clel 2870  df-nfc 2938  df-ne 2988  df-ral 3111  df-rex 3112  df-rab 3115  df-v 3443  df-sbc 3721  df-dif 3884  df-un 3886  df-in 3888  df-ss 3898  df-pss 3900  df-nul 4244  df-if 4426  df-pw 4499  df-sn 4526  df-pr 4528  df-tp 4530  df-op 4532  df-uni 4801  df-br 5031  df-opab 5093  df-tr 5137  df-eprel 5430  df-po 5438  df-so 5439  df-fr 5478  df-we 5480  df-ord 6162  df-on 6163  df-lim 6164  df-suc 6165  df-om 7561
This theorem is referenced by:  findsg  7590  findes  7593  seqomlem1  8069  nna0r  8218  nnm0r  8219  nnawordi  8230  nneob  8262  nneneq  8684  pssnn  8720  inf3lem1  9075  inf3lem2  9076  cantnfval2  9116  cantnfp1lem3  9127  r1fin  9186  ackbij1lem14  9644  ackbij1lem16  9646  ackbij1  9649  ackbij2lem2  9651  ackbij2lem3  9652  infpssrlem4  9717  fin23lem14  9744  fin23lem34  9757  itunitc1  9831  ituniiun  9833  om2uzuzi  13312  om2uzlti  13313  om2uzrdg  13319  uzrdgxfr  13330  hashgadd  13734  mreexexd  16911  satfrel  32727  satfdm  32729  satfrnmapom  32730  satf0op  32737  satf0n0  32738  sat1el2xp  32739  fmlafvel  32745  fmlaomn0  32750  gonar  32755  goalr  32757  satffun  32769  trpredmintr  33183  findfvcl  33913  finxp00  34819
  Copyright terms: Public domain W3C validator