Skip to content

Commit 15cd260

Browse files
bump
1 parent 8ac9254 commit 15cd260

File tree

4 files changed

+13
-15
lines changed

4 files changed

+13
-15
lines changed

FltRegular/FltThree/Edwards.lean

Lines changed: 6 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -83,7 +83,6 @@ theorem step1a {a : ℤ√(-3)} (hcoprime : IsCoprime a.re a.im) (heven : Even a
8383
have := hcoprime.isUnit_of_dvd' hre him
8484
rw [isUnit_iff_dvd_one] at this
8585
norm_num at this
86-
contradiction
8786
#align step1a step1a
8887

8988
theorem step1 {a : ℤ√(-3)} (hcoprime : IsCoprime a.re a.im) (heven : Even a.norm) :
@@ -158,8 +157,8 @@ theorem step1'' {a p : ℤ√(-3)} (hcoprime : IsCoprime a.re a.im) (hp : p.norm
158157

159158
theorem step2 {a p : ℤ√(-3)} (hcoprime : IsCoprime a.re a.im) (hdvd : p.norm ∣ a.norm)
160159
(hpprime : Prime p.norm) :
161-
∃ u : ℤ√(-3), IsCoprime u.re u.im ∧ (a = p * u ∨ a = star p * u) ∧ a.norm = p.norm * u.norm :=
162-
by
160+
∃ u : ℤ√(-3), IsCoprime u.re u.im ∧ (a = p * u ∨ a = star p * u) ∧
161+
a.norm = p.norm * u.norm := by
163162
obtain ⟨u', h, h'⟩ := Spts.mul_of_dvd'' hdvd hpprime
164163
refine' ⟨u', _, h, h'⟩
165164
apply Zsqrtd.coprime_of_dvd_coprime hcoprime
@@ -168,23 +167,22 @@ theorem step2 {a p : ℤ√(-3)} (hcoprime : IsCoprime a.re a.im) (hdvd : p.norm
168167

169168
theorem step1_2 {a p : ℤ√(-3)} (hcoprime : IsCoprime a.re a.im) (hdvd : p.norm ∣ a.norm)
170169
(hp : OddPrimeOrFour p.norm) (hq : p.im ≠ 0) :
171-
∃ u : ℤ√(-3), IsCoprime u.re u.im ∧ (a = p * u ∨ a = star p * u) ∧ a.norm = p.norm * u.norm :=
172-
by
170+
∃ u : ℤ√(-3), IsCoprime u.re u.im ∧ (a = p * u ∨ a = star p * u) ∧
171+
a.norm = p.norm * u.norm := by
173172
obtain hp | ⟨hpprime, -⟩ := hp
174173
· rw [hp] at hdvd⊢
175174
have heven : Even a.norm :=
176175
by
177176
apply even_iff_two_dvd.mpr (dvd_trans _ hdvd)
178-
norm_num; decide
177+
norm_num
179178
exact step1'' hcoprime hp hq heven
180179
· apply step2 hcoprime hdvd hpprime
181180
#align step1_2 step1_2
182181

183182
theorem OddPrimeOrFour.factors' {a : ℤ√(-3)} (h2 : a.norm ≠ 1) (hcoprime : IsCoprime a.re a.im) :
184183
∃ u q : ℤ√(-3),
185184
0 ≤ q.re ∧
186-
q.im ≠ 0 ∧ OddPrimeOrFour q.norm ∧ a = q * u ∧ IsCoprime u.re u.im ∧ u.norm < a.norm :=
187-
by
185+
q.im ≠ 0 ∧ OddPrimeOrFour q.norm ∧ a = q * u ∧ IsCoprime u.re u.im ∧ u.norm < a.norm := by
188186
have h2 : 2 < a.norm := by
189187
apply lt_of_le_of_ne _ (Spts.not_two _).symm
190188
rw [← one_mul (2 : ℤ), mul_two, Int.add_one_le_iff]

FltRegular/FltThree/FltThree.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -279,7 +279,7 @@ theorem gcd1or3 (p q : ℤ) (hp : p ≠ 0) (hcoprime : IsCoprime p q) (hparity :
279279
suffices 32 * p
280280
by
281281
apply Int.dvd_mul_cancel_prime' _ dvd_rfl Int.prime_two this
282-
norm_num; decide
282+
norm_num
283283
have : 3 ∣ (g : ℤ) := by
284284
rw [hg, pow_two, mul_assoc, Int.ofNat_mul]
285285
apply dvd_mul_right
@@ -450,7 +450,7 @@ theorem descent_gcd1 (a b c p q : ℤ) (hp : p ≠ 0) (hcoprime : IsCoprime p q)
450450
have : 32 * p := H.mul_left 2
451451
have := IsCoprime.isUnit_of_dvd' hgcd ‹_› ‹_›
452452
rw [isUnit_iff_dvd_one] at this
453-
norm_num at this; contradiction
453+
norm_num at this
454454
have not_3_dvd_2 : ¬3 ∣ u - 3 * v := by
455455
intro hd2
456456
apply hddd
@@ -586,7 +586,7 @@ theorem descent_gcd3 (a b c p q : ℤ) (hp : p ≠ 0) (hq : q ≠ 0) (hcoprime :
586586
· zify at hgcd
587587
rw [← hgcd]
588588
exact Int.gcd_dvd_left _ _
589-
· norm_num; decide
589+
· norm_num
590590
have h3_ndvd_q : ¬3 ∣ q := by
591591
intro H
592592
have := hcoprime.isUnit_of_dvd' h3_dvd_p H

FltRegular/FltThree/OddPrimeOrFour.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -42,7 +42,7 @@ theorem OddPrimeOrFour.not_unit {z : ℤ} (h : OddPrimeOrFour z) : ¬IsUnit z :=
4242
by
4343
obtain rfl | ⟨h, -⟩ := h
4444
· rw [isUnit_iff_dvd_one]
45-
norm_num; decide
45+
norm_num
4646
· exact h.not_unit
4747
#align odd_prime_or_four.not_unit OddPrimeOrFour.not_unit
4848

@@ -95,7 +95,7 @@ theorem associated_of_dvd {a p : ℤ} (ha : OddPrimeOrFour a) (hp : OddPrimeOrFo
9595
refine' aodd _
9696
rw [even_iff_two_dvd]
9797
refine' dvd_trans _ h
98-
norm_num; decide
98+
norm_num
9999
· rwa [Prime.dvd_prime_iff_associated pp ap] at h
100100
#align associated_of_dvd associated_of_dvd
101101

lake-manifest.json

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@
44
[{"url": "https://github.com/leanprover/std4",
55
"type": "git",
66
"subDir": null,
7-
"rev": "a3b80114adc0948ff493f9acb6ee250f76922d80",
7+
"rev": "e403f680f0beb8610c29e6f799132e8be880554e",
88
"name": "std",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",
@@ -49,7 +49,7 @@
4949
{"url": "https://github.com/leanprover-community/mathlib4.git",
5050
"type": "git",
5151
"subDir": null,
52-
"rev": "81e04e3518080a288dfa9a490c048e08ab890cb0",
52+
"rev": "c26fbb123f5a4e5450ade6106621ace5f5029236",
5353
"name": "mathlib",
5454
"manifestFile": "lake-manifest.json",
5555
"inputRev": null,

0 commit comments

Comments
 (0)