Skip to content

Commit 62bb66b

Browse files
chore: docstring
Co-authored-by: Tobias Grosser <[email protected]>
1 parent f5b9869 commit 62bb66b

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Init/Data/BitVec/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -843,7 +843,7 @@ def smulOverflow {w : Nat} (x y : BitVec w) : Bool :=
843843
(x.toInt * y.toInt ≥ 2 ^ (w - 1)) || (x.toInt * y.toInt < - 2 ^ (w - 1))
844844

845845
/--
846-
Count the number of leading zeroes downward from the `n`-th bit to the `0`-th bit.
846+
Count the number of leading zeros downward from the `n`-th bit to the `0`-th bit.
847847
-/
848848
def clzAux {w : Nat} (x : BitVec w) (n : Nat) : Nat :=
849849
match n with

0 commit comments

Comments
 (0)