@@ -753,6 +753,7 @@ import Mathlib.Algebra.Order.Antidiag.Nat
753753import Mathlib.Algebra.Order.Antidiag.Pi
754754import Mathlib.Algebra.Order.Antidiag.Prod
755755import Mathlib.Algebra.Order.Archimedean.Basic
756+ import Mathlib.Algebra.Order.Archimedean.Class
756757import Mathlib.Algebra.Order.Archimedean.Hom
757758import Mathlib.Algebra.Order.Archimedean.IndicatorCard
758759import Mathlib.Algebra.Order.Archimedean.Submonoid
@@ -827,6 +828,7 @@ import Mathlib.Algebra.Order.GroupWithZero.Action.Synonym
827828import Mathlib.Algebra.Order.GroupWithZero.Bounds
828829import Mathlib.Algebra.Order.GroupWithZero.Canonical
829830import Mathlib.Algebra.Order.GroupWithZero.Finset
831+ import Mathlib.Algebra.Order.GroupWithZero.Lex
830832import Mathlib.Algebra.Order.GroupWithZero.Submonoid
831833import Mathlib.Algebra.Order.GroupWithZero.Synonym
832834import Mathlib.Algebra.Order.GroupWithZero.Unbundled
@@ -860,6 +862,7 @@ import Mathlib.Algebra.Order.Monoid.Basic
860862import Mathlib.Algebra.Order.Monoid.Canonical.Basic
861863import Mathlib.Algebra.Order.Monoid.Canonical.Defs
862864import Mathlib.Algebra.Order.Monoid.Defs
865+ import Mathlib.Algebra.Order.Monoid.Lex
863866import Mathlib.Algebra.Order.Monoid.NatCast
864867import Mathlib.Algebra.Order.Monoid.OrderDual
865868import Mathlib.Algebra.Order.Monoid.Prod
@@ -3802,6 +3805,7 @@ import Mathlib.GroupTheory.QuotientGroup.Basic
38023805import Mathlib.GroupTheory.QuotientGroup.Defs
38033806import Mathlib.GroupTheory.QuotientGroup.Finite
38043807import Mathlib.GroupTheory.Rank
3808+ import Mathlib.GroupTheory.RegularWreathProduct
38053809import Mathlib.GroupTheory.Schreier
38063810import Mathlib.GroupTheory.SchurZassenhaus
38073811import Mathlib.GroupTheory.SemidirectProduct
@@ -4885,6 +4889,7 @@ import Mathlib.Order.Preorder.Chain
48854889import Mathlib.Order.Preorder.Finite
48864890import Mathlib.Order.PrimeIdeal
48874891import Mathlib.Order.PrimeSeparator
4892+ import Mathlib.Order.Prod.Lex.Hom
48884893import Mathlib.Order.PropInstances
48894894import Mathlib.Order.Radical
48904895import Mathlib.Order.Rel.GaloisConnection
@@ -5027,11 +5032,13 @@ import Mathlib.RepresentationTheory.Character
50275032import Mathlib.RepresentationTheory.Coinduced
50285033import Mathlib.RepresentationTheory.Coinvariants
50295034import Mathlib.RepresentationTheory.FDRep
5030- import Mathlib.RepresentationTheory.GroupCohomology.Basic
5031- import Mathlib.RepresentationTheory.GroupCohomology.Functoriality
5032- import Mathlib.RepresentationTheory.GroupCohomology.Hilbert90
5033- import Mathlib.RepresentationTheory.GroupCohomology.LowDegree
5034- import Mathlib.RepresentationTheory.GroupCohomology.Resolution
5035+ import Mathlib.RepresentationTheory.FiniteIndex
5036+ import Mathlib.RepresentationTheory.Homological.GroupCohomology.Basic
5037+ import Mathlib.RepresentationTheory.Homological.GroupCohomology.Functoriality
5038+ import Mathlib.RepresentationTheory.Homological.GroupCohomology.Hilbert90
5039+ import Mathlib.RepresentationTheory.Homological.GroupCohomology.LowDegree
5040+ import Mathlib.RepresentationTheory.Homological.GroupHomology.Basic
5041+ import Mathlib.RepresentationTheory.Homological.Resolution
50355042import Mathlib.RepresentationTheory.Induced
50365043import Mathlib.RepresentationTheory.Invariants
50375044import Mathlib.RepresentationTheory.Maschke
0 commit comments