Skip to content

Commit e0e4b37

Browse files
Merge master into nightly-testing
2 parents 72824e4 + 1825e17 commit e0e4b37

File tree

495 files changed

+1680
-1385
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

495 files changed

+1680
-1385
lines changed

Archive/Imo/Imo1998Q2.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -176,7 +176,7 @@ theorem judge_pairs_card_lower_bound {z : ℕ} (hJ : Fintype.card J = 2 * z + 1)
176176
rw [h]; apply Int.le_of_ofNat_le_ofNat; simp only [Int.natCast_add, Int.natCast_mul]
177177
apply norm_bound_of_odd_sum
178178
suffices x + y = 2 * z + 1 by simp [← Int.natCast_add, this]
179-
rw [Finset.filter_card_add_filter_neg_card_eq_card, ← hJ, Finset.card_univ]
179+
rw [Finset.card_filter_add_card_filter_not, ← hJ, Finset.card_univ]
180180

181181
open scoped Classical in
182182
theorem distinct_judge_pairs_card_lower_bound {z : ℕ} (hJ : Fintype.card J = 2 * z + 1) (c : C) :

Mathlib.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -652,7 +652,6 @@ public import Mathlib.Algebra.Lie.Abelian
652652
public import Mathlib.Algebra.Lie.BaseChange
653653
public import Mathlib.Algebra.Lie.Basic
654654
public import Mathlib.Algebra.Lie.CartanExists
655-
public import Mathlib.Algebra.Lie.CartanMatrix
656655
public import Mathlib.Algebra.Lie.CartanSubalgebra
657656
public import Mathlib.Algebra.Lie.Character
658657
public import Mathlib.Algebra.Lie.Classical
@@ -680,6 +679,7 @@ public import Mathlib.Algebra.Lie.Rank
680679
public import Mathlib.Algebra.Lie.Semisimple.Basic
681680
public import Mathlib.Algebra.Lie.Semisimple.Defs
682681
public import Mathlib.Algebra.Lie.Semisimple.Lemmas
682+
public import Mathlib.Algebra.Lie.SerreConstruction
683683
public import Mathlib.Algebra.Lie.SkewAdjoint
684684
public import Mathlib.Algebra.Lie.Sl2
685685
public import Mathlib.Algebra.Lie.Solvable
@@ -3670,6 +3670,7 @@ public import Mathlib.Data.Matrix.Basic
36703670
public import Mathlib.Data.Matrix.Basis
36713671
public import Mathlib.Data.Matrix.Bilinear
36723672
public import Mathlib.Data.Matrix.Block
3673+
public import Mathlib.Data.Matrix.Cartan
36733674
public import Mathlib.Data.Matrix.ColumnRowPartitioned
36743675
public import Mathlib.Data.Matrix.Composition
36753676
public import Mathlib.Data.Matrix.DMatrix
@@ -6247,6 +6248,7 @@ public import Mathlib.RingTheory.Smooth.NoetherianDescent
62476248
public import Mathlib.RingTheory.Smooth.Pi
62486249
public import Mathlib.RingTheory.Smooth.StandardSmooth
62496250
public import Mathlib.RingTheory.Smooth.StandardSmoothCotangent
6251+
public import Mathlib.RingTheory.Smooth.StandardSmoothOfFree
62506252
public import Mathlib.RingTheory.Spectrum.Maximal.Basic
62516253
public import Mathlib.RingTheory.Spectrum.Maximal.Defs
62526254
public import Mathlib.RingTheory.Spectrum.Maximal.Localization

Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -149,7 +149,7 @@ theorem prod_filter_mul_prod_filter_not
149149
(s : Finset ι) (p : ι → Prop) [DecidablePred p] [∀ x, Decidable (¬p x)] (f : ι → M) :
150150
(∏ x ∈ s with p x, f x) * ∏ x ∈ s with ¬p x, f x = ∏ x ∈ s, f x := by
151151
have := Classical.decEq ι
152-
rw [← prod_union (disjoint_filter_filter_neg s s p), filter_union_filter_neg_eq]
152+
rw [← prod_union (disjoint_filter_filter_not s s p), filter_union_filter_not_eq]
153153

154154
@[to_additive]
155155
lemma prod_filter_not_mul_prod_filter (s : Finset ι) (p : ι → Prop) [DecidablePred p]

Mathlib/Algebra/Category/FGModuleCat/Colimits.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -57,7 +57,7 @@ def forget₂CreatesColimit (F : J ⥤ FGModuleCat k) :
5757
instance : CreatesColimitsOfShape J (forget₂ (FGModuleCat k) (ModuleCat.{v} k)) where
5858
CreatesColimit {F} := forget₂CreatesColimit F
5959

60-
instance (J : Type) [Category J] [FinCategory J] :
60+
instance (J : Type) [SmallCategory J] [FinCategory J] :
6161
HasColimitsOfShape J (FGModuleCat.{v} k) :=
6262
hasColimitsOfShape_of_hasColimitsOfShape_createsColimitsOfShape
6363
(forget₂ (FGModuleCat k) (ModuleCat.{v} k))

