Skip to content

Commit

Permalink
fix tests
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Dec 3, 2024
1 parent ea60bba commit b07115b
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 86 deletions.
1 change: 0 additions & 1 deletion Batteries.lean
Original file line number Diff line number Diff line change
Expand Up @@ -93,7 +93,6 @@ import Batteries.Tactic.ShowUnused
import Batteries.Tactic.SqueezeScope
import Batteries.Tactic.Trans
import Batteries.Tactic.Unreachable
import Batteries.Tactic.Where
import Batteries.Util.Cache
import Batteries.Util.ExtendedBinder
import Batteries.Util.LibraryNote
Expand Down
83 changes: 0 additions & 83 deletions Batteries/Tactic/Where.lean

This file was deleted.

7 changes: 5 additions & 2 deletions BatteriesTest/where.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,7 @@
import Batteries.Tactic.Where
-- None of these imports are really necessary, except to create namespace mentioned below.
import Lean.Elab.Term
import Lean.Elab.Command
import Batteries.Data.UnionFind.Basic

-- Return to pristine state
set_option linter.missingDocs false
Expand Down Expand Up @@ -68,6 +71,6 @@ open Array renaming map -> listMap
info: open Lean Lean.Meta
open Lean.Elab hiding TermElabM
open Lean.Elab.Command Batteries
open listMap → Array.map
open Array renaming map → listMap
-/
#guard_msgs in #where

0 comments on commit b07115b

Please sign in to comment.