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

Theorem comfffval 17758
Description: Value of the functionalized composition operation. (Contributed by Mario Carneiro, 4-Jan-2017.) (Proof shortened by AV, 1-Mar-2024.)
Hypotheses
Ref Expression
comfffval.o 𝑂 = (compf𝐶)
comfffval.b 𝐵 = (Base‘𝐶)
comfffval.h 𝐻 = (Hom ‘𝐶)
comfffval.x · = (comp‘𝐶)
Assertion
Ref Expression
comfffval 𝑂 = (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓)))
Distinct variable groups:   𝑥,𝑦,𝐵   𝑓,𝑔,𝑥,𝑦,𝐶   · ,𝑓,𝑔,𝑥   𝑓,𝐻,𝑔,𝑥
Allowed substitution hints:   𝐵(𝑓,𝑔)   · (𝑦)   𝐻(𝑦)   𝑂(𝑥,𝑦,𝑓,𝑔)

Proof of Theorem comfffval
Dummy variable 𝑐 is distinct from all other variables.
StepHypRef Expression
1 comfffval.o . 2 𝑂 = (compf𝐶)
2 fveq2 6922 . . . . . . 7 (𝑐 = 𝐶 → (Base‘𝑐) = (Base‘𝐶))
3 comfffval.b . . . . . . 7 𝐵 = (Base‘𝐶)
42, 3eqtr4di 2798 . . . . . 6 (𝑐 = 𝐶 → (Base‘𝑐) = 𝐵)
54sqxpeqd 5732 . . . . 5 (𝑐 = 𝐶 → ((Base‘𝑐) × (Base‘𝑐)) = (𝐵 × 𝐵))
6 fveq2 6922 . . . . . . . 8 (𝑐 = 𝐶 → (Hom ‘𝑐) = (Hom ‘𝐶))
7 comfffval.h . . . . . . . 8 𝐻 = (Hom ‘𝐶)
86, 7eqtr4di 2798 . . . . . . 7 (𝑐 = 𝐶 → (Hom ‘𝑐) = 𝐻)
98oveqd 7467 . . . . . 6 (𝑐 = 𝐶 → ((2nd𝑥)(Hom ‘𝑐)𝑦) = ((2nd𝑥)𝐻𝑦))
108fveq1d 6924 . . . . . 6 (𝑐 = 𝐶 → ((Hom ‘𝑐)‘𝑥) = (𝐻𝑥))
11 fveq2 6922 . . . . . . . . 9 (𝑐 = 𝐶 → (comp‘𝑐) = (comp‘𝐶))
12 comfffval.x . . . . . . . . 9 · = (comp‘𝐶)
1311, 12eqtr4di 2798 . . . . . . . 8 (𝑐 = 𝐶 → (comp‘𝑐) = · )
1413oveqd 7467 . . . . . . 7 (𝑐 = 𝐶 → (𝑥(comp‘𝑐)𝑦) = (𝑥 · 𝑦))
1514oveqd 7467 . . . . . 6 (𝑐 = 𝐶 → (𝑔(𝑥(comp‘𝑐)𝑦)𝑓) = (𝑔(𝑥 · 𝑦)𝑓))
169, 10, 15mpoeq123dv 7527 . . . . 5 (𝑐 = 𝐶 → (𝑔 ∈ ((2nd𝑥)(Hom ‘𝑐)𝑦), 𝑓 ∈ ((Hom ‘𝑐)‘𝑥) ↦ (𝑔(𝑥(comp‘𝑐)𝑦)𝑓)) = (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓)))
175, 4, 16mpoeq123dv 7527 . . . 4 (𝑐 = 𝐶 → (𝑥 ∈ ((Base‘𝑐) × (Base‘𝑐)), 𝑦 ∈ (Base‘𝑐) ↦ (𝑔 ∈ ((2nd𝑥)(Hom ‘𝑐)𝑦), 𝑓 ∈ ((Hom ‘𝑐)‘𝑥) ↦ (𝑔(𝑥(comp‘𝑐)𝑦)𝑓))) = (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓))))
18 df-comf 17731 . . . 4 compf = (𝑐 ∈ V ↦ (𝑥 ∈ ((Base‘𝑐) × (Base‘𝑐)), 𝑦 ∈ (Base‘𝑐) ↦ (𝑔 ∈ ((2nd𝑥)(Hom ‘𝑐)𝑦), 𝑓 ∈ ((Hom ‘𝑐)‘𝑥) ↦ (𝑔(𝑥(comp‘𝑐)𝑦)𝑓))))
193fvexi 6936 . . . . . 6 𝐵 ∈ V
2019, 19xpex 7790 . . . . 5 (𝐵 × 𝐵) ∈ V
2120, 19mpoex 8122 . . . 4 (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓))) ∈ V
2217, 18, 21fvmpt 7031 . . 3 (𝐶 ∈ V → (compf𝐶) = (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓))))
23 fvprc 6914 . . . 4 𝐶 ∈ V → (compf𝐶) = ∅)
24 fvprc 6914 . . . . . . 7 𝐶 ∈ V → (Base‘𝐶) = ∅)
253, 24eqtrid 2792 . . . . . 6 𝐶 ∈ V → 𝐵 = ∅)
2625olcd 873 . . . . 5 𝐶 ∈ V → ((𝐵 × 𝐵) = ∅ ∨ 𝐵 = ∅))
27 0mpo0 7535 . . . . 5 (((𝐵 × 𝐵) = ∅ ∨ 𝐵 = ∅) → (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓))) = ∅)
2826, 27syl 17 . . . 4 𝐶 ∈ V → (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓))) = ∅)
2923, 28eqtr4d 2783 . . 3 𝐶 ∈ V → (compf𝐶) = (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓))))
3022, 29pm2.61i 182 . 2 (compf𝐶) = (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓)))
311, 30eqtri 2768 1 𝑂 = (𝑥 ∈ (𝐵 × 𝐵), 𝑦𝐵 ↦ (𝑔 ∈ ((2nd𝑥)𝐻𝑦), 𝑓 ∈ (𝐻𝑥) ↦ (𝑔(𝑥 · 𝑦)𝑓)))
Colors of variables: wff setvar class
Syntax hints:  ¬ wn 3  wo 846   = wceq 1537  wcel 2108  Vcvv 3488  c0 4352   × cxp 5698  cfv 6575  (class class class)co 7450  cmpo 7452  2nd c2nd 8031  Basecbs 17260  Hom chom 17324  compcco 17325  compfccomf 17727
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1793  ax-4 1807  ax-5 1909  ax-6 1967  ax-7 2007  ax-8 2110  ax-9 2118  ax-10 2141  ax-11 2158  ax-12 2178  ax-ext 2711  ax-rep 5303  ax-sep 5317  ax-nul 5324  ax-pow 5383  ax-pr 5447  ax-un 7772
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 847  df-3an 1089  df-tru 1540  df-fal 1550  df-ex 1778  df-nf 1782  df-sb 2065  df-mo 2543  df-eu 2572  df-clab 2718  df-cleq 2732  df-clel 2819  df-nfc 2895  df-ne 2947  df-ral 3068  df-rex 3077  df-reu 3389  df-rab 3444  df-v 3490  df-sbc 3805  df-csb 3922  df-dif 3979  df-un 3981  df-in 3983  df-ss 3993  df-nul 4353  df-if 4549  df-pw 4624  df-sn 4649  df-pr 4651  df-op 4655  df-uni 4932  df-iun 5017  df-br 5167  df-opab 5229  df-mpt 5250  df-id 5593  df-xp 5706  df-rel 5707  df-cnv 5708  df-co 5709  df-dm 5710  df-rn 5711  df-res 5712  df-ima 5713  df-iota 6527  df-fun 6577  df-fn 6578  df-f 6579  df-f1 6580  df-fo 6581  df-f1o 6582  df-fv 6583  df-ov 7453  df-oprab 7454  df-mpo 7455  df-1st 8032  df-2nd 8033  df-comf 17731
This theorem is referenced by:  comffval  17759  comfffval2  17761  comfffn  17764  comfeq  17766
  Copyright terms: Public domain W3C validator