Skip to content

Commit

Permalink
chore: remove useless newline
Browse files Browse the repository at this point in the history
  • Loading branch information
luisacicolini authored Jan 16, 2025
1 parent 4dc9290 commit 32bbf2f
Showing 1 changed file with 0 additions and 1 deletion.
1 change: 0 additions & 1 deletion src/Init/Data/Nat/Bitwise/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -737,7 +737,6 @@ theorem shiftLeft_or_distrib {a b : Nat} : (a ||| b) <<< i = a <<< i ||| b <<< i
theorem shiftLeft_xor_distrib {a b : Nat} : (a ^^^ b) <<< i = a <<< i ^^^ b <<< i :=
shiftLeft_bitwise_distrib


@[simp] theorem decide_shiftRight_mod_two_eq_one :
decide (x >>> i % 2 = 1) = x.testBit i := by
simp only [testBit, one_and_eq_mod_two, mod_two_bne_zero]
Expand Down

0 comments on commit 32bbf2f

Please sign in to comment.