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

Commit

Permalink
refactor: split out tactics
Browse files Browse the repository at this point in the history
  • Loading branch information
hargoniX committed Jul 15, 2024
1 parent 6890bde commit 811cf72
Show file tree
Hide file tree
Showing 119 changed files with 125 additions and 137 deletions.
2 changes: 1 addition & 1 deletion Eval/Popcount.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

/-
This is based on: https://saw.galois.com/intro/IntroToSAW.html#the-code
Expand Down
2 changes: 1 addition & 1 deletion Eval/WillOverflow.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

/-
This file is based on: https://grack.com/blog/2022/12/20/deriving-a-bit-twiddling-hack/
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_152.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_152 :
∀ (x : BitVec 8), x * -1 = 0 - x
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_160.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_160 :
∀ (x C1 C2 : BitVec 7), x <<< C2 * C1 = x * C1 <<< C2
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_229.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_229 :
∀ (X C1 Op1 : BitVec 4), (X + C1) * Op1 = X * Op1 + C1 * Op1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_239.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_239 :
∀ (Y X : BitVec 8), (0 - X) * (0 - Y) = X * Y
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_283.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_283 :
∀ (Y X : BitVec 1), X * Y = X &&& Y
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_290__292.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide
open BitVec

theorem bitvec_290__292 :
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1043.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1043 :
∀ (C1 Z RHS : BitVec 64), (Z &&& C1 ^^^ C1) + 1 + RHS = RHS - (Z ||| ~~~C1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1152.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1152 :
∀ (y x : BitVec 1), x + y = x ^^^ y
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1156.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1156 :
∀ (b : BitVec 64), b + b = b <<< 1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1164.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1164 :
∀ (a b : BitVec 64), 0 - a + b = b - a
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1165.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1165 :
∀ (a b : BitVec 64), 0 - a + (0 - b) = 0 - (a + b)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1176.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1176 :
∀ (a b : BitVec 64), a + (0 - b) = a - b
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1202.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1202 :
∀ (x C : BitVec 64), (x ^^^ -1) + C = C - 1 - x
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1295.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1295 :
∀ (a b : BitVec 64), (a &&& b) + (a ^^^ b) = a ||| b
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1309.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1309 :
∀ (a b : BitVec 64), (a &&& b) + (a ||| b) = a + b
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1539.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1539 :
∀ (a x : BitVec 64), x - (0 - a) = x + a
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1539_2.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1539_2 :
∀ (x C : BitVec 64), x - C = x + -C
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1556.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1556 :
∀ (y x : BitVec 1), x - y = x ^^^ y
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1560.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1560 :
∀ (a : BitVec 64), -1 - a = a ^^^ -1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1564.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1564 :
∀ (x C : BitVec 64), C - (x ^^^ -1) = x + (C + 1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1574.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1574 :
∀ (X C C2 : BitVec 64), C - (X + C2) = C - C2 - X
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1614.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1614 :
∀ (Y X : BitVec 64), X - (X + Y) = 0 - Y
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1619.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1619 :
∀ (Y X : BitVec 64), X - Y - X = 0 - Y
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AddSub_1624.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AddSub_1624 :
∀ (A B : BitVec 64), (A ||| B) - (A ^^^ B) = A &&& B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1230__A__B___A__B.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1230__A__B___A__B :
∀ (notOp0 notOp1 : BitVec 64), (notOp0 ^^^ -1) &&& (notOp1 ^^^ -1) = (notOp0 ||| notOp1) ^^^ -1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1241_AB__AB__AB.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1241_AB__AB__AB :
∀ (A B : BitVec 64), (A ||| B) &&& (A &&& B ^^^ -1) = A ^^^ B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1247_AB__AB__AB.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1247_AB__AB__AB :
∀ (A B : BitVec 64), (A &&& B ^^^ -1) &&& (A ||| B) = A ^^^ B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1253_A__AB___A__B.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1253_A__AB___A__B :
∀ (A B : BitVec 64), (A ^^^ B) &&& A = A &&& (B ^^^ -1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1280_ABA___AB.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1280_ABA___AB :
∀ (A B : BitVec 64), (A ^^^ -1 ||| B) &&& A = A &&& B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1288_A__B__B__C__A___A__B__C.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1288_A__B__B__C__A___A__B__C :
∀ (A C B : BitVec 64), (A ^^^ B) &&& (B ^^^ C ^^^ A) = (A ^^^ B) &&& (C ^^^ -1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1294_A__B__A__B___A__B.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1294_A__B__A__B___A__B :
∀ (A B : BitVec 64), (A ||| B) &&& (A ^^^ -1 ^^^ B) = A &&& B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_135.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_135 :
∀ (X C1 C2 : BitVec 64), (X ^^^ C1) &&& C2 = X &&& C2 ^^^ C1 &&& C2
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_144.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_144 :
∀ (X C1 C2 : BitVec 64), (X ||| C1) &&& C2 = (X ||| C1 &&& C2) &&& C2
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1683_1.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

open BitVec

Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1683_2.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1683_2 :
∀ (a b : BitVec 64), (b ≤ a) || (a != b) = true
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1704.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1704 :
∀ (A B : BitVec 64), ((B == 0) || (A < B)) = (A ≤ B + -1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1705.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1705 :
∀ (A B : BitVec 64), ((B == 0) || (A < B)) = (A ≤ B + -1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_1733.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_1733 :
∀ (A B : BitVec 64), (A != 0) ∨ (B != 0) = (A ||| B != 0)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2063__X__C1__C2____X__C2__C1__C2.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2063__X__C1__C2____X__C2__C1__C2 :
∀ (x C1 C : BitVec 64), x ^^^ C1 ||| C = (x ||| C) ^^^ C1 &&& ~~~C
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2113___A__B__A___A__B.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2113___A__B__A___A__B :
∀ (A B : BitVec 64), (A ^^^ -1) &&& B ||| A = A ||| B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2118___A__B__A___A__B.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2118___A__B__A___A__B :
∀ (A B : BitVec 64), A &&& B ||| A ^^^ -1 = A ^^^ -1 ||| B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2123___A__B__A__B___A__B.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2123___A__B__A__B___A__B :
∀ (A B : BitVec 64), A &&& (B ^^^ -1) ||| A ^^^ B = A ^^^ B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2188.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2188 :
∀ (A D : BitVec 64), A &&& (D ^^^ -1) ||| (A ^^^ -1) &&& D = A ^^^ D
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2231__A__B__B__C__A___A__B__C.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2231__A__B__B__C__A___A__B__C :
∀ (A C B : BitVec 64), A ^^^ B ||| B ^^^ C ^^^ A = A ^^^ B ||| C
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2243__B__C__A__B___B__A__C.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2243__B__C__A__B___B__A__C :
∀ (A C B : BitVec 64), (B ||| C) &&& A ||| B = B ||| A &&& C
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2247__A__B__A__B.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2247__A__B__A__B :
∀ (A B : BitVec 64), A ^^^ -1 ||| B ^^^ -1 = A &&& B ^^^ -1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2263.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2263 :
∀ (B op0 : BitVec 64), op0 ||| op0 ^^^ B = op0 ||| B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2264.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2264 :
∀ (A B : BitVec 64), A ||| A ^^^ -1 ^^^ B = A ||| B ^^^ -1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2265.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2265 :
∀ (A B : BitVec 64), A &&& B ||| A ^^^ B = A ||| B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2284.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2284 :
∀ (A B : BitVec 64), A ||| (A ||| B) ^^^ -1 = A ||| B ^^^ -1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2285.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2285 :
∀ (A B : BitVec 64), A ||| A ^^^ B ^^^ -1 = A ||| B ^^^ -1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2297.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2297 :
∀ (A B : BitVec 64), A &&& B ||| A ^^^ -1 ^^^ B = A ^^^ -1 ^^^ B
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2367.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2367 :
∀ (A C1 op1 : BitVec 64), A ||| C1 ||| op1 = A ||| op1 ||| C1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2416.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2416 :
∀ (nx y : BitVec 64), (nx ^^^ -1) &&& y ^^^ -1 = nx ||| y ^^^ -1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2417.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2417 :
∀ (nx y : BitVec 64), (nx ^^^ -1 ||| y) ^^^ -1 = nx &&& (y ^^^ -1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2429.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2429 :
∀ (y x : BitVec 64), x &&& y ^^^ -1 = x ^^^ -1 ||| y ^^^ -1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2430.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2430 :
∀ (y x : BitVec 64), (x ||| y) ^^^ -1 = (x ^^^ -1) &&& (y ^^^ -1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2443.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

open BitVec

Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2475.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2475 :
∀ (x C : BitVec 64), C - x ^^^ -1 = x + (-1 - C)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2486.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2486 :
∀ (x C : BitVec 64), x + C ^^^ -1 = -1 - C - x
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2581__BAB___A__B.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2581__BAB___A__B :
∀ (a op1 : BitVec 64), (a ||| op1) ^^^ op1 = a &&& (op1 ^^^ -1)
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2587__BAA___B__A.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2587__BAA___B__A :
∀ (a op1 : BitVec 64), a &&& op1 ^^^ op1 = (a ^^^ -1) &&& op1
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2595.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2595 :
∀ (a b : BitVec 64), a &&& b ^^^ (a ||| b) = a ^^^ b
Expand Down
2 changes: 1 addition & 1 deletion Eval/bitvec_AndOrXor_2607.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import LeanSAT.Reflect.Tactics.BVDecide
import LeanSAT.Tactics.BVDecide

theorem bitvec_AndOrXor_2607 :
∀ (a b : BitVec 64), (a ||| b ^^^ -1) ^^^ (a ^^^ -1 ||| b) = a ^^^ b
Expand Down
Loading

0 comments on commit 811cf72

Please sign in to comment.