Skip to content

Commit

Permalink
modify test
Browse files Browse the repository at this point in the history
  • Loading branch information
joneugster committed Sep 26, 2024
1 parent 965ce5f commit ff1f648
Showing 1 changed file with 3 additions and 2 deletions.
5 changes: 3 additions & 2 deletions scripts/autolabel.lean
Original file line number Diff line number Diff line change
Expand Up @@ -89,7 +89,8 @@ def mathlibLabels : Array Label := #[
"Mathlib" / "RingTheory",
"Mathlib" / "GroupTheory",
"Mathlib" / "RepresentationTheory",
"Mathlib" / "LinearAlgebra"] },
"Mathlib" / "LinearAlgebra"],
exclusions := #["Mathlib" / "Algebra" / "NonExistent"] },
{ label := "t-algebraic-geometry",
dirs := #[
"Mathlib" / "AlgebraicGeometry",
Expand Down Expand Up @@ -123,7 +124,7 @@ def mathlibLabels : Array Label := #[
"Mathlib" / "Mathport",
"Mathlib" / "Tactic",
"Mathlib" / "Util"],
exclusions := #["Mathlib" / "Tactic" / "Linters"] },
exclusions := #["Mathlib" / "Tactic" / "Linter"] },
{ label := "t-number-theory" },
{ label := "t-order" },
{ label := "t-set-theory" },
Expand Down

0 comments on commit ff1f648

Please sign in to comment.