Skip to content

Commit

Permalink
chore: remove open Std (BitVec) (#535)
Browse files Browse the repository at this point in the history
... as well as outdated BitVec imports.
  • Loading branch information
tobiasgrosser authored Aug 15, 2024
1 parent e7dd381 commit b281345
Show file tree
Hide file tree
Showing 248 changed files with 0 additions and 257 deletions.
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/AliveAutoGenerated.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,6 @@ import SSA.Projects.InstCombine.Refinement
import SSA.Projects.InstCombine.Tactic

open MLIR AST
open Std (BitVec)
open Ctxt (Var)

namespace AliveAutoGenerated
Expand Down
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/AliveHandwrittenExamples.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,6 @@ import SSA.Projects.InstCombine.ForStd
import SSA.Core.ErasedContext

open MLIR AST
open Std (BitVec)
open Ctxt (Var DerivedCtxt)
open InstCombine (MOp)

Expand Down
2 changes: 0 additions & 2 deletions SSA/Projects/InstCombine/AliveHandwrittenLargeExamples.lean
Original file line number Diff line number Diff line change
Expand Up @@ -114,7 +114,6 @@ def MulDivRem805_rhs (w : ℕ) : Com InstCombine.LLVM
/- r = -/ Com.var (select w /-%c-/ 1 /-X-/ 5 /-c0-/ 0) <|
Com.ret ⟨/-r-/0, by simp [Ctxt.snoc]⟩

open Std (BitVec) in
def alive_simplifyMulDivRem805 (w : Nat) :
MulDivRem805_lhs w ⊑ MulDivRem805_rhs w := by
unfold MulDivRem805_lhs MulDivRem805_rhs
Expand Down Expand Up @@ -223,7 +222,6 @@ info: 'AliveHandwritten.MulDivRem.alive_simplifyMulDivRem805' depends on axioms:
-/
#guard_msgs in #print axioms alive_simplifyMulDivRem805

open Std (BitVec) in
def alive_simplifyMulDivRem805' (w : Nat) :
MulDivRem805_lhs w ⊑ MulDivRem805_rhs w := by
unfold MulDivRem805_lhs MulDivRem805_rhs
Expand Down
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/ForMathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ import Mathlib.Data.Nat.Bitwise
import Mathlib.Algebra.Group.Fin.Basic
import Mathlib.Data.Nat.Bits
import Mathlib.Data.ZMod.Defs
import Batteries.Data.BitVec

namespace BitVec
open Nat
Expand Down
5 changes: 0 additions & 5 deletions SSA/Projects/InstCombine/HackersDelight.lean
Original file line number Diff line number Diff line change
@@ -1,11 +1,6 @@
import Init.Data.BitVec.Basic
import Init.Data.BitVec.Lemmas
import Init.Data.BitVec.Bitblast
import SSA.Projects.InstCombine.ForMathlib
import SSA.Projects.InstCombine.ForStd
import SSA.Projects.InstCombine.TacticAuto
import Init.Data.Nat.Bitwise.Basic
import Init.Data.Nat.Bitwise.Lemmas

set_option linter.unusedTactic false
set_option linter.unreachableTactic false
Expand Down
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/LLVM/EDSL.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
-/
import Qq
import SSA.Projects.InstCombine.Base
import Batteries.Data.BitVec
import SSA.Core.MLIRSyntax.EDSL
import SSA.Projects.InstCombine.LLVM.CLITests

Expand Down
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/LLVM/Enumerator.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,6 @@
Released under Apache 2.0 license as described in the file LICENSE.
-/
-- Script that exhaustive enumerates the our LLVM semantics.
import Batteries.Data.BitVec
import Init.System.IO
import SSA.Core.Util
import SSA.Projects.InstCombine.LLVM.Semantics
Expand Down
3 changes: 0 additions & 3 deletions SSA/Projects/InstCombine/PaperExamples.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,9 +7,6 @@ import SSA.Projects.InstCombine.Tactic
import SSA.Projects.InstCombine.TacticAuto
import SSA.Projects.InstCombine.Base
import SSA.Projects.InstCombine.ForLean
import Init.Data.BitVec.Bitblast
import Init.Data.BitVec.Lemmas
import Init.Data.BitVec.Folds
import Lean


Expand Down
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,6 @@ import SSA.Projects.InstCombine.ForStd
import Mathlib.Tactic
import SSA.Core.ErasedContext
import SSA.Core.Tactic
import Batteries.Data.BitVec

open MLIR AST

Expand Down
3 changes: 0 additions & 3 deletions SSA/Projects/InstCombine/TacticAuto.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,11 +2,8 @@
Released under Apache 2.0 license as described in the file LICENSE.
-/
import Mathlib.Tactic.Ring
import Batteries.Data.BitVec
import SSA.Projects.InstCombine.ForLean

import SSA.Projects.InstCombine.LLVM.EDSL
import Batteries.Data.BitVec

attribute [simp_llvm_case_bash]
BitVec.Refinement.refl BitVec.Refinement.some_some BitVec.Refinement.none_left
Expand Down
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/TestLLVMOps.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ import SSA.Projects.InstCombine.LLVM.PrettyEDSL
import SSA.Projects.InstCombine.LLVM.CLITests

open MLIR AST
open Std (BitVec)
open Ctxt (Var)

-- Hardcoding the i4 for now, should change to w once I get
Expand Down
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/scripts/mlir-tool.py
Original file line number Diff line number Diff line change
Expand Up @@ -175,7 +175,6 @@ def {name}_after := [llvm|
open BitVec
open MLIR AST
open Std (BitVec)
open Ctxt (Var)
set_option linter.deprecated false
Expand Down
1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/scripts/types.py
Original file line number Diff line number Diff line change
Expand Up @@ -49,7 +49,6 @@ def process_file(file_path):
with open(proof_name + ".lean", "a") as file:
file.write(
"""
open Std (BitVec)
"""
)
for _, n, m in named:
Expand Down

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/g2008h05h31hBools.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gadd2.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gadd2_proof.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gadd4.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gadd4_proof.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gadd_or_sub.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gadd_or_sub_proof.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gaddhmask.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gaddhmask_proof.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gaddhmaskhneg.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gaddhshift.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 0 additions & 1 deletion SSA/Projects/InstCombine/tests/LLVM/gaddhshift_proof.lean

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Loading

0 comments on commit b281345

Please sign in to comment.