Users' Mathboxes Mathbox for Alexander van der Vekens < Previous   Next >
Nearby theorems
Mirrors  >  Home  >  MPE Home  >  Th. List  >   Mathboxes  >  df-dig Structured version   Visualization version   GIF version

Definition df-dig 42390
Description: Definition of an operation to obtain the 𝑘 th digit of a nonnegative real number 𝑟 in the positional system with base 𝑏. 𝑘 = − 1 corresponds to the first digit of the fractional part (for 𝑏 = 10 the first digit after the decimal point), 𝑘 = 0 corresponds to the last digit of the integer part (for 𝑏 = 10 the first digit before the decimal point). See also digit1 12998. Examples (not formal): ( 234.567 ( digit ` 10 ) 0 ) = 4; ( 2.567 ( digit ` 10 ) -2 ) = 6; ( 2345.67 ( digit ` 10 ) 2 ) = 3. (Contributed by AV, 16-May-2020.)
Assertion
Ref Expression
df-dig digit = (𝑏 ∈ ℕ ↦ (𝑘 ∈ ℤ, 𝑟 ∈ (0[,)+∞) ↦ ((⌊‘((𝑏↑-𝑘) · 𝑟)) mod 𝑏)))
Distinct variable group:   𝑘,𝑏,𝑟

Detailed syntax breakdown of Definition df-dig
StepHypRef Expression
1 cdig 42389 . 2 class digit
2 vb . . 3 setvar 𝑏
3 cn 11020 . . 3 class
4 vk . . . 4 setvar 𝑘
5 vr . . . 4 setvar 𝑟
6 cz 11377 . . . 4 class
7 cc0 9936 . . . . 5 class 0
8 cpnf 10071 . . . . 5 class +∞
9 cico 12177 . . . . 5 class [,)
107, 8, 9co 6650 . . . 4 class (0[,)+∞)
112cv 1482 . . . . . . . 8 class 𝑏
124cv 1482 . . . . . . . . 9 class 𝑘
1312cneg 10267 . . . . . . . 8 class -𝑘
14 cexp 12860 . . . . . . . 8 class
1511, 13, 14co 6650 . . . . . . 7 class (𝑏↑-𝑘)
165cv 1482 . . . . . . 7 class 𝑟
17 cmul 9941 . . . . . . 7 class ·
1815, 16, 17co 6650 . . . . . 6 class ((𝑏↑-𝑘) · 𝑟)
19 cfl 12591 . . . . . 6 class
2018, 19cfv 5888 . . . . 5 class (⌊‘((𝑏↑-𝑘) · 𝑟))
21 cmo 12668 . . . . 5 class mod
2220, 11, 21co 6650 . . . 4 class ((⌊‘((𝑏↑-𝑘) · 𝑟)) mod 𝑏)
234, 5, 6, 10, 22cmpt2 6652 . . 3 class (𝑘 ∈ ℤ, 𝑟 ∈ (0[,)+∞) ↦ ((⌊‘((𝑏↑-𝑘) · 𝑟)) mod 𝑏))
242, 3, 23cmpt 4729 . 2 class (𝑏 ∈ ℕ ↦ (𝑘 ∈ ℤ, 𝑟 ∈ (0[,)+∞) ↦ ((⌊‘((𝑏↑-𝑘) · 𝑟)) mod 𝑏)))
251, 24wceq 1483 1 wff digit = (𝑏 ∈ ℕ ↦ (𝑘 ∈ ℤ, 𝑟 ∈ (0[,)+∞) ↦ ((⌊‘((𝑏↑-𝑘) · 𝑟)) mod 𝑏)))
Colors of variables: wff setvar class
This definition is referenced by:  digfval  42391
  Copyright terms: Public domain W3C validator