Mathlib/Algebra/Category/FGModuleCat/Limits.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -65,7 +65,7 @@ def forget₂CreatesLimit (F : J ⥤ FGModuleCat k) :
6565
instance : CreatesLimitsOfShape J (forget₂ (FGModuleCat k) (ModuleCat.{v} k)) where
6666
CreatesLimit {F} := forget₂CreatesLimit F
6767

68-
instance (J : Type) [Category J] [FinCategory J] :
68+
instance (J : Type) [SmallCategory J] [FinCategory J] :
6969
HasLimitsOfShape J (FGModuleCat.{v} k) :=
7070
hasLimitsOfShape_of_hasLimitsOfShape_createsLimitsOfShape
7171
(forget₂ (FGModuleCat k) (ModuleCat.{v} k))

Mathlib/Algebra/Category/Grp/AB.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -23,7 +23,7 @@ universe u
2323

2424
open CategoryTheory Limits
2525

26-
instance {J C : Type*} [Category J] [Category C] [HasColimitsOfShape J C] [Preadditive C] :
26+
instance {J C : Type*} [Category* J] [Category* C] [HasColimitsOfShape J C] [Preadditive C] :
2727
(colim (J := J) (C := C)).Additive where
2828

2929
variable {J : Type u} [SmallCategory J] [IsFiltered J]

Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -212,7 +212,7 @@ namespace CategoryTheory
212212

213213
universe v u
214214

