Skip to content

Commit

Permalink
chore: replace omega with proper theorem
Browse files Browse the repository at this point in the history
Co-authored-by: Alex Keizer <[email protected]>
  • Loading branch information
luisacicolini and alexkeizer authored Jan 21, 2025
1 parent f794c9e commit 4481757
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Init/Data/BitVec/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3796,7 +3796,7 @@ theorem getElem_replicate {n w : Nat} {x : BitVec w} (h : i < w * n) :
by_cases h' : w = 0 <;> simp [h'] <;> omega

@[simp]
theorem replicate_one {w : Nat} {x : BitVec w} (h : w = w * 1 := by omega) :
theorem replicate_one {w : Nat} {x : BitVec w} (h : w = w * 1 := Nat.mul_one _) :
(x.replicate 1) = x.cast h := by
simp [replicate, h]

Expand Down

0 comments on commit 4481757

Please sign in to comment.