We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 6612208 commit 3861ddaCopy full SHA for 3861dda
src/Init/Data/BitVec/Bitblast.lean
@@ -326,8 +326,8 @@ theorem zeroExtend_truncate_succ_eq_zeroExtend_truncate_add_twoPow (x : BitVec w
326
by_cases hi : x.getLsb i <;> simp [hi] <;> omega
327
328
/--
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,
+Recurrence lemma: multiplying `x` with the first `s` bits of `y` is the
+same as truncating `y` to `s` bits, then zero extending to the original length,
331
and performing the multplication. -/
332
theorem mulRec_eq_mul_signExtend_truncate (x y : BitVec w) (s : Nat) :
333
mulRec x y s = x * ((y.truncate (s + 1)).zeroExtend w) := by
0 commit comments