Skip to content

Commit

Permalink
chore: replace Std with Batteries and recycle a doc-string (#859)
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani authored Jun 25, 2024
1 parent da2d1d4 commit 93343d4
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Batteries/Linter/UnnecessarySeqFocus.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@ import Lean.Elab.Command
import Lean.Linter.Util
import Batteries.Lean.AttributeExtra

namespace Std.Linter
namespace Batteries.Linter
open Lean Elab Command Linter

/--
Expand Down Expand Up @@ -147,7 +147,7 @@ partial def markUsedTactics : InfoTree → M ω Unit

end

/-- The main entry point to the unused tactic linter. -/
@[inherit_doc Batteries.Linter.linter.unnecessarySeqFocus]
def unnecessarySeqFocusLinter : Linter where run := withSetOptionIn fun stx => do
unless getLinterUnnecessarySeqFocus (← getOptions) && (← getInfoState).enabled do
return
Expand Down

0 comments on commit 93343d4

Please sign in to comment.