Skip to content

Commit

Permalink
.
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 5, 2024
1 parent 03f864a commit c9e8dbb
Showing 1 changed file with 2 additions and 5 deletions.
7 changes: 2 additions & 5 deletions src/Lean/SimpLC/Whitelists/BitVec.lean
Original file line number Diff line number Diff line change
Expand Up @@ -56,11 +56,8 @@ simp_lc whitelist BitVec.udiv_one BitVec.udiv_self
-- example (x : BitVec 1) : x = if x = 0#1 then 0#1 else 1#1 := by bv_decide
simp_lc whitelist BitVec.udiv_eq_and BitVec.udiv_self

-- TODO: move to library
@[simp] theorem BitVec.ofFin_zero_sub {w : Nat} (i : Fin (2^w)) :
ofFin (0 - i) = - ofFin i := by
apply BitVec.eq_of_toNat_eq
simp [Fin.coe_sub]
example (w : Nat) : w = 00#w = 1#w := by rintro rfl; simp
simp_lc whitelist BitVec.sdiv_self BitVec.sdiv_one

/-
The actual checks happen in `tests/lean/run/simplc.lean`.
Expand Down

0 comments on commit c9e8dbb

Please sign in to comment.