Skip to content

Commit

Permalink
removed simp
Browse files Browse the repository at this point in the history
  • Loading branch information
luisacicolini committed Sep 26, 2024
1 parent eace028 commit 87df10f
Showing 1 changed file with 0 additions and 1 deletion.
1 change: 0 additions & 1 deletion src/Init/Data/BitVec/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1512,7 +1512,6 @@ theorem shiftRight_add {w : Nat} (x : BitVec w) (n m : Nat) :
ext i
simp [Nat.add_assoc n m i]

@[simp]
theorem shiftLeft_ushiftRight {x : BitVec w} {n : Nat}:
x >>> n <<< n = x &&& BitVec.allOnes w <<< n := by
induction n generalizing x
Expand Down

0 comments on commit 87df10f

Please sign in to comment.