Skip to content

Commit eafed89

Browse files
committed
more deprecations
1 parent 13ffc81 commit eafed89

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

Mathlib/NumberTheory/Cyclotomic/Discriminant.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -102,8 +102,8 @@ theorem discr_prime_pow_ne_two [IsCyclotomicExtension {p ^ (k + 1)} K L] [hp : F
102102
replace H := congr_arg (Algebra.norm K) H
103103
have hnorm : (norm K) (ζ ^ (p : ℕ) ^ k - 1) = (p : K) ^ (p : ℕ) ^ k := by
104104
by_cases hp : p = 2
105-
· exact mod_cast hζ.pow_sub_one_norm_prime_pow_of_ne_zero hirr le_rfl (hp2 hp)
106-
· exact mod_cast hζ.pow_sub_one_norm_prime_ne_two hirr le_rfl hp
105+
· exact mod_cast hζ.norm_pow_sub_one_eq_prime_pow_of_ne_zero hirr le_rfl (hp2 hp)
106+
· exact mod_cast hζ.norm_pow_sub_one_of_prime_ne_two hirr le_rfl hp
107107
rw [MonoidHom.map_mul, hnorm, MonoidHom.map_mul, ← map_natCast (algebraMap K L),
108108
Algebra.norm_algebraMap, finrank L hirr] at H
109109
conv_rhs at H => -- Porting note: need to drill down to successfully rewrite the totient

0 commit comments

Comments
 (0)