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

Theorem brfi1uzind 14465
Description: Properties of a binary relation with a finite first component with at least L elements, proven by finite induction on the size of the first component. This theorem can be applied for graphs (as binary relation between the set of vertices and an edge function) with a finite number of vertices, usually with 𝐿 = 0 (see brfi1ind 14466) or 𝐿 = 1. (Contributed by Alexander van der Vekens, 7-Jan-2018.) (Proof shortened by AV, 23-Oct-2020.) (Revised by AV, 28-Mar-2021.)
Hypotheses
Ref Expression
brfi1uzind.r Rel 𝐺
brfi1uzind.f 𝐹 ∈ V
brfi1uzind.l 𝐿 ∈ ℕ0
brfi1uzind.1 ((𝑣 = 𝑉𝑒 = 𝐸) → (𝜓𝜑))
brfi1uzind.2 ((𝑣 = 𝑤𝑒 = 𝑓) → (𝜓𝜃))
brfi1uzind.3 ((𝑣𝐺𝑒𝑛𝑣) → (𝑣 ∖ {𝑛})𝐺𝐹)
brfi1uzind.4 ((𝑤 = (𝑣 ∖ {𝑛}) ∧ 𝑓 = 𝐹) → (𝜃𝜒))
brfi1uzind.base ((𝑣𝐺𝑒 ∧ (♯‘𝑣) = 𝐿) → 𝜓)
brfi1uzind.step ((((𝑦 + 1) ∈ ℕ0 ∧ (𝑣𝐺𝑒 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)) ∧ 𝜒) → 𝜓)
Assertion
Ref Expression
brfi1uzind ((𝑉𝐺𝐸𝑉 ∈ Fin ∧ 𝐿 ≤ (♯‘𝑉)) → 𝜑)
Distinct variable groups:   𝑒,𝐸,𝑛,𝑣   𝑓,𝐹,𝑤   𝑒,𝐺,𝑓,𝑛,𝑣,𝑤,𝑦   𝑒,𝐿,𝑛,𝑣,𝑦   𝑒,𝑉,𝑛,𝑣   𝜓,𝑓,𝑛,𝑤,𝑦   𝜃,𝑒,𝑛,𝑣   𝜒,𝑓,𝑤   𝜑,𝑒,𝑛,𝑣
Allowed substitution hints:   𝜑(𝑦,𝑤,𝑓)   𝜓(𝑣,𝑒)   𝜒(𝑦,𝑣,𝑒,𝑛)   𝜃(𝑦,𝑤,𝑓)   𝐸(𝑦,𝑤,𝑓)   𝐹(𝑦,𝑣,𝑒,𝑛)   𝐿(𝑤,𝑓)   𝑉(𝑦,𝑤,𝑓)

