Skip to content

Commit c1da100

Browse files
committed
chore: remove debug.byAsSorry
1 parent 6c97c4c commit c1da100

File tree

1 file changed

+0
-2
lines changed

1 file changed

+0
-2
lines changed

src/Init/Data/BitVec/Lemmas.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -570,7 +570,6 @@ theorem msb_zeroExtend (x : BitVec w) : (x.zeroExtend v).msb = (decide (0 < v) &
570570
theorem msb_zeroExtend' (x : BitVec w) (h : w ≤ v) : (x.zeroExtend' h).msb = (decide (0 < v) && x.getLsbD (v - 1)) := by
571571
rw [zeroExtend'_eq, msb_zeroExtend]
572572

573-
set_option debug.byAsSorry true in
574573
/-- zero extending a bitvector to width 1 equals the boolean of the lsb. -/
575574
theorem zeroExtend_one_eq_ofBool_getLsb_zero (x : BitVec w) :
576575
x.zeroExtend 1 = BitVec.ofBool (x.getLsbD 0) := by
@@ -587,7 +586,6 @@ theorem zeroExtend_ofNat_one_eq_ofNat_one_of_lt {v w : Nat} (hv : 0 < v) :
587586
have hv := Nat.testBit_one_eq_true_iff_self_eq_zero.mp hi₁
588587
omega
589588

590-
set_option debug.byAsSorry true in
591589
/-- Truncating to width 1 produces a bitvector equal to the least significant bit. -/
592590
theorem truncate_one {x : BitVec w} :
593591
x.truncate 1 = ofBool (x.getLsbD 0) := by

0 commit comments

Comments
 (0)