Skip to content

Commit

Permalink
also import Batteries.Tactic.Lint
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Aug 22, 2024
1 parent d747f07 commit b187647
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion scripts/runLinter.lean
Original file line number Diff line number Diff line change
Expand Up @@ -52,7 +52,7 @@ unsafe def main (args : List String) : IO Unit := do
readJsonFile NoLints nolintsFile
else
pure #[]
withImportModules #[{module}] {} (trustLevel := 1024) fun env =>
withImportModules #[{module}, { module := `Batteries.Tactic.Lint }] {} (trustLevel := 1024) fun env =>
let ctx := { fileName := "", fileMap := default }
let state := { env }
Prod.fst <$> (CoreM.toIO · ctx state) do
Expand Down

0 comments on commit b187647

Please sign in to comment.