Skip to content

Commit d50909f

Browse files
committed
chore: undo change
1 parent 6c94430 commit d50909f

File tree

1 file changed

+4
-1
lines changed

1 file changed

+4
-1
lines changed

src/Init/Data/BitVec/Lemmas.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1147,7 +1147,10 @@ theorem signExtend_eq_not_zeroExtend_not_of_msb_false {x : BitVec w} {v : Nat} (
11471147
x.signExtend v = x.zeroExtend v := by
11481148
ext i
11491149
by_cases hv : i < v
1150-
· simp [signExtend, toInt_eq_msb_cond, hmsb]
1150+
· simp only [signExtend, getLsbD, getLsbD_zeroExtend, hv, decide_True, Bool.true_and, toNat_ofInt,
1151+
BitVec.toInt_eq_msb_cond, hmsb, ↓reduceIte, reduceCtorEq]
1152+
rw [Int.ofNat_mod_ofNat, Int.toNat_ofNat, Nat.testBit_mod_two_pow]
1153+
simp [BitVec.testBit_toNat]
11511154
· simp only [getLsbD_zeroExtend, hv, decide_False, Bool.false_and]
11521155
apply getLsbD_ge
11531156
omega

0 commit comments

Comments
 (0)