Skip to content
This repository has been archived by the owner on Aug 29, 2024. It is now read-only.

Commit

Permalink
test: adapt test for arbitrary shiftRight
Browse files Browse the repository at this point in the history
  • Loading branch information
hargoniX committed Aug 1, 2024
1 parent d71085f commit 20ff265
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions Test/Bv/Shift.lean
Original file line number Diff line number Diff line change
Expand Up @@ -26,9 +26,8 @@ set_option trace.bv true in
theorem shift_unit_5 {x y z : BitVec 16} : (x <<< y) <<< z = (x <<< z) <<< y := by
bv_decide

-- This demonstrates we correctly abstract shifts of arbitrary width as atoms instead of giving up.
set_option trace.bv true in
theorem shift_unit_6 {x y : BitVec 64} : (x >>> y) + y = y + (x >>> y) := by
theorem shift_unit_6 {x y z : BitVec 16} : (x >>> y) >>> z = (x >>> z) >>> y := by
bv_decide

set_option trace.bv true in
Expand Down

0 comments on commit 20ff265

Please sign in to comment.