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

Theorem logbval 26824
Description: Define the value of the logb function, the logarithm generalized to an arbitrary base, when used as infix. Most Metamath statements select variables in order of their use, but to make the order clearer we use "B" for base and "X" for the argument of the logarithm function here. (Contributed by David A. Wheeler, 21-Jan-2017.) (Revised by David A. Wheeler, 16-Jul-2017.)
Assertion
Ref Expression
logbval ((𝐵 ∈ (ℂ ∖ {0, 1}) ∧ 𝑋 ∈ (ℂ ∖ {0})) → (𝐵 logb 𝑋) = ((log‘𝑋) / (log‘𝐵)))

Proof of Theorem logbval
Dummy variables 𝑥 𝑦 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 fveq2 6907 . . 3 (𝑥 = 𝐵 → (log‘𝑥) = (log‘𝐵))
21oveq2d 7447 . 2 (𝑥 = 𝐵 → ((log‘𝑦) / (log‘𝑥)) = ((log‘𝑦) / (log‘𝐵)))
3 fveq2 6907 . . 3 (𝑦 = 𝑋 → (log‘𝑦) = (log‘𝑋))
43oveq1d 7446 . 2 (𝑦 = 𝑋 → ((log‘𝑦) / (log‘𝐵)) = ((log‘𝑋) / (log‘𝐵)))
5 df-logb 26823 . 2 logb = (𝑥 ∈ (ℂ ∖ {0, 1}), 𝑦 ∈ (ℂ ∖ {0}) ↦ ((log‘𝑦) / (log‘𝑥)))
6 ovex 7464 . 2 ((log‘𝑋) / (log‘𝐵)) ∈ V
72, 4, 5, 6ovmpo 7593 1 ((𝐵 ∈ (ℂ ∖ {0, 1}) ∧ 𝑋 ∈ (ℂ ∖ {0})) → (𝐵 logb 𝑋) = ((log‘𝑋) / (log‘𝐵)))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 395   = wceq 1537  wcel 2106  cdif 3960  {csn 4631  {cpr 4633  cfv 6563  (class class class)co 7431  cc 11151  0cc0 11153  1c1 11154   / cdiv 11918  logclog 26611   logb clogb 26822
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1792  ax-4 1806  ax-5 1908  ax-6 1965  ax-7 2005  ax-8 2108  ax-9 2116  ax-10 2139  ax-11 2155  ax-12 2175  ax-ext 2706  ax-sep 5302  ax-nul 5312  ax-pr 5438
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 848  df-3an 1088  df-tru 1540  df-fal 1550  df-ex 1777  df-nf 1781  df-sb 2063  df-mo 2538  df-eu 2567  df-clab 2713  df-cleq 2727  df-clel 2814  df-nfc 2890  df-ne 2939  df-ral 3060  df-rex 3069  df-rab 3434  df-v 3480  df-sbc 3792  df-dif 3966  df-un 3968  df-ss 3980  df-nul 4340  df-if 4532  df-sn 4632  df-pr 4634  df-op 4638  df-uni 4913  df-br 5149  df-opab 5211  df-id 5583  df-xp 5695  df-rel 5696  df-cnv 5697  df-co 5698  df-dm 5699  df-iota 6516  df-fun 6565  df-fv 6571  df-ov 7434  df-oprab 7435  df-mpo 7436  df-logb 26823
This theorem is referenced by:  logbcl  26825  logbid1  26826  logb1  26827  elogb  26828  logbchbase  26829  relogbval  26830  relogbcl  26831  relogbreexp  26833  relogbmul  26835  nnlogbexp  26839  relogbcxp  26843  cxplogb  26844  logbgt0b  26851  dvrelog2b  42048  dvrelogpow2b  42050  rege1logbrege0  48408  logb2aval  48995
  Copyright terms: Public domain W3C validator