File tree Expand file tree Collapse file tree 1 file changed +0
-2
lines changed Expand file tree Collapse file tree 1 file changed +0
-2
lines changed Original file line number Diff line number Diff line change @@ -570,7 +570,6 @@ theorem msb_zeroExtend (x : BitVec w) : (x.zeroExtend v).msb = (decide (0 < v) &
570
570
theorem msb_zeroExtend' (x : BitVec w) (h : w ≤ v) : (x.zeroExtend' h).msb = (decide (0 < v) && x.getLsbD (v - 1 )) := by
571
571
rw [zeroExtend'_eq, msb_zeroExtend]
572
572
573
- set_option debug.byAsSorry true in
574
573
/-- zero extending a bitvector to width 1 equals the boolean of the lsb. -/
575
574
theorem zeroExtend_one_eq_ofBool_getLsb_zero (x : BitVec w) :
576
575
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) :
587
586
have hv := Nat.testBit_one_eq_true_iff_self_eq_zero.mp hi₁
588
587
omega
589
588
590
- set_option debug.byAsSorry true in
591
589
/-- Truncating to width 1 produces a bitvector equal to the least significant bit. -/
592
590
theorem truncate_one {x : BitVec w} :
593
591
x.truncate 1 = ofBool (x.getLsbD 0 ) := by
You can’t perform that action at this time.
0 commit comments