Skip to content

Commit 83f382f

Browse files
committed
chore: docs
1 parent 6edbfcd commit 83f382f

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Init/Data/BitVec/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5628,7 +5628,7 @@ theorem msb_replicate {n w : Nat} {x : BitVec w} :
56285628
simp only [BitVec.msb, getMsbD_replicate, Nat.zero_mod]
56295629
cases n <;> cases w <;> simp
56305630

5631-
/-! ### Leading zeroes -/
5631+
/-! ### Count leading zeroes -/
56325632

56335633
theorem clzAux_eq_zero_iff {x : BitVec w} {n : Nat} :
56345634
clzAux x n = 0 ↔ x.getLsbD n = true := by

0 commit comments

Comments
 (0)