@@ -30,7 +30,7 @@ theorem aux_cong0k₁ {k : Fin p} (hcong : k ≡ -1 [ZMOD p]) :
30
30
refine' Fin.ext _
31
31
rw [Fin.val_mk, ← ZMod.val_cast_of_lt (Fin.is_lt k)]
32
32
suffices ((k : ℤ) : ZMod p).val = p.pred by simpa
33
- rw [← ZMod.int_cast_eq_int_cast_iff ] at hcong
33
+ rw [← ZMod.intCast_eq_intCast_iff ] at hcong
34
34
rw [hcong, cast_neg, Int.cast_one, pred_eq_sub_one]
35
35
haveI : NeZero p := ⟨hpri.ne_zero⟩
36
36
haveI : Fact p.Prime := ⟨hpri⟩
@@ -84,7 +84,7 @@ theorem aux_cong0k₂ {k : Fin p} (hcong : k ≡ 1 [ZMOD p]) : k = ⟨1, hpri.on
84
84
refine' Fin.ext _
85
85
rw [Fin.val_mk, ← ZMod.val_cast_of_lt (Fin.is_lt k)]
86
86
suffices ((k : ℤ) : ZMod p).val = 1 by simpa
87
- rw [← ZMod.int_cast_eq_int_cast_iff ] at hcong
87
+ rw [← ZMod.intCast_eq_intCast_iff ] at hcong
88
88
rw [hcong, Int.cast_one]
89
89
haveI : Fact p.Prime := ⟨hpri⟩
90
90
simp [ZMod.val_one]
@@ -106,8 +106,8 @@ theorem aux0k₂ {a b : ℤ} {ζ : R} (hp5 : 5 ≤ p) (hζ : IsPrimitiveRoot ζ
106
106
symm
107
107
intro habs
108
108
replace hcong := hcong.symm
109
- rw [show (k₂ : ℤ) = 0 by simpa using habs, ← ZMod.int_cast_eq_int_cast_iff , Int.cast_sub,
110
- Int.cast_zero, sub_eq_zero, ZMod.int_cast_eq_int_cast_iff ] at hcong
109
+ rw [show (k₂ : ℤ) = 0 by simpa using habs, ← ZMod.intCast_eq_intCast_iff , Int.cast_sub,
110
+ Int.cast_zero, sub_eq_zero, ZMod.intCast_eq_intCast_iff ] at hcong
111
111
rw [habs, _root_.pow_zero, mul_one, aux_cong0k₂ hpri hcong, Fin.val_mk, pow_one, add_sub_assoc,
112
112
← sub_mul, add_sub_right_comm, show ζ = ζ ^ ((⟨1 , hpri.one_lt⟩ : Fin p) : ℕ) by simp] at hdiv
113
113
have key : ↑(p : ℤ) ∣ ∑ j in range p, f0k₂ a b j • ζ ^ j := by
@@ -119,7 +119,7 @@ theorem aux0k₂ {a b : ℤ} {ζ : R} (hp5 : 5 ≤ p) (hζ : IsPrimitiveRoot ζ
119
119
rw [sum_range] at key
120
120
refine' hab _
121
121
symm
122
- rw [← ZMod.int_cast_eq_int_cast_iff , ZMod.int_cast_eq_int_cast_iff_dvd_sub ]
122
+ rw [← ZMod.intCast_eq_intCast_iff , ZMod.intCast_eq_intCast_iff_dvd_sub ]
123
123
have hpri₁ : (P : ℕ).Prime := hpri
124
124
simpa [f0k₂] using dvd_coeff_cycl_integer hpri₁ hζ (auxf0k₂ hpri hp5 a b) key ⟨0 , hpri.pos⟩
125
125
@@ -131,7 +131,7 @@ theorem aux_cong1k₁ {k : Fin p} (hcong : k ≡ 0 [ZMOD p]) : k = ⟨0, hpri.po
131
131
refine' Fin.ext _
132
132
rw [Fin.val_mk, ← ZMod.val_cast_of_lt (Fin.is_lt k)]
133
133
suffices ((k : ℤ) : ZMod p).val = 0 by simpa
134
- rw [← ZMod.int_cast_eq_int_cast_iff ] at hcong
134
+ rw [← ZMod.intCast_eq_intCast_iff ] at hcong
135
135
rw [hcong, Int.cast_zero]
136
136
haveI : Fact p.Prime := ⟨hpri⟩
137
137
simp
@@ -158,7 +158,7 @@ theorem aux_cong1k₂ {k : Fin p} (hpri : p.Prime) (hp5 : 5 ≤ p) (hcong : k
158
158
refine' Fin.ext _
159
159
rw [Fin.val_mk, ← ZMod.val_cast_of_lt (Fin.is_lt k)]
160
160
suffices ((k : ℤ) : ZMod p).val = 2 by simpa
161
- rw [← ZMod.int_cast_eq_int_cast_iff ] at hcong
161
+ rw [← ZMod.intCast_eq_intCast_iff ] at hcong
162
162
rw [hcong]
163
163
simp only [Int.cast_add, algebraMap.coe_one]
164
164
haveI : Fact p.Prime := ⟨hpri⟩
@@ -187,8 +187,8 @@ theorem aux1k₂ {a b c : ℤ} {ζ : R} (hp5 : 5 ≤ p) (hζ : IsPrimitiveRoot
187
187
symm
188
188
intro habs
189
189
replace hcong := hcong.symm
190
- rw [show (k₂ : ℤ) = 1 by simpa using habs, ← ZMod.int_cast_eq_int_cast_iff , Int.cast_sub,
191
- sub_eq_iff_eq_add, ← Int.cast_add, ZMod.int_cast_eq_int_cast_iff ] at hcong
190
+ rw [show (k₂ : ℤ) = 1 by simpa using habs, ← ZMod.intCast_eq_intCast_iff , Int.cast_sub,
191
+ sub_eq_iff_eq_add, ← Int.cast_add, ZMod.intCast_eq_intCast_iff ] at hcong
192
192
rw [habs, pow_one, aux_cong1k₂ hpri hp5 hcong] at hdiv
193
193
ring_nf at hdiv
194
194
have key : ↑(p : ℤ) ∣ ∑ j in range p, f1k₂ a j • ζ ^ j := by
@@ -212,7 +212,7 @@ theorem auxk₁k₂ {k₁ k₂ : Fin p} (hpri : p.Prime) (hcong : k₂ ≡ k₁
212
212
(k₁ : ℕ) ≠ (k₂ : ℕ) := by
213
213
haveI := (⟨hpri⟩ : Fact p.Prime)
214
214
intro habs
215
- rw [habs, ← ZMod.int_cast_eq_int_cast_iff , Int.cast_sub, ← sub_eq_zero] at hcong
215
+ rw [habs, ← ZMod.intCast_eq_intCast_iff , Int.cast_sub, ← sub_eq_zero] at hcong
216
216
simp at hcong
217
217
218
218
end KoneKtwo
0 commit comments