WARNING: THIS SITE IS A MIRROR OF GITHUB.COM / IT CANNOT LOGIN OR REGISTER ACCOUNTS / THE CONTENTS ARE PROVIDED AS-IS / THIS SITE ASSUMES NO RESPONSIBILITY FOR ANY DISPLAYED CONTENT OR LINKS / IF YOU FOUND SOMETHING MAY NOT GOOD FOR EVERYONE, CONTACT ADMIN AT ilovescratch@foxmail.com
Skip to content

Commit 3258daa

Browse files
authored
chore: bump mathlib to v4.23.0-rc2 (#699)
1 parent f298392 commit 3258daa

File tree

7 files changed

+18
-61
lines changed

7 files changed

+18
-61
lines changed

FLT.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -74,7 +74,6 @@ import FLT.Mathlib.MeasureTheory.Measure.OpenPos
7474
import FLT.Mathlib.MeasureTheory.Measure.Regular
7575
import FLT.Mathlib.MeasureTheory.Measure.Typeclasses.Finite
7676
import FLT.Mathlib.NumberTheory.NumberField.Completion
77-
import FLT.Mathlib.NumberTheory.NumberField.Embeddings
7877
import FLT.Mathlib.NumberTheory.Padics.PadicIntegers
7978
import FLT.Mathlib.NumberTheory.RamificationInertia.Basic
8079
import FLT.Mathlib.RepresentationTheory.Basic

FLT/AutomorphicRepresentation/Example.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -857,7 +857,7 @@ instance : Zero 𝓞 := ⟨zero⟩
857857
@[simp] lemma zero_im_oi : im_oi (0 : 𝓞) = 0 := rfl
858858

859859
lemma toQuaternion_zero : toQuaternion 0 = 0 := by
860-
ext <;> (simp [toQuaternion]; aesop)
860+
ext <;> (simp [toQuaternion])
861861

862862
@[simp]
863863
lemma toQuaternion_eq_zero_iff {z} : toQuaternion z = 0 ↔ z = 0 :=
@@ -879,7 +879,7 @@ instance : One 𝓞 := ⟨one⟩
879879
@[simp] lemma one_im_oi : im_oi (1 : 𝓞) = 0 := rfl
880880

881881
lemma toQuaternion_one : toQuaternion 1 = 1 := by
882-
ext <;> (simp [toQuaternion]; aesop)
882+
ext <;> (simp [toQuaternion])
883883

884884
/-! ## Neg (-) -/
885885

FLT/Mathlib/NumberTheory/NumberField/Embeddings.lean

Lines changed: 0 additions & 24 deletions
This file was deleted.

FLT/Mathlib/Topology/Algebra/Module/ModuleTopology.lean

Lines changed: 0 additions & 17 deletions
Original file line numberDiff line numberDiff line change
@@ -337,23 +337,6 @@ theorem of_inverse (f : N →ₗ[R] M) (g : M → N) (hc : Continuous g) (hi : F
337337
apply of_isQuotientMap N f
338338
exact Topology.IsQuotientMap.of_inverse hc (continuous_of_linearMap f) hi
339339

340-
omit [ContinuousAdd M] [ContinuousSMul R M] in
341-
/-- A linear surjection between modules with the module topology is an open quotient map. -/
342-
theorem isOpenQuotientMap_of_surjective [IsModuleTopology R M] {φ : M →ₗ[R] N}
343-
(hφ : Function.Surjective φ) : IsOpenQuotientMap φ :=
344-
have := toContinuousAdd R M
345-
AddMonoidHom.isOpenQuotientMap_of_isQuotientMap <| isQuotientMap_of_surjective hφ
346-
347-
/-- A linear surjection to a module with the module topology is open. -/
348-
theorem isOpenMap_of_surjective {φ : M →ₗ[R] N} (hφ : Function.Surjective φ) :
349-
IsOpenMap φ := by
350-
have hOpenMap :=
351-
letI : TopologicalSpace M := moduleTopology R M
352-
have : IsModuleTopology R M := isModuleTopology R M
353-
isOpenQuotientMap_of_surjective N hφ |>.isOpenMap
354-
intro U hU
355-
exact hOpenMap U <| moduleTopology_le R M U hU
356-
357340
end quotientMap
358341

359342
/-

FLT/NumberField/InfinitePlace/Dimension.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,6 @@ Authors: Salvatore Mercuri
66
import Mathlib.NumberTheory.NumberField.Completion
77
import FLT.NumberField.InfinitePlace.Extension
88
import FLT.Mathlib.Analysis.Normed.Ring.WithAbs
9-
import FLT.Mathlib.NumberTheory.NumberField.Embeddings
109

1110
/-!
1211
# Dimensions of completions at infinite places

lake-manifest.json

Lines changed: 15 additions & 15 deletions
Original file line numberDiff line numberDiff line change
@@ -15,20 +15,20 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "",
18-
"rev": "79e94a093aff4a60fb1b1f92d9681e407124c2ca",
18+
"rev": "9e0bebc63f8bcc1df0884cafebaab2673c6d57b0",
1919
"name": "mathlib",
2020
"manifestFile": "lake-manifest.json",
21-
"inputRev": "v4.22.0",
21+
"inputRev": null,
2222
"inherited": false,
2323
"configFile": "lakefile.lean"},
2424
{"url": "https://github.com/leanprover-community/plausible",
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "b100ad4c5d74a464f497aaa8e7c74d86bf39a56f",
28+
"rev": "240eddc1bb31420fbbc57fe5cc579435c2522493",
2929
"name": "plausible",
3030
"manifestFile": "lake-manifest.json",
31-
"inputRev": "v4.22.0",
31+
"inputRev": "main",
3232
"inherited": true,
3333
"configFile": "lakefile.toml"},
3434
{"url": "https://github.com/leanprover-community/LeanSearchClient",
@@ -45,57 +45,57 @@
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "eb164a46de87078f27640ee71e6c3841defc2484",
48+
"rev": "dba7fbc707774d1ba830fd44d7f92a717e9bf57f",
4949
"name": "importGraph",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "v4.22.0",
51+
"inputRev": "main",
5252
"inherited": true,
5353
"configFile": "lakefile.toml"},
5454
{"url": "https://github.com/leanprover-community/ProofWidgets4",
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "1253a071e6939b0faf5c09d2b30b0bfc79dae407",
58+
"rev": "6e47cc88cfbf1601ab364e9a4de5f33f13401ff8",
5959
"name": "proofwidgets",
6060
"manifestFile": "lake-manifest.json",
61-
"inputRev": "v0.0.68",
61+
"inputRev": "v0.0.71",
6262
"inherited": true,
6363
"configFile": "lakefile.lean"},
6464
{"url": "https://github.com/leanprover-community/aesop",
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "1256a18522728c2eeed6109b02dd2b8f207a2a3c",
68+
"rev": "3b779e9d1c73837a3764d516d81f942de391b6f0",
6969
"name": "aesop",
7070
"manifestFile": "lake-manifest.json",
71-
"inputRev": "v4.22.0",
71+
"inputRev": "master",
7272
"inherited": true,
7373
"configFile": "lakefile.toml"},
7474
{"url": "https://github.com/leanprover-community/quote4",
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "917bfa5064b812b7fbd7112d018ea0b4def25ab3",
78+
"rev": "f85ad59c9b60647ef736719c23edd4578f723806",
7979
"name": "Qq",
8080
"manifestFile": "lake-manifest.json",
81-
"inputRev": "v4.22.0",
81+
"inputRev": "master",
8282
"inherited": true,
8383
"configFile": "lakefile.toml"},
8484
{"url": "https://github.com/leanprover-community/batteries",
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover-community",
88-
"rev": "240676e9568c254a69be94801889d4b13f3b249f",
88+
"rev": "6e89c7370ca3a91b7d1f29ef7d727a9d027d7b0d",
8989
"name": "batteries",
9090
"manifestFile": "lake-manifest.json",
91-
"inputRev": "v4.22.0",
91+
"inputRev": "main",
9292
"inherited": true,
9393
"configFile": "lakefile.toml"},
9494
{"url": "https://github.com/leanprover/lean4-cli",
9595
"type": "git",
9696
"subDir": null,
9797
"scope": "leanprover",
98-
"rev": "c682c91d2d4dd59a7187e2ab977ac25bd1f87329",
98+
"rev": "cacb481a1eaa4d7d4530a27b606c60923da21caf",
9999
"name": "Cli",
100100
"manifestFile": "lake-manifest.json",
101101
"inputRev": "main",

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.22.0
1+
leanprover/lean4:v4.23.0-rc2

0 commit comments

Comments
 (0)