Skip to content

Commit c38e2e1

Browse files
luisacicolinibollu
andauthored
chore: docstring
Co-authored-by: Siddharth <[email protected]>
1 parent dbc980f commit c38e2e1

File tree

1 file changed

+1
-3
lines changed

1 file changed

+1
-3
lines changed

src/Init/Data/BitVec/Basic.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -842,9 +842,7 @@ treating `x` and `y` as 2's complement signed bitvectors.
842842
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

845-
/--
846-
Count the number of leading zeros downward from the `n`-th bit to the `0`-th bit.
847-
-/
845+
/-- Count the number of leading zeros downward from the `n`-th bit to the `0`-th bit. -/
848846
def clzAux {w : Nat} (x : BitVec w) (n : Nat) : Nat :=
849847
match n with
850848
| 0 => if x.getLsbD 0 then 0 else 1

0 commit comments

Comments
 (0)