Skip to content

Commit e75f135

Browse files
bump
1 parent c03f0c9 commit e75f135

File tree

7 files changed

+22
-22
lines changed

7 files changed

+22
-22
lines changed

FltRegular/NumberTheory/Finrank.lean

+2-3
Original file line numberDiff line numberDiff line change
@@ -181,9 +181,8 @@ lemma FiniteDimensional.exists_of_finrank_lt [IsDomain R] [IsPrincipalIdealRing
181181
∃ m : M, ∀ r : R, r ≠ 0 → r • m ∉ N := by
182182
obtain ⟨s, hs, hs'⟩ :=
183183
FiniteDimensional.exists_finset_card_eq_finrank_and_linearIndependent R (M ⧸ N)
184-
obtain ⟨v, hv⟩ : s.Nonempty
185-
· rwa [Finset.nonempty_iff_ne_empty, ne_eq, ← Finset.card_eq_zero, hs,
186-
FiniteDimensional.finrank_quotient, tsub_eq_zero_iff_le, not_le]
184+
obtain ⟨v, hv⟩ : s.Nonempty := by rwa [Finset.nonempty_iff_ne_empty, ne_eq, ← Finset.card_eq_zero,
185+
hs, FiniteDimensional.finrank_quotient, tsub_eq_zero_iff_le, not_le]
187186
obtain ⟨v, rfl⟩ := N.mkQ_surjective v
188187
use v
189188
intro r hr

FltRegular/NumberTheory/Hilbert92.lean

+5-5
Original file line numberDiff line numberDiff line change
@@ -747,7 +747,6 @@ lemma Hilbert92ish_aux2 (E : (𝓞 K)ˣ) (ζ : k) (hE : algebraMap k K ζ = E /
747747
· exact even_iff_two_dvd.1 (hp.even_sub_one hpodd)
748748
· simp
749749

750-
751750
attribute [-instance] Fintype.decidableForallFintype
752751
lemma unit_to_U_pow (x) (n : ℕ) : mkG (x ^ n) = n • (mkG x) := by
753752
induction n with
@@ -838,8 +837,8 @@ lemma Hilbert92ish (hpodd : (p : ℕ) ≠ 2) :
838837
· refine ha'' ?_ this
839838
ext
840839
simpa using hζ
841-
obtain ⟨ε', hε'⟩ : ∃ ε' : (𝓞 k)ˣ, ε' ^ (p : ℕ) = NE
842-
· rw [← (Nat.prime_iff_prime_int.mp hp).coprime_iff_not_dvd] at ha'
840+
obtain ⟨ε', hε'⟩ : ∃ ε' : (𝓞 k)ˣ, ε' ^ (p : ℕ) = NE := by
841+
rw [← (Nat.prime_iff_prime_int.mp hp).coprime_iff_not_dvd] at ha'
843842
obtain ⟨α, β, hαβ⟩ := ha'
844843
choose ι' hι' using hε'
845844
rw [Fin.sum_univ_castSucc] at ha
@@ -852,8 +851,9 @@ lemma Hilbert92ish (hpodd : (p : ℕ) ≠ 2) :
852851
exact ⟨_, ha.symm⟩
853852
have hζ'' := (hζ.pow (p ^ h.succ).pos (pow_succ _ _)).map_of_injective
854853
(algebraMap k K).injective
855-
obtain ⟨ε'', hε''⟩ : ∃ ε'' : (𝓞 k)ˣ, E = Units.map (algebraMap (𝓞 k) (𝓞 K)).toMonoidHom ε''
856-
· rw [← hε', map_pow, eq_comm, ← mul_inv_eq_one, ← inv_pow, ← mul_pow] at NE_p_pow
854+
obtain ⟨ε'', hε''⟩ :
855+
∃ ε'' : (𝓞 k)ˣ, E = Units.map (algebraMap (𝓞 k) (𝓞 K)).toMonoidHom ε'' := by
856+
rw [← hε', map_pow, eq_comm, ← mul_inv_eq_one, ← inv_pow, ← mul_pow] at NE_p_pow
857857
apply_fun ((↑) : (𝓞 K)ˣ → K) at NE_p_pow
858858
simp only [RingHom.toMonoidHom_eq_coe, Units.val_pow_eq_pow_val, Units.val_mul,
859859
Units.coe_map_inv, MonoidHom.coe_coe, SubmonoidClass.coe_pow, Submonoid.coe_mul,

FltRegular/NumberTheory/KummersLemma/Field.lean

+3-2
Original file line numberDiff line numberDiff line change
@@ -239,8 +239,9 @@ lemma separable_poly_aux {L : Type*} [Field L] [Algebra K L] (α : L)
239239
refine separable_prod' ?_ (fun _ _ => separable_X_sub_C)
240240
intros i hi j hj hij
241241
apply isCoprime_X_sub_C_of_isUnit_sub
242-
obtain ⟨v, hv⟩ : Associated (hζ.unit' - 1 : 𝓞 K) ((hζ.unit' : 𝓞 K) ^ j - (hζ.unit' : 𝓞 K) ^ i)
243-
· refine hζ.unit'_coe.associated_sub_one hpri.out ?_ ?_ ?_
242+
obtain ⟨v, hv⟩ :
243+
Associated (hζ.unit' - 1 : 𝓞 K) ((hζ.unit' : 𝓞 K) ^ j - (hζ.unit' : 𝓞 K) ^ i) := by
244+
refine hζ.unit'_coe.associated_sub_one hpri.out ?_ ?_ ?_
244245
· rw [mem_nthRootsFinset p.pos, ← pow_mul, mul_comm, pow_mul, hζ.unit'_coe.pow_eq_one, one_pow]
245246
· rw [mem_nthRootsFinset p.pos, ← pow_mul, mul_comm, pow_mul, hζ.unit'_coe.pow_eq_one, one_pow]
246247
· exact mt (hζ.unit'_coe.injOn_pow hj hi) hij.symm

FltRegular/NumberTheory/KummersLemma/KummersLemma.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -50,8 +50,8 @@ theorem eq_pow_prime_of_unit_of_congruent (u : (𝓞 K)ˣ)
5050
∃ v, u = v ^ (p : ℕ) := by
5151
haveI : Fact (Nat.Prime p) := hpri
5252
obtain ⟨ζ, hζ⟩ := IsCyclotomicExtension.exists_prim_root (S := {p}) ℚ (B := K) (n := p) rfl
53-
obtain ⟨x, hx⟩ : (p : 𝓞 K) ∣ (↑(u ^ (p - 1 : ℕ)) : 𝓞 K) - 1
54-
· obtain ⟨n, hn⟩ := hcong
53+
obtain ⟨x, hx⟩ : (p : 𝓞 K) ∣ (↑(u ^ (p - 1 : ℕ)) : 𝓞 K) - 1 := by
54+
obtain ⟨n, hn⟩ := hcong
5555
have hn' : (p : ℤ) ∣ n ^ (p - 1 : ℕ) - 1
5656
· refine Int.modEq_iff_dvd.mp (Int.ModEq.pow_card_sub_one_eq_one hpri.out (n := n) ?_).symm
5757
rw [isCoprime_comm, (Nat.prime_iff_prime_int.mp hpri.out).coprime_iff_not_dvd]

FltRegular/NumberTheory/QuotientTrace.lean

+6-6
Original file line numberDiff line numberDiff line change
@@ -169,8 +169,8 @@ lemma comap_map_eq_map_of_isLocalization_algebraMapSubmonoid :
169169
rw [IsScalarTower.algebraMap_eq R S Sₚ, ← Ideal.map_map, eq_comm]
170170
apply Ideal.le_comap_map.antisymm
171171
intro x hx
172-
obtain ⟨α, hα, hαx⟩ : ∃ α ∉ p, α • x ∈ pS
173-
· have ⟨⟨y, s⟩, hy⟩ := (IsLocalization.mem_map_algebraMap_iff
172+
obtain ⟨α, hα, hαx⟩ : ∃ α ∉ p, α • x ∈ pS := by
173+
have ⟨⟨y, s⟩, hy⟩ := (IsLocalization.mem_map_algebraMap_iff
174174
(Algebra.algebraMapSubmonoid S p.primeCompl) Sₚ).mp hx
175175
rw [← map_mul,
176176
IsLocalization.eq_iff_exists (Algebra.algebraMapSubmonoid S p.primeCompl)] at hy
@@ -179,8 +179,8 @@ lemma comap_map_eq_map_of_isLocalization_algebraMapSubmonoid :
179179
refine ⟨α, hα, ?_⟩
180180
rw [Algebra.smul_def, e, Submonoid.coe_mul, mul_assoc, mul_comm _ x, hc]
181181
exact Ideal.mul_mem_left _ _ y.prop
182-
obtain ⟨β, γ, hγ, hβ⟩ : ∃ β γ, γ ∈ p ∧ β * α = 1 + γ
183-
· obtain ⟨β, hβ⟩ := Ideal.Quotient.mk_surjective (I := p) (Ideal.Quotient.mk p α)⁻¹
182+
obtain ⟨β, γ, hγ, hβ⟩ : ∃ β γ, γ ∈ p ∧ β * α = 1 + γ := by
183+
obtain ⟨β, hβ⟩ := Ideal.Quotient.mk_surjective (I := p) (Ideal.Quotient.mk p α)⁻¹
184184
refine ⟨β, β * α - 1, ?_, ?_⟩
185185
· rw [← Ideal.Quotient.eq_zero_iff_mem, map_sub, map_one,
186186
map_mul, hβ, inv_mul_cancel, sub_self]
@@ -210,8 +210,8 @@ def quotMapEquivQuotMapMaximalIdealOfIsLocalization : S ⧸ pS ≃+* Sₚ ⧸ pS
210210
obtain ⟨x, s, rfl⟩ := IsLocalization.mk'_surjective
211211
(Algebra.algebraMapSubmonoid S p.primeCompl) x
212212
obtain ⟨α, hα : α ∉ p, e⟩ := s.prop
213-
obtain ⟨β, γ, hγ, hβ⟩ : ∃ β γ, γ ∈ p ∧ α * β = 1 + γ
214-
· obtain ⟨β, hβ⟩ := Ideal.Quotient.mk_surjective (I := p) (Ideal.Quotient.mk p α)⁻¹
213+
obtain ⟨β, γ, hγ, hβ⟩ : ∃ β γ, γ ∈ p ∧ α * β = 1 + γ := by
214+
obtain ⟨β, hβ⟩ := Ideal.Quotient.mk_surjective (I := p) (Ideal.Quotient.mk p α)⁻¹
215215
refine ⟨β, α * β - 1, ?_, ?_⟩
216216
· rw [← Ideal.Quotient.eq_zero_iff_mem, map_sub, map_one,
217217
map_mul, hβ, mul_inv_cancel, sub_self]

lake-manifest.json

+3-3
Original file line numberDiff line numberDiff line change
@@ -31,10 +31,10 @@
3131
{"url": "https://github.com/leanprover-community/ProofWidgets4",
3232
"type": "git",
3333
"subDir": null,
34-
"rev": "e6b6247c61280c77ade6bbf0bc3c66a44fe2e0c5",
34+
"rev": "fc8f85bab627d5196b2342bd2f08c0ace749ec89",
3535
"name": "proofwidgets",
3636
"manifestFile": "lake-manifest.json",
37-
"inputRev": "v0.0.36",
37+
"inputRev": "v0.0.37",
3838
"inherited": true,
3939
"configFile": "lakefile.lean"},
4040
{"url": "https://github.com/leanprover/lean4-cli",
@@ -58,7 +58,7 @@
5858
{"url": "https://github.com/leanprover-community/mathlib4.git",
5959
"type": "git",
6060
"subDir": null,
61-
"rev": "0eb87504b21018e2a4200d4417d57fc06c99c960",
61+
"rev": "397d87803ee60c11623fdd680199366acaaedaef",
6262
"name": "mathlib",
6363
"manifestFile": "lake-manifest.json",
6464
"inputRev": null,

lean-toolchain

+1-1
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.9.0-rc2
1+
leanprover/lean4:v4.9.0-rc3

0 commit comments

Comments
 (0)