215-
/-- `Free R C` is a type synonym for `C`, which, given `[CommRing R]` and `[Category C]`,
215+
/-- `Free R C` is a type synonym for `C`, which, given `[CommRing R]` and `[Category* C]`,
216216
we will equip with a category structure where the morphisms are formal `R`-linear combinations
217217
of the morphisms in `C`.
218218
-/

Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -855,15 +855,15 @@ instance {R : Type u₁} {S : Type u₂} [CommRing R] [CommRing S] (f : R →+*
855855
(extendRestrictScalarsAdj f).isRightAdjoint
856856

857857
noncomputable instance preservesLimit_restrictScalars
858-
{R : Type*} {S : Type*} [Ring R] [Ring S] (f : R →+* S) {J : Type*} [Category J]
858+
{R : Type*} {S : Type*} [Ring R] [Ring S] (f : R →+* S) {J : Type*} [Category* J]
859859
(F : J ⥤ ModuleCat.{v} S) [Small.{v} (F ⋙ forget _).sections] :
860860
PreservesLimit F (restrictScalars f) :=
861861
fun {c} hc => ⟨by
862862
have hc' := isLimitOfPreserves (forget₂ _ AddCommGrpCat) hc
863863
exact isLimitOfReflects (forget₂ _ AddCommGrpCat) hc'⟩⟩
864864

865865
instance preservesColimit_restrictScalars {R S : Type*} [Ring R] [Ring S]
866-
(f : R →+* S) {J : Type*} [Category J] (F : J ⥤ ModuleCat.{v} S)
866+
(f : R →+* S) {J : Type*} [Category* J] (F : J ⥤ ModuleCat.{v} S)
867867
[HasColimit (F ⋙ forget₂ _ AddCommGrpCat)] :
868868
PreservesColimit F (ModuleCat.restrictScalars.{v} f) := by
869869
have : HasColimit ((F ⋙ restrictScalars f) ⋙ forget₂ (ModuleCat R) AddCommGrpCat) :=

Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -29,7 +29,7 @@ open CategoryTheory MonoidalCategory Category
2929

3030
universe v u v₁ u₁
3131

32-
variable {C : Type*} [Category C] {R : Cᵒᵖ ⥤ CommRingCat.{u}}
32+
variable {C : Type*} [Category* C] {R : Cᵒᵖ ⥤ CommRingCat.{u}}
3333

3434
instance (X : Cᵒᵖ) : CommRing ((R ⋙ forget₂ _ RingCat).obj X) :=
3535
inferInstanceAs (CommRing (R.obj X))

Mathlib/Algebra/Category/ModuleCat/Topology/Basic.lean

Lines changed: 10 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -214,7 +214,7 @@ def toCoinduced (i) : X i ⟶ coinduced f :=
214214

215215
/-- The cocone of topological modules associated to a cocone over the underlying modules, where
216216
the cocone point is given the coinduced topology. This is colimiting when the given cocone is. -/
217-
def ofCocone {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
217+
def ofCocone {J : Type*} [Category* J] {F : J ⥤ TopModuleCat R}
218218
(c : Cocone (F ⋙ forget₂ _ (ModuleCat R))) : Cocone F where
219219
pt := coinduced c.ι.app
220220
ι :=
@@ -223,7 +223,7 @@ def ofCocone {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
223223

224224
/-- Given a colimit cocone over the underlying modules, equipping the cocone point with
225225
the coinduced topology gives a colimit cocone in `TopModuleCat R`. -/
226-
def isColimit {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
226+
def isColimit {J : Type*} [Category* J] {F : J ⥤ TopModuleCat R}
227227
{c : Cocone (F ⋙ forget₂ _ (ModuleCat R))} (hc : IsColimit c) :
228228
IsColimit (ofCocone c) where
229229
desc s := ofHom (X := (ofCocone c).pt) ⟨(hc.desc ((forget₂ _ _).mapCocone s)).hom, by
@@ -242,11 +242,11 @@ def isColimit {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
242242
ext y
243243
exact congr($(H j).hom y)
244244

245-
instance {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
245+
instance {J : Type*} [Category* J] {F : J ⥤ TopModuleCat R}
246246
[HasColimit (F ⋙ forget₂ _ (ModuleCat R))] : HasColimit F :=
247247
⟨_, isColimit (colimit.isColimit _)⟩
248248

249-
instance {J : Type*} [Category J] [HasColimitsOfShape J (ModuleCat.{v} R)] :
249+
instance {J : Type*} [Category* J] [HasColimitsOfShape J (ModuleCat.{v} R)] :
250250
HasColimitsOfShape J (TopModuleCat.{v} R) where
251251

252252
instance : HasColimits (TopModuleCat.{v} R) where
@@ -275,7 +275,7 @@ open Limits
275275

276276
/-- The cone of topological modules associated to a cone over the underlying modules, where
277277
the cone point is given the induced topology. This is limiting when the given cone is. -/
278-
def ofCone {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
278+
def ofCone {J : Type*} [Category* J] {F : J ⥤ TopModuleCat R}
279279
(c : Cone (F ⋙ forget₂ _ (ModuleCat R))) : Cone F where
280280
pt := induced c.π.app
281281
π :=
@@ -284,7 +284,7 @@ def ofCone {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
284284

285285
/-- Given a limit cone over the underlying modules, equipping the cone point with
286286
the induced topology gives a limit cone in `TopModuleCat R`. -/
287-
def isLimit {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
287+
def isLimit {J : Type*} [Category* J] {F : J ⥤ TopModuleCat R}
288288
{c : Cone (F ⋙ forget₂ _ (ModuleCat R))} (hc : IsLimit c) :
289289
IsLimit (ofCone c) where
290290
lift s := ofHom (Y := (ofCone c).pt) ⟨(hc.lift ((forget₂ _ _).mapCone s)).hom, by
@@ -302,18 +302,18 @@ def isLimit {J : Type*} [Category J] {F : J ⥤ TopModuleCat R}
302302
ext y
303303
exact congr($(H j).hom y)
304304

305-
instance hasLimit_of_hasLimit_forget₂ {J : Type*} [Category J] {F : J ⥤ TopModuleCat.{v} R}
305+
instance hasLimit_of_hasLimit_forget₂ {J : Type*} [Category* J] {F : J ⥤ TopModuleCat.{v} R}
306306
[HasLimit (F ⋙ forget₂ _ (ModuleCat.{v} R))] : HasLimit F :=
307307
⟨_, isLimit (limit.isLimit _)⟩
308308

309-
instance {J : Type*} [Category J] [HasLimitsOfShape J (ModuleCat.{v} R)] :
309+
instance {J : Type*} [Category* J] [HasLimitsOfShape J (ModuleCat.{v} R)] :
310310
HasLimitsOfShape J (TopModuleCat.{v} R) where
311311
has_limit _ := hasLimit_of_hasLimit_forget₂
312312

313313
instance : HasLimits (TopModuleCat.{v} R) where
314314
has_limits_of_shape _ _ := ⟨fun _ ↦ hasLimit_of_hasLimit_forget₂⟩
315315

316-
instance {J : Type*} [Category J] {F : J ⥤ TopModuleCat.{v} R}
316+
instance {J : Type*} [Category* J] {F : J ⥤ TopModuleCat.{v} R}
317317
[HasLimit (F ⋙ forget₂ _ (ModuleCat.{v} R))]
318318
[PreservesLimit (F ⋙ forget₂ _ (ModuleCat.{v} R)) (forget _)] :
319319
PreservesLimit F (forget₂ _ TopCat) :=
@@ -322,7 +322,7 @@ instance {J : Type*} [Category J] {F : J ⥤ TopModuleCat.{v} R}
322322
((forget _).mapCone (getLimitCone (F ⋙ forget₂ _ (ModuleCat.{v} R))).1:)
323323
(isLimitOfPreserves (forget (ModuleCat R)) (limit.isLimit _)))
324324

325-
instance {J : Type*} [Category J]
325+
instance {J : Type*} [Category* J]
326326
[HasLimitsOfShape J (ModuleCat.{v} R)]
327327
[PreservesLimitsOfShape J (forget (ModuleCat.{v} R))] :
328328
PreservesLimitsOfShape J (forget₂ (TopModuleCat.{v} R) TopCat) where

0 commit comments

Comments
 (0)