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

Theorem frgr1v 28056
Description: Any graph with (at most) one vertex is a friendship graph. (Contributed by Alexander van der Vekens, 4-Oct-2017.) (Revised by AV, 29-Mar-2021.)
Assertion
Ref Expression
frgr1v ((𝐺 ∈ USGraph ∧ (Vtx‘𝐺) = {𝑁}) → 𝐺 ∈ FriendGraph )

Proof of Theorem frgr1v
Dummy variables 𝑘 𝑙 𝑥 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 simpl 486 . 2 ((𝐺 ∈ USGraph ∧ (Vtx‘𝐺) = {𝑁}) → 𝐺 ∈ USGraph)
2 ral0 4414 . . . . 5 𝑙 ∈ ∅ ∃!𝑥 ∈ {𝑁} {{𝑥, 𝑁}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)
3 sneq 4535 . . . . . . . . 9 (𝑘 = 𝑁 → {𝑘} = {𝑁})
43difeq2d 4050 . . . . . . . 8 (𝑘 = 𝑁 → ({𝑁} ∖ {𝑘}) = ({𝑁} ∖ {𝑁}))
5 difid 4284 . . . . . . . 8 ({𝑁} ∖ {𝑁}) = ∅
64, 5eqtrdi 2849 . . . . . . 7 (𝑘 = 𝑁 → ({𝑁} ∖ {𝑘}) = ∅)
7 preq2 4630 . . . . . . . . . 10 (𝑘 = 𝑁 → {𝑥, 𝑘} = {𝑥, 𝑁})
87preq1d 4635 . . . . . . . . 9 (𝑘 = 𝑁 → {{𝑥, 𝑘}, {𝑥, 𝑙}} = {{𝑥, 𝑁}, {𝑥, 𝑙}})
98sseq1d 3946 . . . . . . . 8 (𝑘 = 𝑁 → ({{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺) ↔ {{𝑥, 𝑁}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
109reubidv 3342 . . . . . . 7 (𝑘 = 𝑁 → (∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺) ↔ ∃!𝑥 ∈ {𝑁} {{𝑥, 𝑁}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
116, 10raleqbidv 3354 . . . . . 6 (𝑘 = 𝑁 → (∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺) ↔ ∀𝑙 ∈ ∅ ∃!𝑥 ∈ {𝑁} {{𝑥, 𝑁}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
1211ralsng 4573 . . . . 5 (𝑁 ∈ V → (∀𝑘 ∈ {𝑁}∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺) ↔ ∀𝑙 ∈ ∅ ∃!𝑥 ∈ {𝑁} {{𝑥, 𝑁}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
132, 12mpbiri 261 . . . 4 (𝑁 ∈ V → ∀𝑘 ∈ {𝑁}∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺))
14 snprc 4613 . . . . 5 𝑁 ∈ V ↔ {𝑁} = ∅)
15 rzal 4411 . . . . 5 ({𝑁} = ∅ → ∀𝑘 ∈ {𝑁}∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺))
1614, 15sylbi 220 . . . 4 𝑁 ∈ V → ∀𝑘 ∈ {𝑁}∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺))
1713, 16pm2.61i 185 . . 3 𝑘 ∈ {𝑁}∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)
18 id 22 . . . . 5 ((Vtx‘𝐺) = {𝑁} → (Vtx‘𝐺) = {𝑁})
19 difeq1 4043 . . . . . 6 ((Vtx‘𝐺) = {𝑁} → ((Vtx‘𝐺) ∖ {𝑘}) = ({𝑁} ∖ {𝑘}))
20 reueq1 3360 . . . . . 6 ((Vtx‘𝐺) = {𝑁} → (∃!𝑥 ∈ (Vtx‘𝐺){{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺) ↔ ∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
2119, 20raleqbidv 3354 . . . . 5 ((Vtx‘𝐺) = {𝑁} → (∀𝑙 ∈ ((Vtx‘𝐺) ∖ {𝑘})∃!𝑥 ∈ (Vtx‘𝐺){{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺) ↔ ∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
2218, 21raleqbidv 3354 . . . 4 ((Vtx‘𝐺) = {𝑁} → (∀𝑘 ∈ (Vtx‘𝐺)∀𝑙 ∈ ((Vtx‘𝐺) ∖ {𝑘})∃!𝑥 ∈ (Vtx‘𝐺){{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺) ↔ ∀𝑘 ∈ {𝑁}∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
2322adantl 485 . . 3 ((𝐺 ∈ USGraph ∧ (Vtx‘𝐺) = {𝑁}) → (∀𝑘 ∈ (Vtx‘𝐺)∀𝑙 ∈ ((Vtx‘𝐺) ∖ {𝑘})∃!𝑥 ∈ (Vtx‘𝐺){{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺) ↔ ∀𝑘 ∈ {𝑁}∀𝑙 ∈ ({𝑁} ∖ {𝑘})∃!𝑥 ∈ {𝑁} {{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
2417, 23mpbiri 261 . 2 ((𝐺 ∈ USGraph ∧ (Vtx‘𝐺) = {𝑁}) → ∀𝑘 ∈ (Vtx‘𝐺)∀𝑙 ∈ ((Vtx‘𝐺) ∖ {𝑘})∃!𝑥 ∈ (Vtx‘𝐺){{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺))
25 eqid 2798 . . 3 (Vtx‘𝐺) = (Vtx‘𝐺)
26 eqid 2798 . . 3 (Edg‘𝐺) = (Edg‘𝐺)
2725, 26isfrgr 28045 . 2 (𝐺 ∈ FriendGraph ↔ (𝐺 ∈ USGraph ∧ ∀𝑘 ∈ (Vtx‘𝐺)∀𝑙 ∈ ((Vtx‘𝐺) ∖ {𝑘})∃!𝑥 ∈ (Vtx‘𝐺){{𝑥, 𝑘}, {𝑥, 𝑙}} ⊆ (Edg‘𝐺)))
281, 24, 27sylanbrc 586 1 ((𝐺 ∈ USGraph ∧ (Vtx‘𝐺) = {𝑁}) → 𝐺 ∈ FriendGraph )
Colors of variables: wff setvar class
Syntax hints:  ¬ wn 3  wi 4  wb 209  wa 399   = wceq 1538  wcel 2111  wral 3106  ∃!wreu 3108  Vcvv 3441  cdif 3878  wss 3881  c0 4243  {csn 4525  {cpr 4527  cfv 6324  Vtxcvtx 26789  Edgcedg 26840  USGraphcusgr 26942   FriendGraph cfrgr 28043
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 2770  ax-nul 5174
This theorem depends on definitions:  df-bi 210  df-an 400  df-or 845  df-3an 1086  df-tru 1541  df-ex 1782  df-nf 1786  df-sb 2070  df-mo 2598  df-eu 2629  df-clab 2777  df-cleq 2791  df-clel 2870  df-nfc 2938  df-ne 2988  df-ral 3111  df-rex 3112  df-reu 3113  df-rab 3115  df-v 3443  df-sbc 3721  df-dif 3884  df-un 3886  df-in 3888  df-ss 3898  df-nul 4244  df-sn 4526  df-pr 4528  df-op 4532  df-uni 4801  df-br 5031  df-iota 6283  df-fv 6332  df-frgr 28044
This theorem is referenced by: (None)
  Copyright terms: Public domain W3C validator