Skip to content

Commit

Permalink
chore: fix non-term simp
Browse files Browse the repository at this point in the history
  • Loading branch information
luisacicolini committed Jan 16, 2025
1 parent 6537834 commit 6092449
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 @@ -3459,7 +3459,7 @@ theorem replicate_append_self {x : BitVec w} :
| succ n ih =>
rw [replicate_succ]
conv => lhs; rw [ih]
simp [cast_cast, cast_eq]
simp only [cast_cast, cast_eq]
rw [← cast_append_left]
· rw [append_assoc]; congr
· rw [Nat.add_comm, Nat.mul_add, Nat.mul_one]; omega
Expand Down

0 comments on commit 6092449

Please sign in to comment.