Skip to content

Commit

Permalink
Two more
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Oct 31, 2024
1 parent 737eda7 commit 69bd919
Show file tree
Hide file tree
Showing 2 changed files with 6 additions and 1 deletion.
4 changes: 3 additions & 1 deletion Mathlib/Tactic/DeclarationNames.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,9 @@ Authors: Damiano Testa, Moritz Firsching

import Lean.DeclarationRange
import Lean.ResolveName
-- transitively imported in Mathlib.Init
-- Import this linter explicitly to ensure that
-- this file has a valid copyright header and module docstring.
import Mathlib.Tactic.Linter.Header

/-!
This file contains functions that are used by multiple linters.
Expand Down
3 changes: 3 additions & 0 deletions Mathlib/Tactic/Finiteness/Attr.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Floris van Doorn
-/
import Aesop
-- Import this linter explicitly to ensure that
-- this file has a valid copyright header and module docstring.
import Mathlib.Tactic.Linter.Header

/-! # Finiteness tactic attribute -/

Expand Down

0 comments on commit 69bd919

Please sign in to comment.