Skip to content

Commit

Permalink
Drop unused lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
tobiasgrosser committed Sep 18, 2024
1 parent fee34f8 commit 3c53089
Showing 1 changed file with 0 additions and 9 deletions.
9 changes: 0 additions & 9 deletions src/Init/Data/BitVec/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -232,15 +232,6 @@ theorem ofNat_one (n : Nat) : BitVec.ofNat 1 n = BitVec.ofBool (n % 2 = 1) := b
theorem ofBool_eq_iff_eq : ∀ {b b' : Bool}, BitVec.ofBool b = BitVec.ofBool b' ↔ b = b' := by
decide

@[simp] theorem and_ofBool : ofBool a &&& ofBool b = ofBool (a && b) := by
cases a <;> cases b <;> rfl

@[simp] theorem or_ofBool : ofBool a ||| ofBool b = ofBool (a || b) := by
cases a <;> cases b <;> rfl

@[simp] theorem xor_ofBool : ofBool a ^^^ ofBool b = ofBool (a ^^ b) := by
cases a <;> cases b <;> rfl

@[simp] theorem not_ofBool : ~~~ (ofBool b) = ofBool (!b) := by cases b <;> rfl

@[simp] theorem ofBool_and_ofBool : ofBool b &&& ofBool b' = ofBool (b && b') := by
Expand Down

0 comments on commit 3c53089

Please sign in to comment.