We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent fabf410 commit 2245d6aCopy full SHA for 2245d6a
src/Init/Data/BitVec/Lemmas.lean
@@ -6426,7 +6426,7 @@ theorem cpopNatRec_cons_eq_toNat_add_cpopNatRec_of_lt {x : BitVec w} {b : Bool}
6426
induction n generalizing acc
6427
· omega
6428
· case _ n ihn =>
6429
- simp
+ simp only [cpopNatRec_succ]
6430
by_cases hlt : w < n
6431
· specialize ihn (acc := acc + ((cons b x).getLsbD n).toNat) (by omega)
6432
rw [ihn, Nat.add_left_cancel_iff, getLsbD_cons]
0 commit comments