Skip to content

Commit

Permalink
shake update
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Oct 19, 2024
1 parent 4f6fe87 commit 407a445
Show file tree
Hide file tree
Showing 3 changed files with 4 additions and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/Algebra/BigOperators/Group/List.lean
Original file line number Diff line number Diff line change
Expand Up @@ -13,6 +13,7 @@ import Mathlib.Data.List.Range
import Mathlib.Data.List.Rotate
import Mathlib.Data.List.Pairwise
import Mathlib.Data.List.Join
import Mathlib.Data.List.ProdSigma

/-!
# Sums and products from lists
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Order/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Leonardo de Moura
-/
import Batteries.Classes.Order
import Batteries.Tactic.Trans
import Mathlib.Data.Ordering.Basic
import Mathlib.Tactic.Lemma
import Mathlib.Tactic.SplitIfs
Expand Down
2 changes: 2 additions & 0 deletions scripts/noshake.json
Original file line number Diff line number Diff line change
Expand Up @@ -325,6 +325,7 @@
"Mathlib.Order.RelClasses": ["Batteries.WF"],
"Mathlib.Order.Filter.ListTraverse":
["Mathlib.Control.Traversable.Instances"],
"Mathlib.Order.Defs": ["Batteries.Tactic.Trans"],
"Mathlib.NumberTheory.Harmonic.Defs":
["Mathlib.Algebra.Order.BigOperators.Ring.Finset",
"Mathlib.Algebra.Order.Field.Basic"],
Expand Down Expand Up @@ -427,6 +428,7 @@
["Mathlib.CategoryTheory.ConcreteCategory.ReflectsIso"],
"Mathlib.Algebra.Category.MonCat.Basic":
["Mathlib.Algebra.Ring.Action.Group"],
"Mathlib.Algebra.BigOperators.Group.List": ["Mathlib.Data.List.ProdSigma"],
"Mathlib.Algebra.Algebra.Subalgebra.Order":
["Mathlib.Algebra.Module.Submodule.Order"],
"Batteries.Tactic.OpenPrivate": ["Lean.Parser.Module"],
Expand Down

0 comments on commit 407a445

Please sign in to comment.