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

Theorem brfi1uzind 14466
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 14467) 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 5731 . . 3 (𝑉𝐺𝐸 → (𝑉 ∈ V ∧ 𝐸 ∈ V))
3 simpl 482 . . . . 5 ((𝑉 ∈ V ∧ 𝐸 ∈ V) → 𝑉 ∈ V)
4 simplr 766 . . . . . 6 (((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) → 𝐸 ∈ V)
5 breq12 5153 . . . . . . 7 ((𝑎 = 𝑉𝑏 = 𝐸) → (𝑎𝐺𝑏𝑉𝐺𝐸))
65adantll 711 . . . . . 6 ((((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) ∧ 𝑏 = 𝐸) → (𝑎𝐺𝑏𝑉𝐺𝐸))
74, 6sbcied 3822 . . . . 5 (((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) → ([𝐸 / 𝑏]𝑎𝐺𝑏𝑉𝐺𝐸))
83, 7sbcied 3822 . . . 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 3477 . . . . 5 𝑣 ∈ V
16 vex 3477 . . . . 5 𝑒 ∈ V
17 breq12 5153 . . . . 5 ((𝑎 = 𝑣𝑏 = 𝑒) → (𝑎𝐺𝑏𝑣𝐺𝑒))
1815, 16, 17sbc2ie 3860 . . . 4 ([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏𝑣𝐺𝑒)
19 brfi1uzind.3 . . . . 5 ((𝑣𝐺𝑒𝑛𝑣) → (𝑣 ∖ {𝑛})𝐺𝐹)
2015difexi 5328 . . . . . 6 (𝑣 ∖ {𝑛}) ∈ V
21 breq12 5153 . . . . . 6 ((𝑎 = (𝑣 ∖ {𝑛}) ∧ 𝑏 = 𝐹) → (𝑎𝐺𝑏 ↔ (𝑣 ∖ {𝑛})𝐺𝐹))
2220, 11, 21sbc2ie 3860 . . . . 5 ([(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏 ↔ (𝑣 ∖ {𝑛})𝐺𝐹)
2319, 22sylibr 233 . . . 4 ((𝑣𝐺𝑒𝑛𝑣) → [(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏)
2418, 23sylanb 580 . . 3 (([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏𝑛𝑣) → [(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏)
25 brfi1uzind.4 . . 3 ((𝑤 = (𝑣 ∖ {𝑛}) ∧ 𝑓 = 𝐹) → (𝜃𝜒))
26 brfi1uzind.base . . . 4 ((𝑣𝐺𝑒 ∧ (♯‘𝑣) = 𝐿) → 𝜓)
2718, 26sylanb 580 . . 3 (([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = 𝐿) → 𝜓)
28183anbi1i 1156 . . . . 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 14465 . 2 (([𝑉 / 𝑎][𝐸 / 𝑏]𝑎𝐺𝑏𝑉 ∈ Fin ∧ 𝐿 ≤ (♯‘𝑉)) → 𝜑)
3310, 32syl3an1 1162 1 ((𝑉𝐺𝐸𝑉 ∈ Fin ∧ 𝐿 ≤ (♯‘𝑉)) → 𝜑)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 205  wa 395  w3a 1086   = wceq 1540  wcel 2105  Vcvv 3473  [wsbc 3777  cdif 3945  {csn 4628   class class class wbr 5148  Rel wrel 5681  cfv 6543  (class class class)co 7412  Fincfn 8945  1c1 11117   + caddc 11119  cle 11256  0cn0 12479  chash 14297
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 1912  ax-6 1970  ax-7 2010  ax-8 2107  ax-9 2115  ax-10 2136  ax-11 2153  ax-12 2170  ax-ext 2702  ax-sep 5299  ax-nul 5306  ax-pow 5363  ax-pr 5427  ax-un 7729  ax-cnex 11172  ax-resscn 11173  ax-1cn 11174  ax-icn 11175  ax-addcl 11176  ax-addrcl 11177  ax-mulcl 11178  ax-mulrcl 11179  ax-mulcom 11180  ax-addass 11181  ax-mulass 11182  ax-distr 11183  ax-i2m1 11184  ax-1ne0 11185  ax-1rid 11186  ax-rnegex 11187  ax-rrecex 11188  ax-cnre 11189  ax-pre-lttri 11190  ax-pre-lttrn 11191  ax-pre-ltadd 11192  ax-pre-mulgt0 11193
This theorem depends on definitions:  df-bi 206  df-an 396  df-or 845  df-3or 1087  df-3an 1088  df-tru 1543  df-fal 1553  df-ex 1781  df-nf 1785  df-sb 2067  df-mo 2533  df-eu 2562  df-clab 2709  df-cleq 2723  df-clel 2809  df-nfc 2884  df-ne 2940  df-nel 3046  df-ral 3061  df-rex 3070  df-reu 3376  df-rab 3432  df-v 3475  df-sbc 3778  df-csb 3894  df-dif 3951  df-un 3953  df-in 3955  df-ss 3965  df-pss 3967  df-nul 4323  df-if 4529  df-pw 4604  df-sn 4629  df-pr 4631  df-op 4635  df-uni 4909  df-int 4951  df-iun 4999  df-br 5149  df-opab 5211  df-mpt 5232  df-tr 5266  df-id 5574  df-eprel 5580  df-po 5588  df-so 5589  df-fr 5631  df-we 5633  df-xp 5682  df-rel 5683  df-cnv 5684  df-co 5685  df-dm 5686  df-rn 5687  df-res 5688  df-ima 5689  df-pred 6300  df-ord 6367  df-on 6368  df-lim 6369  df-suc 6370  df-iota 6495  df-fun 6545  df-fn 6546  df-f 6547  df-f1 6548  df-fo 6549  df-f1o 6550  df-fv 6551  df-riota 7368  df-ov 7415  df-oprab 7416  df-mpo 7417  df-om 7860  df-1st 7979  df-2nd 7980  df-frecs 8272  df-wrecs 8303  df-recs 8377  df-rdg 8416  df-1o 8472  df-oadd 8476  df-er 8709  df-en 8946  df-dom 8947  df-sdom 8948  df-fin 8949  df-dju 9902  df-card 9940  df-pnf 11257  df-mnf 11258  df-xr 11259  df-ltxr 11260  df-le 11261  df-sub 11453  df-neg 11454  df-nn 12220  df-n0 12480  df-xnn0 12552  df-z 12566  df-uz 12830  df-fz 13492  df-hash 14298
This theorem is referenced by:  brfi1ind  14467
  Copyright terms: Public domain W3C validator