Skip to content

Commit 261941d

Browse files
committed
fix: restore accidental edit
1 parent 25de019 commit 261941d

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Init/Data/Nat/Bitwise/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -616,7 +616,7 @@ theorem or_mod_two_pow : (a ||| b) % 2 ^ n = a % 2 ^ n ||| b % 2 ^ n :=
616616

617617
@[simp, grind =] theorem testBit_xor (x y i : Nat) :
618618
(x ^^^ y).testBit i = ((x.testBit i) ^^ (y.testBit i)) := by
619-
simp [HXor.hXor, XorOp.xor, xor, testBit_bitwise]
619+
simp [HXor.hXor, XorOp.xor, xor, testBit_bitwise ]
620620

621621
@[simp, grind =] theorem zero_xor (x : Nat) : 0 ^^^ x = x := by
622622
apply Nat.eq_of_testBit_eq

0 commit comments

Comments
 (0)