Metamath Proof Explorer |
< Previous
Next >
Nearby theorems |
||
Mirrors > Home > MPE Home > Th. List > finds | Structured version Visualization version GIF version |
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.) |
Ref | Expression |
---|---|
finds.1 | ⊢ (𝑥 = ∅ → (𝜑 ↔ 𝜓)) |
finds.2 | ⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜒)) |
finds.3 | ⊢ (𝑥 = suc 𝑦 → (𝜑 ↔ 𝜃)) |
finds.4 | ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜏)) |
finds.5 | ⊢ 𝜓 |
finds.6 | ⊢ (𝑦 ∈ ω → (𝜒 → 𝜃)) |
Ref | Expression |
---|---|
finds | ⊢ (𝐴 ∈ ω → 𝜏) |
Step | Hyp | Ref | Expression |
---|---|---|---|
1 | finds.5 | . . . . 5 ⊢ 𝜓 | |
2 | 0ex 5231 | . . . . . 6 ⊢ ∅ ∈ V | |
3 | finds.1 | . . . . . 6 ⊢ (𝑥 = ∅ → (𝜑 ↔ 𝜓)) | |
4 | 2, 3 | elab 3609 | . . . . 5 ⊢ (∅ ∈ {𝑥 ∣ 𝜑} ↔ 𝜓) |
5 | 1, 4 | mpbir 230 | . . . 4 ⊢ ∅ ∈ {𝑥 ∣ 𝜑} |
6 | finds.6 | . . . . . 6 ⊢ (𝑦 ∈ ω → (𝜒 → 𝜃)) | |
7 | vex 3436 | . . . . . . 7 ⊢ 𝑦 ∈ V | |
8 | finds.2 | . . . . . . 7 ⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜒)) | |
9 | 7, 8 | elab 3609 | . . . . . 6 ⊢ (𝑦 ∈ {𝑥 ∣ 𝜑} ↔ 𝜒) |
10 | 7 | sucex 7656 | . . . . . . 7 ⊢ suc 𝑦 ∈ V |
11 | finds.3 | . . . . . . 7 ⊢ (𝑥 = suc 𝑦 → (𝜑 ↔ 𝜃)) | |
12 | 10, 11 | elab 3609 | . . . . . 6 ⊢ (suc 𝑦 ∈ {𝑥 ∣ 𝜑} ↔ 𝜃) |
13 | 6, 9, 12 | 3imtr4g 296 | . . . . 5 ⊢ (𝑦 ∈ ω → (𝑦 ∈ {𝑥 ∣ 𝜑} → suc 𝑦 ∈ {𝑥 ∣ 𝜑})) |
14 | 13 | rgen 3074 | . . . 4 ⊢ ∀𝑦 ∈ ω (𝑦 ∈ {𝑥 ∣ 𝜑} → suc 𝑦 ∈ {𝑥 ∣ 𝜑}) |
15 | peano5 7740 | . . . 4 ⊢ ((∅ ∈ {𝑥 ∣ 𝜑} ∧ ∀𝑦 ∈ ω (𝑦 ∈ {𝑥 ∣ 𝜑} → suc 𝑦 ∈ {𝑥 ∣ 𝜑})) → ω ⊆ {𝑥 ∣ 𝜑}) | |
16 | 5, 14, 15 | mp2an 689 | . . 3 ⊢ ω ⊆ {𝑥 ∣ 𝜑} |
17 | 16 | sseli 3917 | . 2 ⊢ (𝐴 ∈ ω → 𝐴 ∈ {𝑥 ∣ 𝜑}) |
18 | finds.4 | . . 3 ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜏)) | |
19 | 18 | elabg 3607 | . 2 ⊢ (𝐴 ∈ ω → (𝐴 ∈ {𝑥 ∣ 𝜑} ↔ 𝜏)) |
20 | 17, 19 | mpbid 231 | 1 ⊢ (𝐴 ∈ ω → 𝜏) |
Colors of variables: wff setvar class |
Syntax hints: → wi 4 ↔ wb 205 = wceq 1539 ∈ wcel 2106 {cab 2715 ∀wral 3064 ⊆ wss 3887 ∅c0 4256 suc csuc 6268 ωcom 7712 |
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 1913 ax-6 1971 ax-7 2011 ax-8 2108 ax-9 2116 ax-11 2154 ax-ext 2709 ax-sep 5223 ax-nul 5230 ax-pr 5352 ax-un 7588 |
This theorem depends on definitions: df-bi 206 df-an 397 df-or 845 df-3or 1087 df-3an 1088 df-tru 1542 df-fal 1552 df-ex 1783 df-sb 2068 df-clab 2716 df-cleq 2730 df-clel 2816 df-ne 2944 df-ral 3069 df-rex 3070 df-rab 3073 df-v 3434 df-dif 3890 df-un 3892 df-in 3894 df-ss 3904 df-pss 3906 df-nul 4257 df-if 4460 df-pw 4535 df-sn 4562 df-pr 4564 df-op 4568 df-uni 4840 df-br 5075 df-opab 5137 df-tr 5192 df-eprel 5495 df-po 5503 df-so 5504 df-fr 5544 df-we 5546 df-ord 6269 df-on 6270 df-lim 6271 df-suc 6272 df-om 7713 |
This theorem is referenced by: findsg 7746 findes 7749 seqomlem1 8281 nna0r 8440 nnm0r 8441 nnawordi 8452 nneob 8486 enrefnn 8837 pssnn 8951 nneneq 8992 nneneqOLD 9004 pssnnOLD 9040 inf3lem1 9386 inf3lem2 9387 cantnfval2 9427 cantnfp1lem3 9438 ttrclss 9478 ttrclselem2 9484 r1fin 9531 ackbij1lem14 9989 ackbij1lem16 9991 ackbij1 9994 ackbij2lem2 9996 ackbij2lem3 9997 infpssrlem4 10062 fin23lem14 10089 fin23lem34 10102 itunitc1 10176 ituniiun 10178 om2uzuzi 13669 om2uzlti 13670 om2uzrdg 13676 uzrdgxfr 13687 hashgadd 14092 mreexexd 17357 satfrel 33329 satfdm 33331 satfrnmapom 33332 satf0op 33339 satf0n0 33340 sat1el2xp 33341 fmlafvel 33347 fmlaomn0 33352 gonar 33357 goalr 33359 satffun 33371 findfvcl 34641 finxp00 35573 |
Copyright terms: Public domain | W3C validator |