Skip to content

Commit 3861dda

Browse files
committed
Recurrence
1 parent 6612208 commit 3861dda

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/Init/Data/BitVec/Bitblast.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -326,8 +326,8 @@ theorem zeroExtend_truncate_succ_eq_zeroExtend_truncate_add_twoPow (x : BitVec w
326326
by_cases hi : x.getLsb i <;> simp [hi] <;> omega
327327

328328
/--
329-
Recurrence lemma: multiplying `l` with the first `s` bits of `r` is the
330-
same as truncating `r` to `s` bits, then zero extending to the original length,
329+
Recurrence lemma: multiplying `x` with the first `s` bits of `y` is the
330+
same as truncating `y` to `s` bits, then zero extending to the original length,
331331
and performing the multplication. -/
332332
theorem mulRec_eq_mul_signExtend_truncate (x y : BitVec w) (s : Nat) :
333333
mulRec x y s = x * ((y.truncate (s + 1)).zeroExtend w) := by

0 commit comments

Comments
 (0)