Skip to content

Commit b579a9f

Browse files
committed
chore: wip
1 parent 6ca2e9f commit b579a9f

File tree

2 files changed

+233
-209
lines changed

2 files changed

+233
-209
lines changed

src/Init/Data/BitVec/Bitblast.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2561,7 +2561,6 @@ def pps_layer {w : Nat} (iter_num : Nat) (old_layer : BitVec (old_length * w))
25612561
termination_by old_length - (iter_num * 2)
25622562

25632563

2564-
25652564
theorem extractLsb'_extractLsb'_eq_of_lt (a : BitVec w) (hlt : i + k ≤ len) :
25662565
extractLsb' i k (extractLsb' 0 len a) =
25672566
extractLsb' i k a := by
@@ -3002,6 +3001,7 @@ def pps (l : BitVec (l_length * w)) (k : BitVec w)
30023001
apply rec_add_eq_rec_add_iff (a := new_layer) (by omega) (b := l) (by omega) (by omega) (by omega) (n := (l_length + 1) / 2) (by omega)
30033002
pps new_layer k proof_sum_eq proof_new_layer_length hw
30043003

3004+
30053005
@[simp]
30063006
theorem cpopNatRec_zero_eq_self {x : BitVec w} :
30073007
x.cpopNatRec 0 acc = acc := rfl

0 commit comments

Comments
 (0)