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 48cda55

Browse files
chore: bump to v4.19.0-rc3 (#413)
* chore: bump to `v4.19.0-rc3` * remove `import Mathlib` * set_option maxSynthPendingDepth 2 fixes * placate linter --------- Co-authored-by: Kevin Buzzard <[email protected]>
1 parent 2fe04f8 commit 48cda55

File tree

6 files changed

+31
-21
lines changed

6 files changed

+31
-21
lines changed

FLT/AutomorphicRepresentation/Example.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -520,8 +520,8 @@ lemma leftInvOn_toQuaternion_fromQuaternion :
520520
simp only [toQuaternion, fromQuaternion]
521521
obtain ⟨a, b, c, d, rfl|rfl⟩ := hq <;>
522522
ext <;>
523-
simp only [h₀, add_sub_add_right_eq_sub, Int.floor_sub_int, Int.floor_intCast, Int.cast_sub,
524-
Int.cast_add, Int.cast_one, Int.floor_add_one, Int.floor_add_int] <;>
523+
simp only [h₀, add_sub_add_right_eq_sub, Int.floor_sub_intCast, Int.floor_intCast, Int.cast_sub,
524+
Int.cast_add, Int.cast_one, Int.floor_add_one, Int.floor_sub_intCast] <;>
525525
field_simp <;>
526526
norm_cast <;>
527527
ring

FLT/DedekindDomain/FiniteAdeleRing/BaseChange.lean

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -378,10 +378,12 @@ noncomputable def adicCompletionComapSemialgHom' (v : HeightOneSpectrum A) :
378378
v.adicCompletion K →ₛₐ[algebraMap K L] ∀ w : v.Extension B, w.1.adicCompletion L :=
379379
Pi.semialgHom _ _ fun i ↦ adicCompletionComapSemialgHom A K L B v i.1 i.2
380380

381+
set_option maxSynthPendingDepth 2 in
381382
noncomputable instance comap_pi_algebra (v : HeightOneSpectrum A) :
382383
Algebra (v.adicCompletion K) (Π (w : v.Extension B), w.1.adicCompletion L) :=
383384
(adicCompletionComapSemialgHom' A K L B v).toAlgebra
384385

386+
set_option maxSynthPendingDepth 2 in
385387
omit [IsIntegralClosure B A L] [Algebra.IsSeparable K L] [Module.Finite A B] in
386388
lemma prodAdicCompletionComap_isModuleTopology (v : HeightOneSpectrum A) :
387389
-- TODO: the `let _` in the statement below should not be required as it is an instance
@@ -432,6 +434,7 @@ variable (v : HeightOneSpectrum A) in
432434
instance : IsModuleTopology (adicCompletion K v) (L ⊗[K] adicCompletion K v) :=
433435
⟨rfl⟩
434436

437+
set_option maxSynthPendingDepth 2 in
435438
attribute [local instance] Algebra.TensorProduct.rightAlgebra in
436439
/-- `adicCompletionComapAlgEquiv` as a `K_v`-algebra equivalence -/
437440
noncomputable def adicCompletionComapRightAlgEquiv (v : HeightOneSpectrum A) :
@@ -444,6 +447,7 @@ noncomputable def adicCompletionComapRightAlgEquiv (v : HeightOneSpectrum A) :
444447
simp [hmap, adicCompletionComapAlgEquiv,
445448
tensorAdicCompletionComapAlgHom, SemialgHom.algebraMap_apply]
446449

450+
set_option maxSynthPendingDepth 2 in
447451
noncomputable def adicCompletionComapContinuousAlgEquiv (v : HeightOneSpectrum A) :
448452
L ⊗[K] v.adicCompletion K ≃A[L] ∀ w : v.Extension B, w.1.adicCompletion L :=
449453
let _ := comap_pi_algebra A K L B v |>.toModule
@@ -542,6 +546,7 @@ open scoped TensorProduct -- ⊗ notation for tensor product
542546

543547
-- Note that this is only true because L/K is finite; in general tensor product doesn't
544548
-- commute with infinite products, but it does here.
549+
set_option maxSynthPendingDepth 2 in
545550
noncomputable def ProdAdicCompletions.baseChangeEquiv :
546551
L ⊗[K] ProdAdicCompletions A K ≃ₐ[L] ProdAdicCompletions B L :=
547552
AlgEquiv.ofBijective

FLT/Mathlib/Algebra/Order/AbsoluteValue/Basic.lean

Lines changed: 15 additions & 11 deletions
Original file line numberDiff line numberDiff line change
@@ -1,19 +1,20 @@
11
import Mathlib.Algebra.Order.AbsoluteValue.Basic
2-
import Mathlib.Tactic
2+
import Mathlib.Tactic.Linarith
33

44
namespace AbsoluteValue
55

6-
variable {F S : Type*} [Field F] [LinearOrderedField S] {v w : AbsoluteValue F S}
6+
variable {F S : Type*} [Field F] [Field S] [LinearOrder S]
7+
{v w : AbsoluteValue F S}
78

8-
theorem inv_pos {x : F} (h : 0 < v x) : 0 < v x⁻¹ := by
9+
theorem inv_pos [IsStrictOrderedRing S] {x : F} (h : 0 < v x) : 0 < v x⁻¹ := by
910
rwa [IsAbsoluteValue.abv_inv v, _root_.inv_pos]
1011

11-
theorem ne_zero_of_lt_one {F S : Type*} [Field F] [LinearOrderedField S]
12+
theorem ne_zero_of_lt_one {F S : Type*} [Field F] [Field S] [LinearOrder S] [IsStrictOrderedRing S]
1213
{v : AbsoluteValue F S} {x : F} (hv : 1 < v x) : x ≠ 0 :=
1314
fun hx => by linarith [map_zero v ▸ hx ▸ hv]
1415

15-
theorem isNontrivial_iff_exists_abv_gt_one {F S : Type*} [Field F] [LinearOrderedField S]
16-
{v : AbsoluteValue F S} :
16+
theorem isNontrivial_iff_exists_abv_gt_one {F S : Type*} [Field F] [Field S] [LinearOrder S]
17+
[IsStrictOrderedRing S] {v : AbsoluteValue F S} :
1718
v.IsNontrivial ↔ ∃ x, 1 < v x := by
1819
refine ⟨fun h => h.exists_abv_gt_one, fun ⟨x, hx⟩ => ?_⟩
1920
refine ⟨x⁻¹, ?_, ?_⟩
@@ -23,10 +24,12 @@ theorem isNontrivial_iff_exists_abv_gt_one {F S : Type*} [Field F] [LinearOrdere
2324
theorem nonpos_iff (x : F) : v x ≤ 0 ↔ v x = 0 := by
2425
simp only [le_antisymm_iff, v.nonneg _, and_true]
2526

27+
variable [IsStrictOrderedRing S]
2628
theorem inv_lt_one_iff {x : F} : v x⁻¹ < 1 ↔ x = 01 < v x := by
2729
simp only [map_inv₀, inv_lt_one_iff₀, nonpos_iff, map_eq_zero]
2830

29-
theorem mul_one_div_lt_iff {y : F} (x : F) (h : 0 < v y) : v (x * (1 / y)) < 1 ↔ v x < v y := by
31+
theorem mul_one_div_lt_iff {y : F} (x : F) (h : 0 < v y) :
32+
v (x * (1 / y)) < 1 ↔ v x < v y := by
3033
rw [map_mul, one_div, map_inv₀, mul_inv_lt_iff₀ h, one_mul]
3134

3235
theorem mul_one_div_pow_lt_iff {n : ℕ} {y : F} (x : F) (h : 0 < v y) :
@@ -51,17 +54,18 @@ theorem eq_one_iff_of_lt_one_iff (h : ∀ x, v x < 1 ↔ w x < 1) (x : F) : v x
5154

5255
variable (w)
5356

57+
omit [IsStrictOrderedRing S] in
5458
theorem pos_of_pos {a : F} (hv : 0 < v a) : 0 < w a := by
5559
rwa [AbsoluteValue.pos_iff] at hv ⊢
5660

57-
variable {R S : Type*} [OrderedRing S] [Semiring R] (v : AbsoluteValue R S) [IsDomain S]
58-
[Nontrivial R]
61+
variable {R S : Type*} [Ring S] [PartialOrder S] [Semiring R]
62+
(v : AbsoluteValue R S) [IsDomain S] [Nontrivial R]
5963

6064
theorem one_add_pow_le (a : R) (n : ℕ) : v (1 + a ^ n) ≤ 1 + v a ^ n :=
6165
le_trans (v.add_le _ _) (by rw [map_one, map_pow])
6266

63-
variable {R S : Type*} [OrderedCommRing S] [Ring R] (v : AbsoluteValue R S) [NoZeroDivisors S]
64-
[IsDomain S] [Nontrivial R]
67+
variable {R S : Type*} [CommRing S] [PartialOrder S] [IsOrderedRing S] [Ring R]
68+
(v : AbsoluteValue R S) [NoZeroDivisors S] [IsDomain S] [Nontrivial R]
6569

6670
theorem one_sub_pow_le (a : R) (n : ℕ) : 1 - v a ^ n ≤ v (1 + a ^ n) :=
6771
le_trans (by rw [map_one, map_pow]) (v.le_add 1 (a ^ n))

FLT/Mathlib/Topology/Algebra/Order/Field.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,8 @@ open scoped Topology
66

77
namespace AbsoluteValue
88

9-
variable {F S : Type*} [Field F] [LinearOrderedField S] {v w : AbsoluteValue F S}
9+
variable {F S : Type*} [Field F] [Field S] [LinearOrder S] [IsStrictOrderedRing S]
10+
{v w : AbsoluteValue F S}
1011

1112
/--
1213
If `v` is a nontrivial absolute value, and `w` is another absolute value such that `w x < 1`

lake-manifest.json

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "75d7aea6c81efeb68701164edaaa9116f06b91ba",
8+
"rev": "3d425859e73fcfbef85b9638c2a91708ef4a22d4",
99
"name": "checkdecls",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": null,
@@ -15,10 +15,10 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "",
18-
"rev": "6c7393e439bdc19b55044ff3fd636b969a9a1393",
18+
"rev": "ff99cdaecce8cab2fcc3d3828ab7f79717fbf77a",
1919
"name": "mathlib",
2020
"manifestFile": "lake-manifest.json",
21-
"inputRev": null,
21+
"inputRev": "v4.19.0-rc3",
2222
"inherited": false,
2323
"configFile": "lakefile.lean"},
2424
{"url": "https://github.com/leanprover-community/plausible",
@@ -35,7 +35,7 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "8d29bc2c3ebe1f863c2f02df816b4f3dd1b65226",
38+
"rev": "25078369972d295301f5a1e53c3e5850cf6d9d4c",
3939
"name": "LeanSearchClient",
4040
"manifestFile": "lake-manifest.json",
4141
"inputRev": "main",
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "57185dfad68d78356f9462af984882d6f262aa5d",
68+
"rev": "323e9f0b9bd41161ba116fe3bff86fc464d454f2",
6969
"name": "aesop",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "master",
@@ -85,7 +85,7 @@
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover-community",
88-
"rev": "f1a7afdb343196b33bf9137b232eb69446065925",
88+
"rev": "f523fcb75db2b472cda7d94d6caa5d745b1a0c26",
8989
"name": "batteries",
9090
"manifestFile": "lake-manifest.json",
9191
"inputRev": "main",

lean-toolchain

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

0 commit comments

Comments
 (0)