Skip to content

Commit

Permalink
move: new Mathlib.Tactic.Linter dir (#11807)
Browse files Browse the repository at this point in the history
Create a new `Mathlib/Tactic/Linter` dir and move there the linters.  Currently the new dir contains only one file, but there are more linters in PRs.
  • Loading branch information
adomani committed May 22, 2024
1 parent b072923 commit f485750
Show file tree
Hide file tree
Showing 6 changed files with 15 additions and 4 deletions.
2 changes: 1 addition & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3765,8 +3765,8 @@ import Mathlib.Tactic.Linarith.SimplexAlgorithm.PositiveVector
import Mathlib.Tactic.Linarith.SimplexAlgorithm.SimplexAlgorithm
import Mathlib.Tactic.Linarith.Verification
import Mathlib.Tactic.LinearCombination
import Mathlib.Tactic.Lint
import Mathlib.Tactic.Linter
import Mathlib.Tactic.Linter.Lint
import Mathlib.Tactic.Measurability
import Mathlib.Tactic.Measurability.Init
import Mathlib.Tactic.MkIffOfInductiveProp
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -111,8 +111,8 @@ import Mathlib.Tactic.Linarith.SimplexAlgorithm.PositiveVector
import Mathlib.Tactic.Linarith.SimplexAlgorithm.SimplexAlgorithm
import Mathlib.Tactic.Linarith.Verification
import Mathlib.Tactic.LinearCombination
import Mathlib.Tactic.Lint
import Mathlib.Tactic.Linter
import Mathlib.Tactic.Linter.Lint
import Mathlib.Tactic.Measurability
import Mathlib.Tactic.Measurability.Init
import Mathlib.Tactic.MkIffOfInductiveProp
Expand Down
11 changes: 11 additions & 0 deletions Mathlib/Tactic/Common.lean
Original file line number Diff line number Diff line change
Expand Up @@ -11,6 +11,14 @@ import Qq
-- Tools for analysing imports, like `#find_home`, `#minimize_imports`, ...
import ImportGraph.Imports

-- Currently we don't need to import all of ProofWidgets,
-- but without this, if you don't run `lake build ProofWidgets` then `make test` will fail.
-- Hopefully `lake` will be able to handle tests later.
import ProofWidgets

-- Import Mathlib-specific linters.
import Mathlib.Tactic.Linter.Lint

-- Now import all tactics defined in Mathlib that do not require theory files.
import Mathlib.Mathport.Rename
import Mathlib.Tactic.ApplyCongr
Expand Down Expand Up @@ -114,6 +122,9 @@ thereby making tactics widely available without needing specific imports.
We include some commented out imports here, with an explanation of their theory requirements,
to save some time for anyone wondering why they are not here.
We also import theory-free linters, commands, and utilities which are useful to have low in the
import hierarchy.
-/

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Tactic/Linter.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,4 +7,4 @@ This file is ignored by `Shake`:
* it is in `ignoreImport`, meaning that where it is imported, it is considered necessary.
-/

import Mathlib.Tactic.Lint
import Mathlib.Tactic.Linter.Lint
File renamed without changes.
2 changes: 1 addition & 1 deletion test/Lint.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import Mathlib.Tactic.Lint
import Mathlib.Tactic.Linter.Lint
import Mathlib.Tactic.ToAdditive

-- Adaptation note: test disabled.
Expand Down

0 comments on commit f485750

Please sign in to comment.