Commit 2023-11-30 23:41 1c6d0cef
View on Github →chore: bump Std, changes for leanprover/std4#366 (#8700)
Notably leanprover/std4#366 changed the definition of testBit
(to something equivalent) when upstreaming it, which broke a handful of proofs.
Other conflicting changes in Std, resolved for now by priming the mathlib name:
Std.BitVec.adc
: the type was changed fromBitVec (n + 1)
toBool × BitVec w
Nat.mul_add_mod
: the type was changed from(a * b + c) % b = c % b
to(b * a + c) % b = c % b
Zulip thread