File tree Expand file tree Collapse file tree 2 files changed +1
-3
lines changed
Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Operations Expand file tree Collapse file tree 2 files changed +1
-3
lines changed Original file line number Diff line number Diff line change @@ -3270,8 +3270,6 @@ theorem addRecAux_extractAndExtendPopulateAux_le_of_le {x : BitVec w} (hn : n
32703270 · have := Nat.lt_two_pow_self (n := w + 1 + 1 )
32713271 omega
32723272
3273-
3274-
32753273theorem addRecAux_extractAndExtendPopulateAux_le_of_le_of_lt {x : BitVec (w + 1 )} (hn : n ≤ w) :
32763274 ((extractAndExtendPopulate w x).addRecAux n 0 #w).toNat ≤ n := by
32773275 induction n
Original file line number Diff line number Diff line change @@ -181,7 +181,7 @@ theorem denote_blastAddVec
181181 (new_layer : AIG.RefVec aig (iter_num * w))
182182 (hold' : 2 * (iter_num - 1 ) < old_length)
183183 (old_layer_bv : BitVec (old_length * w))
184- (hval : 0 < l_length)
184+ (_hval : 0 < l_length)
185185 (hw : 0 < w)
186186 -- the bits added already denote to the corresponding entry in acc
187187 (hold : ∀ (idx : Nat) (hidx : idx < old_length * w),
You can’t perform that action at this time.
0 commit comments