Skip to content

Commit 1733bb0

Browse files
ops
1 parent 4a662f0 commit 1733bb0

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

FltRegular/CaseI/Statement.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -138,7 +138,7 @@ theorem exists_ideal {a b c : ℤ} (h5p : 5 ≤ p) (H : a ^ p + b ^ p = c ^ p)
138138
have H₁ := congr_arg (algebraMap ℤ R) H
139139
simp only [eq_intCast, Int.cast_add, Int.cast_pow] at H₁
140140
have hζ' := (zeta_spec P ℚ K).unit'_coe
141-
rw [pow_add_pow_eq_prod_add_zeta_runity_mul
141+
rw [pow_add_pow_eq_prod_add_zeta_runity_mul _ _
142142
(hpri.out.eq_two_or_odd.resolve_left fun h => by simp [h] at h5p) hζ'] at H₁
143143
replace H₁ := congr_arg (fun x => span ({ x } : Set R)) H₁
144144
simp only [← prod_span_singleton, ← span_singleton_pow] at H₁

0 commit comments

Comments
 (0)