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

Theorem finds2 7721
Description: Principle of Finite Induction (inference schema), using implicit substitutions. The first three hypotheses establish the substitutions we need. The last two are the basis and the induction step. Theorem Schema 22 of [Suppes] p. 136. (Contributed by NM, 29-Nov-2002.)
Hypotheses
Ref Expression
finds2.1 (𝑥 = ∅ → (𝜑𝜓))
finds2.2 (𝑥 = 𝑦 → (𝜑𝜒))
finds2.3 (𝑥 = suc 𝑦 → (𝜑𝜃))
finds2.4 (𝜏𝜓)
finds2.5 (𝑦 ∈ ω → (𝜏 → (𝜒𝜃)))
Assertion
Ref Expression
finds2 (𝑥 ∈ ω → (𝜏𝜑))
Distinct variable groups:   𝑥,𝑦,𝜏   𝜓,𝑥   𝜒,𝑥   𝜃,𝑥   𝜑,𝑦
Allowed substitution hints:   𝜑(𝑥)   𝜓(𝑦)   𝜒(𝑦)   𝜃(𝑦)

Proof of Theorem finds2
StepHypRef Expression
1 finds2.4 . . . . 5 (𝜏𝜓)
2 0ex 5226 . . . . . 6 ∅ ∈ V
3 finds2.1 . . . . . . 7 (𝑥 = ∅ → (𝜑𝜓))
43imbi2d 340 . . . . . 6 (𝑥 = ∅ → ((𝜏𝜑) ↔ (𝜏𝜓)))
52, 4elab 3602 . . . . 5 (∅ ∈ {𝑥 ∣ (𝜏𝜑)} ↔ (𝜏𝜓))
61, 5mpbir 230 . . . 4 ∅ ∈ {𝑥 ∣ (𝜏𝜑)}
7 finds2.5 . . . . . . 7 (𝑦 ∈ ω → (𝜏 → (𝜒𝜃)))
87a2d 29 . . . . . 6 (𝑦 ∈ ω → ((𝜏𝜒) → (𝜏𝜃)))
9 vex 3426 . . . . . . 7 𝑦 ∈ V
10 finds2.2 . . . . . . . 8 (𝑥 = 𝑦 → (𝜑𝜒))
1110imbi2d 340 . . . . . . 7 (𝑥 = 𝑦 → ((𝜏𝜑) ↔ (𝜏𝜒)))
129, 11elab 3602 . . . . . 6 (𝑦 ∈ {𝑥 ∣ (𝜏𝜑)} ↔ (𝜏𝜒))
139sucex 7633 . . . . . . 7 suc 𝑦 ∈ V
14 finds2.3 . . . . . . . 8 (𝑥 = suc 𝑦 → (𝜑𝜃))
1514imbi2d 340 . . . . . . 7 (𝑥 = suc 𝑦 → ((𝜏𝜑) ↔ (𝜏𝜃)))
1613, 15elab 3602 . . . . . 6 (suc 𝑦 ∈ {𝑥 ∣ (𝜏𝜑)} ↔ (𝜏𝜃))
178, 12, 163imtr4g 295 . . . . 5 (𝑦 ∈ ω → (𝑦 ∈ {𝑥 ∣ (𝜏𝜑)} → suc 𝑦 ∈ {𝑥 ∣ (𝜏𝜑)}))
1817rgen 3073 . . . 4 𝑦 ∈ ω (𝑦 ∈ {𝑥 ∣ (𝜏𝜑)} → suc 𝑦 ∈ {𝑥 ∣ (𝜏𝜑)})
19 peano5 7714 . . . 4 ((∅ ∈ {𝑥 ∣ (𝜏𝜑)} ∧ ∀𝑦 ∈ ω (𝑦 ∈ {𝑥 ∣ (𝜏𝜑)} → suc 𝑦 ∈ {𝑥 ∣ (𝜏𝜑)})) → ω ⊆ {𝑥 ∣ (𝜏𝜑)})
206, 18, 19mp2an 688 . . 3 ω ⊆ {𝑥 ∣ (𝜏𝜑)}
2120sseli 3913 . 2 (𝑥 ∈ ω → 𝑥 ∈ {𝑥 ∣ (𝜏𝜑)})
22 abid 2719 . 2 (𝑥 ∈ {𝑥 ∣ (𝜏𝜑)} ↔ (𝜏𝜑))
2321, 22sylib 217 1 (𝑥 ∈ ω → (𝜏𝜑))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 205   = wceq 1539  wcel 2108  {cab 2715  wral 3063  wss 3883  c0 4253  suc csuc 6253  ωcom 7687
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1799  ax-4 1813  ax-5 1914  ax-6 1972  ax-7 2012  ax-8 2110  ax-9 2118  ax-11 2156  ax-12 2173  ax-ext 2709  ax-sep 5218  ax-nul 5225  ax-pr 5347  ax-un 7566
This theorem depends on definitions:  df-bi 206  df-an 396  df-or 844  df-3or 1086  df-3an 1087  df-tru 1542  df-fal 1552  df-ex 1784  df-sb 2069  df-clab 2716  df-cleq 2730  df-clel 2817  df-ne 2943  df-ral 3068  df-rex 3069  df-rab 3072  df-v 3424  df-dif 3886  df-un 3888  df-in 3890  df-ss 3900  df-pss 3902  df-nul 4254  df-if 4457  df-pw 4532  df-sn 4559  df-pr 4561  df-tp 4563  df-op 4565  df-uni 4837  df-br 5071  df-opab 5133  df-tr 5188  df-eprel 5486  df-po 5494  df-so 5495  df-fr 5535  df-we 5537  df-ord 6254  df-on 6255  df-lim 6256  df-suc 6257  df-om 7688
This theorem is referenced by:  finds1  7722  onnseq  8146  nnacl  8404  nnmcl  8405  nnecl  8406  nnacom  8410  nnaass  8415  nndi  8416  nnmass  8417  nnmsucr  8418  nnmcom  8419  nnmordi  8424  omsmolem  8447  isinf  8965  unblem2  8997  fiint  9021  dffi3  9120  card2inf  9244  cantnfle  9359  cantnflt  9360  cantnflem1  9377  cnfcom  9388  trcl  9417  fseqenlem1  9711  nnadju  9884  infpssrlem3  9992  fin23lem26  10012  axdc3lem2  10138  axdc4lem  10142  axdclem2  10207  wunr1om  10406  wuncval2  10434  tskr1om  10454  grothomex  10516  peano5nni  11906  neibastop2lem  34476  finxpreclem6  35494  domalom  35502
  Copyright terms: Public domain W3C validator