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

Theorem logbval 25336
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 6663 . . 3 (𝑥 = 𝐵 → (log‘𝑥) = (log‘𝐵))
21oveq2d 7164 . 2 (𝑥 = 𝐵 → ((log‘𝑦) / (log‘𝑥)) = ((log‘𝑦) / (log‘𝐵)))
3 fveq2 6663 . . 3 (𝑦 = 𝑋 → (log‘𝑦) = (log‘𝑋))
43oveq1d 7163 . 2 (𝑦 = 𝑋 → ((log‘𝑦) / (log‘𝐵)) = ((log‘𝑋) / (log‘𝐵)))
5 df-logb 25335 . 2 logb = (𝑥 ∈ (ℂ ∖ {0, 1}), 𝑦 ∈ (ℂ ∖ {0}) ↦ ((log‘𝑦) / (log‘𝑥)))
6 ovex 7181 . 2 ((log‘𝑋) / (log‘𝐵)) ∈ V
72, 4, 5, 6ovmpo 7302 1 ((𝐵 ∈ (ℂ ∖ {0, 1}) ∧ 𝑋 ∈ (ℂ ∖ {0})) → (𝐵 logb 𝑋) = ((log‘𝑋) / (log‘𝐵)))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 398   = wceq 1531  wcel 2108  cdif 3931  {csn 4559  {cpr 4561  cfv 6348  (class class class)co 7148  cc 10527  0cc0 10529  1c1 10530   / cdiv 11289  logclog 25130   logb clogb 25334
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1790  ax-4 1804  ax-5 1905  ax-6 1964  ax-7 2009  ax-8 2110  ax-9 2118  ax-10 2139  ax-11 2154  ax-12 2170  ax-ext 2791  ax-sep 5194  ax-nul 5201  ax-pr 5320
This theorem depends on definitions:  df-bi 209  df-an 399  df-or 844  df-3an 1084  df-tru 1534  df-ex 1775  df-nf 1779  df-sb 2064  df-mo 2616  df-eu 2648  df-clab 2798  df-cleq 2812  df-clel 2891  df-nfc 2961  df-ral 3141  df-rex 3142  df-rab 3145  df-v 3495  df-sbc 3771  df-dif 3937  df-un 3939  df-in 3941  df-ss 3950  df-nul 4290  df-if 4466  df-sn 4560  df-pr 4562  df-op 4566  df-uni 4831  df-br 5058  df-opab 5120  df-id 5453  df-xp 5554  df-rel 5555  df-cnv 5556  df-co 5557  df-dm 5558  df-iota 6307  df-fun 6350  df-fv 6356  df-ov 7151  df-oprab 7152  df-mpo 7153  df-logb 25335
This theorem is referenced by:  logbcl  25337  logbid1  25338  logb1  25339  elogb  25340  logbchbase  25341  relogbval  25342  relogbcl  25343  relogbreexp  25345  relogbmul  25347  nnlogbexp  25351  relogbcxp  25355  cxplogb  25356  logbgt0b  25363  rege1logbrege0  44608  logb2aval  44853
  Copyright terms: Public domain W3C validator