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

Theorem finds 7610
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 5213 . . . . . 6 ∅ ∈ V
3 finds.1 . . . . . 6 (𝑥 = ∅ → (𝜑𝜓))
42, 3elab 3669 . . . . 5 (∅ ∈ {𝑥𝜑} ↔ 𝜓)
51, 4mpbir 233 . . . 4 ∅ ∈ {𝑥𝜑}
6 finds.6 . . . . . 6 (𝑦 ∈ ω → (𝜒𝜃))
7 vex 3499 . . . . . . 7 𝑦 ∈ V
8 finds.2 . . . . . . 7 (𝑥 = 𝑦 → (𝜑𝜒))
97, 8elab 3669 . . . . . 6 (𝑦 ∈ {𝑥𝜑} ↔ 𝜒)
107sucex 7528 . . . . . . 7 suc 𝑦 ∈ V
11 finds.3 . . . . . . 7 (𝑥 = suc 𝑦 → (𝜑𝜃))
1210, 11elab 3669 . . . . . 6 (suc 𝑦 ∈ {𝑥𝜑} ↔ 𝜃)
136, 9, 123imtr4g 298 . . . . 5 (𝑦 ∈ ω → (𝑦 ∈ {𝑥𝜑} → suc 𝑦 ∈ {𝑥𝜑}))
1413rgen 3150 . . . 4 𝑦 ∈ ω (𝑦 ∈ {𝑥𝜑} → suc 𝑦 ∈ {𝑥𝜑})
15 peano5 7607 . . . 4 ((∅ ∈ {𝑥𝜑} ∧ ∀𝑦 ∈ ω (𝑦 ∈ {𝑥𝜑} → suc 𝑦 ∈ {𝑥𝜑})) → ω ⊆ {𝑥𝜑})
165, 14, 15mp2an 690 . . 3 ω ⊆ {𝑥𝜑}
1716sseli 3965 . 2 (𝐴 ∈ ω → 𝐴 ∈ {𝑥𝜑})
18 finds.4 . . 3 (𝑥 = 𝐴 → (𝜑𝜏))
1918elabg 3668 . 2 (𝐴 ∈ ω → (𝐴 ∈ {𝑥𝜑} ↔ 𝜏))
2017, 19mpbid 234 1 (𝐴 ∈ ω → 𝜏)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 208   = wceq 1537  wcel 2114  {cab 2801  wral 3140  wss 3938  c0 4293  suc csuc 6195  ωcom 7582
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1796  ax-4 1810  ax-5 1911  ax-6 1970  ax-7 2015  ax-8 2116  ax-9 2124  ax-10 2145  ax-11 2161  ax-12 2177  ax-ext 2795  ax-sep 5205  ax-nul 5212  ax-pr 5332  ax-un 7463
This theorem depends on definitions:  df-bi 209  df-an 399  df-or 844  df-3or 1084  df-3an 1085  df-tru 1540  df-ex 1781  df-nf 1785  df-sb 2070  df-mo 2622  df-eu 2654  df-clab 2802  df-cleq 2816  df-clel 2895  df-nfc 2965  df-ne 3019  df-ral 3145  df-rex 3146  df-rab 3149  df-v 3498  df-sbc 3775  df-dif 3941  df-un 3943  df-in 3945  df-ss 3954  df-pss 3956  df-nul 4294  df-if 4470  df-pw 4543  df-sn 4570  df-pr 4572  df-tp 4574  df-op 4576  df-uni 4841  df-br 5069  df-opab 5131  df-tr 5175  df-eprel 5467  df-po 5476  df-so 5477  df-fr 5516  df-we 5518  df-ord 6196  df-on 6197  df-lim 6198  df-suc 6199  df-om 7583
This theorem is referenced by:  findsg  7611  findes  7614  seqomlem1  8088  nna0r  8237  nnm0r  8238  nnawordi  8249  nneob  8281  nneneq  8702  pssnn  8738  inf3lem1  9093  inf3lem2  9094  cantnfval2  9134  cantnfp1lem3  9145  r1fin  9204  ackbij1lem14  9657  ackbij1lem16  9659  ackbij1  9662  ackbij2lem2  9664  ackbij2lem3  9665  infpssrlem4  9730  fin23lem14  9757  fin23lem34  9770  itunitc1  9844  ituniiun  9846  om2uzuzi  13320  om2uzlti  13321  om2uzrdg  13327  uzrdgxfr  13338  hashgadd  13741  mreexexd  16921  satfrel  32616  satfdm  32618  satfrnmapom  32619  satf0op  32626  satf0n0  32627  sat1el2xp  32628  fmlafvel  32634  fmlaomn0  32639  gonar  32644  goalr  32646  satffun  32658  trpredmintr  33072  findfvcl  33802  finxp00  34685
  Copyright terms: Public domain W3C validator