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

Theorem brfi1uzind 13908
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 13909) 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 5576 . . 3 (𝑉𝐺𝐸 → (𝑉 ∈ V ∧ 𝐸 ∈ V))
3 simpl 486 . . . . 5 ((𝑉 ∈ V ∧ 𝐸 ∈ V) → 𝑉 ∈ V)
4 simplr 768 . . . . . 6 (((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) → 𝐸 ∈ V)
5 breq12 5037 . . . . . . 7 ((𝑎 = 𝑉𝑏 = 𝐸) → (𝑎𝐺𝑏𝑉𝐺𝐸))
65adantll 713 . . . . . 6 ((((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) ∧ 𝑏 = 𝐸) → (𝑎𝐺𝑏𝑉𝐺𝐸))
74, 6sbcied 3739 . . . . 5 (((𝑉 ∈ V ∧ 𝐸 ∈ V) ∧ 𝑎 = 𝑉) → ([𝐸 / 𝑏]𝑎𝐺𝑏𝑉𝐺𝐸))
83, 7sbcied 3739 . . . 4 ((𝑉 ∈ V ∧ 𝐸 ∈ V) → ([𝑉 / 𝑎][𝐸 / 𝑏]𝑎𝐺𝑏𝑉𝐺𝐸))
98biimprcd 253 . . 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 3413 . . . . 5 𝑣 ∈ V
16 vex 3413 . . . . 5 𝑒 ∈ V
17 breq12 5037 . . . . 5 ((𝑎 = 𝑣𝑏 = 𝑒) → (𝑎𝐺𝑏𝑣𝐺𝑒))
1815, 16, 17sbc2ie 3773 . . . 4 ([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏𝑣𝐺𝑒)
19 brfi1uzind.3 . . . . 5 ((𝑣𝐺𝑒𝑛𝑣) → (𝑣 ∖ {𝑛})𝐺𝐹)
2015difexi 5198 . . . . . 6 (𝑣 ∖ {𝑛}) ∈ V
21 breq12 5037 . . . . . 6 ((𝑎 = (𝑣 ∖ {𝑛}) ∧ 𝑏 = 𝐹) → (𝑎𝐺𝑏 ↔ (𝑣 ∖ {𝑛})𝐺𝐹))
2220, 11, 21sbc2ie 3773 . . . . 5 ([(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏 ↔ (𝑣 ∖ {𝑛})𝐺𝐹)
2319, 22sylibr 237 . . . 4 ((𝑣𝐺𝑒𝑛𝑣) → [(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏)
2418, 23sylanb 584 . . 3 (([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏𝑛𝑣) → [(𝑣 ∖ {𝑛}) / 𝑎][𝐹 / 𝑏]𝑎𝐺𝑏)
25 brfi1uzind.4 . . 3 ((𝑤 = (𝑣 ∖ {𝑛}) ∧ 𝑓 = 𝐹) → (𝜃𝜒))
26 brfi1uzind.base . . . 4 ((𝑣𝐺𝑒 ∧ (♯‘𝑣) = 𝐿) → 𝜓)
2718, 26sylanb 584 . . 3 (([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = 𝐿) → 𝜓)
28183anbi1i 1154 . . . . 5 (([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣) ↔ (𝑣𝐺𝑒 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣))
2928anbi2i 625 . . . 4 (((𝑦 + 1) ∈ ℕ0 ∧ ([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)) ↔ ((𝑦 + 1) ∈ ℕ0 ∧ (𝑣𝐺𝑒 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)))
30 brfi1uzind.step . . . 4 ((((𝑦 + 1) ∈ ℕ0 ∧ (𝑣𝐺𝑒 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)) ∧ 𝜒) → 𝜓)
3129, 30sylanb 584 . . 3 ((((𝑦 + 1) ∈ ℕ0 ∧ ([𝑣 / 𝑎][𝑒 / 𝑏]𝑎𝐺𝑏 ∧ (♯‘𝑣) = (𝑦 + 1) ∧ 𝑛𝑣)) ∧ 𝜒) → 𝜓)
3211, 12, 13, 14, 24, 25, 27, 31fi1uzind 13907 . 2 (([𝑉 / 𝑎][𝐸 / 𝑏]𝑎𝐺𝑏𝑉 ∈ Fin ∧ 𝐿 ≤ (♯‘𝑉)) → 𝜑)
3310, 32syl3an1 1160 1 ((𝑉𝐺𝐸𝑉 ∈ Fin ∧ 𝐿 ≤ (♯‘𝑉)) → 𝜑)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 209  wa 399  w3a 1084   = wceq 1538  wcel 2111  Vcvv 3409  [wsbc 3696  cdif 3855  {csn 4522   class class class wbr 5032  Rel wrel 5529  cfv 6335  (class class class)co 7150  Fincfn 8527  1c1 10576   + caddc 10578  cle 10714  0cn0 11934  chash 13740
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1797  ax-4 1811  ax-5 1911  ax-6 1970  ax-7 2015  ax-8 2113  ax-9 2121  ax-10 2142  ax-11 2158  ax-12 2175  ax-ext 2729  ax-sep 5169  ax-nul 5176  ax-pow 5234  ax-pr 5298  ax-un 7459  ax-cnex 10631  ax-resscn 10632  ax-1cn 10633  ax-icn 10634  ax-addcl 10635  ax-addrcl 10636  ax-mulcl 10637  ax-mulrcl 10638  ax-mulcom 10639  ax-addass 10640  ax-mulass 10641  ax-distr 10642  ax-i2m1 10643  ax-1ne0 10644  ax-1rid 10645  ax-rnegex 10646  ax-rrecex 10647  ax-cnre 10648  ax-pre-lttri 10649  ax-pre-lttrn 10650  ax-pre-ltadd 10651  ax-pre-mulgt0 10652
This theorem depends on definitions:  df-bi 210  df-an 400  df-or 845  df-3or 1085  df-3an 1086  df-tru 1541  df-fal 1551  df-ex 1782  df-nf 1786  df-sb 2070  df-mo 2557  df-eu 2588  df-clab 2736  df-cleq 2750  df-clel 2830  df-nfc 2901  df-ne 2952  df-nel 3056  df-ral 3075  df-rex 3076  df-reu 3077  df-rab 3079  df-v 3411  df-sbc 3697  df-csb 3806  df-dif 3861  df-un 3863  df-in 3865  df-ss 3875  df-pss 3877  df-nul 4226  df-if 4421  df-pw 4496  df-sn 4523  df-pr 4525  df-tp 4527  df-op 4529  df-uni 4799  df-int 4839  df-iun 4885  df-br 5033  df-opab 5095  df-mpt 5113  df-tr 5139  df-id 5430  df-eprel 5435  df-po 5443  df-so 5444  df-fr 5483  df-we 5485  df-xp 5530  df-rel 5531  df-cnv 5532  df-co 5533  df-dm 5534  df-rn 5535  df-res 5536  df-ima 5537  df-pred 6126  df-ord 6172  df-on 6173  df-lim 6174  df-suc 6175  df-iota 6294  df-fun 6337  df-fn 6338  df-f 6339  df-f1 6340  df-fo 6341  df-f1o 6342  df-fv 6343  df-riota 7108  df-ov 7153  df-oprab 7154  df-mpo 7155  df-om 7580  df-1st 7693  df-2nd 7694  df-wrecs 7957  df-recs 8018  df-rdg 8056  df-1o 8112  df-oadd 8116  df-er 8299  df-en 8528  df-dom 8529  df-sdom 8530  df-fin 8531  df-dju 9363  df-card 9401  df-pnf 10715  df-mnf 10716  df-xr 10717  df-ltxr 10718  df-le 10719  df-sub 10910  df-neg 10911  df-nn 11675  df-n0 11935  df-xnn0 12007  df-z 12021  df-uz 12283  df-fz 12940  df-hash 13741
This theorem is referenced by:  brfi1ind  13909
  Copyright terms: Public domain W3C validator