Skip to content

Commit

Permalink
chore: remove unused theorem
Browse files Browse the repository at this point in the history
  • Loading branch information
tobiasgrosser committed Apr 29, 2024
1 parent b047683 commit 75fc12c
Showing 1 changed file with 2 additions and 6 deletions.
8 changes: 2 additions & 6 deletions SSA/Projects/InstCombine/AliveHandwrittenLargeExamples.lean
Original file line number Diff line number Diff line change
Expand Up @@ -62,9 +62,6 @@ axioms: [propext, Classical.choice, Quot.sound] -/
end DivRemOfSelect

namespace AndOrXor

open LLVMTheory

/-
Name: AndOrXor:2515 ((X^C1) >> C2)^C3 = (X>>C2) ^ ((C1>>C2)^C3)
%e1 = xor %x, C1
Expand All @@ -78,6 +75,8 @@ Name: AndOrXor:2515 ((X^C1) >> C2)^C3 = (X>>C2) ^ ((C1>>C2)^C3)
-/

open ComWrappers
open LLVMTheory

def AndOrXor2515_lhs (w : ℕ):
Com InstCombine.LLVM
[/- C1 -/ InstCombine.Ty.bitvec w,
Expand Down Expand Up @@ -110,9 +109,6 @@ def xor_assoc (c1 c2 c3 : BitVec w): c1 ^^^ c2 ^^^ c3 = c1 ^^^ (c2 ^^^ c3) := by
ext i
simp

def help'' {a b : Nat } : a = b ↔ (↑a : Int) = ↑b := by
simp only [Nat.cast_inj]

def alive_simplifyAndOrXor2515 (w : Nat) :
AndOrXor2515_lhs w ⊑ AndOrXor2515_rhs w := by
simp only [AndOrXor2515_lhs, AndOrXor2515_rhs]
Expand Down

0 comments on commit 75fc12c

Please sign in to comment.