Proof of Theorem brfi1uzind
Dummy variables 𝑎 𝑏 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 brfi1uzind.r . . . 4 Rel 𝐺
21brrelex12i 5724 . . 3 (𝑉𝐺𝐸 → (𝑉 ∈ V ∧ 𝐸 ∈ V))
3 simpl 482 . . . . 5 ((𝑉 ∈ V ∧ 𝐸 ∈ V) → 𝑉 ∈ V)
4 simplr 766 . . . . . 6 (((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) → 𝐸 ∈ V)
5 breq12 5146 . . . . . . 7 ((𝑎 = 𝑉𝑏 = 𝐸) → (𝑎𝐺𝑏𝑉𝐺𝐸))
65adantll 711 . . . . . 6 ((((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) ∧ 𝑏 = 𝐸) → (𝑎𝐺𝑏𝑉𝐺𝐸))
74, 6sbcied 3817 . . . . 5 (((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) → ([𝐸 / 𝑏]𝑎𝐺𝑏𝑉𝐺𝐸))
83, 7sbcied 3817 . . . 4 ((𝑉 ∈ V ∧ 𝐸 ∈ V) → ([𝑉 / 𝑎][𝐸 / 𝑏]𝑎𝐺𝑏𝑉𝐺𝐸))
98biimprcd 249 . . 3 (𝑉𝐺𝐸 → ((𝑉 ∈ V ∧ 𝐸 ∈ V) → [𝑉 / 𝑎][𝐸 / 𝑏]𝑎𝐺𝑏))
102, 9mpd 15 . 2 (𝑉𝐺𝐸[𝑉 / 𝑎][𝐸 / 𝑏]𝑎𝐺𝑏)
11 brfi1uzind.f . . 3 𝐹 ∈ V
12 brfi1uzind.l . . 3 𝐿 ∈ ℕ0
13 brfi1uzind.1 . . 3 ((𝑣 = 𝑉𝑒 = 𝐸) → (𝜓𝜑))
14 brfi1uzind.2 . . 3 ((𝑣 = 𝑤𝑒 = 𝑓) → (𝜓𝜃))
15 vex 3472 . . . . 5 𝑣 ∈ V
16 vex 3472 . . . . 5 𝑒 ∈ V
17 breq12 5146 . . . . 5 ((𝑎 = 𝑣𝑏 = 𝑒) → (𝑎𝐺𝑏𝑣𝐺𝑒))
1815, 16, 17sbc2ie 3855 . . . 4 ([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏𝑣𝐺𝑒)
19 brfi1uzind.3 . . . . 5 ((𝑣𝐺𝑒𝑛𝑣) → (𝑣 ∖ {𝑛})𝐺𝐹)
2015difexi 5321 . . . . . 6 (𝑣 ∖ {𝑛}) ∈ V
21 breq12 5146 . . . . . 6 ((𝑎 = (𝑣 ∖ {𝑛}) ∧ 𝑏 = 𝐹) → (𝑎𝐺𝑏 ↔ (𝑣 ∖ {𝑛})𝐺𝐹))
2220, 11, 21sbc2ie 3855 . . . . 5 ([(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏 ↔ (𝑣 ∖ {𝑛})𝐺𝐹)
2319, 22sylibr 233 . . . 4 ((𝑣𝐺𝑒𝑛𝑣) → [(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏)
2418, 23sylanb 580 . . 3 (([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏𝑛𝑣) → [(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏)
25 brfi1uzind.4 . . 3 ((𝑤 = (𝑣 ∖ {𝑛}) ∧ 𝑓 = 𝐹) → (𝜃𝜒))
26 brfi1uzind.base . . . 4 ((𝑣𝐺𝑒 ∧ (♯‘𝑣) = 𝐿) → 𝜓)
2718, 26sylanb 580 . . 3 (([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = 𝐿) → 𝜓)
28183anbi1i 1154 . . . . 5 (([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣) ↔ (𝑣𝐺𝑒 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣))
2928anbi2i 622 . . . 4 (((𝑦 + 1) ∈ ℕ0 ∧ ([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)) ↔ ((𝑦 + 1) ∈ ℕ0 ∧ (𝑣𝐺𝑒 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)))
30 brfi1uzind.step . . . 4 ((((𝑦 + 1) ∈ ℕ0 ∧ (𝑣𝐺𝑒 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)) ∧ 𝜒) → 𝜓)
3129, 30sylanb 580 . . 3 ((((𝑦 + 1) ∈ ℕ0 ∧ ([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)) ∧ 𝜒) → 𝜓)
3211, 12, 13, 14, 24, 25, 27, 31fi1uzind 14464 . 2 (([𝑉 / 𝑎][𝐸 / 𝑏]𝑎𝐺𝑏𝑉 ∈ Fin ∧ 𝐿 ≤ (♯‘𝑉)) → 𝜑)
3310, 32syl3an1 1160 1 ((𝑉𝐺𝐸𝑉 ∈ Fin ∧ 𝐿 ≤ (♯‘𝑉)) → 𝜑)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 205  wa 395  w3a 1084   = wceq 1533  wcel 2098  Vcvv 3468  [wsbc 3772  cdif 3940  {csn 4623   class class class wbr 5141  Rel wrel 5674  cfv 6537  (class class class)co 7405  Fincfn 8941  1c1 11113   + caddc 11115  cle 11253  0cn0 12476  chash 14295
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1789  ax-4 1803  ax-5 1905  ax-6 1963  ax-7 2003  ax-8 2100  ax-9 2108  ax-10 2129  ax-11 2146  ax-12 2163  ax-ext 2697  ax-sep 5292  ax-nul 5299  ax-pow 5356  ax-pr 5420  ax-un 7722  ax-cnex 11168  ax-resscn 11169  ax-1cn 11170  ax-icn 11171  ax-addcl 11172  ax-addrcl 11173  ax-mulcl 11174  ax-mulrcl 11175  ax-mulcom 11176  ax-addass 11177  ax-mulass 11178  ax-distr 11179  ax-i2m1 11180  ax-1ne0 11181  ax-1rid 11182  ax-rnegex 11183  ax-rrecex 11184  ax-cnre 11185  ax-pre-lttri 11186  ax-pre-lttrn 11187  ax-pre-ltadd 11188  ax-pre-mulgt0 11189
This theorem depends on definitions:  df-bi 206  df-an 396  df-or 845  df-3or 1085  df-3an 1086  df-tru 1536  df-fal 1546  df-ex 1774  df-nf 1778  df-sb 2060  df-mo 2528  df-eu 2557  df-clab 2704  df-cleq 2718  df-clel 2804  df-nfc 2879  df-ne 2935  df-nel 3041  df-ral 3056  df-rex 3065  df-reu 3371  df-rab 3427  df-v 3470  df-sbc 3773  df-csb 3889  df-dif 3946  df-un 3948  df-in 3950  df-ss 3960  df-pss 3962  df-nul 4318  df-if 4524  df-pw 4599  df-sn 4624  df-pr 4626  df-op 4630  df-uni 4903  df-int 4944  df-iun 4992  df-br 5142  df-opab 5204  df-mpt 5225  df-tr 5259  df-id 5567  df-eprel 5573  df-po 5581  df-so 5582  df-fr 5624  df-we 5626  df-xp 5675  df-rel 5676  df-cnv 5677  df-co 5678  df-dm 5679  df-rn 5680  df-res 5681  df-ima 5682  df-pred 6294  df-ord 6361  df-on 6362  df-lim 6363  df-suc 6364  df-iota 6489  df-fun 6539  df-fn 6540  df-f 6541  df-f1 6542  df-fo 6543  df-f1o 6544  df-fv 6545  df-riota 7361  df-ov 7408  df-oprab 7409  df-mpo 7410  df-om 7853  df-1st 7974  df-2nd 7975  df-frecs 8267  df-wrecs 8298  df-recs 8372  df-rdg 8411  df-1o 8467  df-oadd 8471  df-er 8705  df-en 8942  df-dom 8943  df-sdom 8944  df-fin 8945  df-dju 9898  df-card 9936  df-pnf 11254  df-mnf 11255  df-xr 11256  df-ltxr 11257  df-le 11258  df-sub 11450  df-neg 11451  df-nn 12217  df-n0 12477  df-xnn0 12549  df-z 12563  df-uz 12827  df-fz 13491  df-hash 14296
This theorem is referenced by:  brfi1ind  14466
  Copyright terms: Public domain W3C validator