Skip to content

Commit

Permalink
chore: delete unused letI and nolint (#6523)
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 committed Aug 11, 2023
1 parent ecc61a3 commit 5b3ada4
Showing 1 changed file with 0 additions and 3 deletions.
3 changes: 0 additions & 3 deletions Mathlib/FieldTheory/IsAlgClosed/Classification.lean
Expand Up @@ -207,13 +207,10 @@ private theorem ringEquivOfCardinalEqOfCharP (p : ℕ) [Fact p.Prime] [CharP K p

/-- Two uncountable algebraically closed fields are isomorphic
if they have the same cardinality and the same characteristic. -/
@[nolint defLemma]
theorem ringEquivOfCardinalEqOfCharEq (p : ℕ) [CharP K p] [CharP L p] (hK : ℵ₀ < #K)
(hKL : #K = #L) : Nonempty (K ≃+* L) := by
rcases CharP.char_is_prime_or_zero K p with (hp | hp)
· haveI : Fact p.Prime := ⟨hp⟩
letI : Algebra (ZMod p) K := ZMod.algebra _ _
letI : Algebra (ZMod p) L := ZMod.algebra _ _
exact ringEquivOfCardinalEqOfCharP p hK hKL
· simp only [hp] at *
letI : CharZero K := CharP.charP_to_charZero K
Expand Down

0 comments on commit 5b3ada4

Please sign in to comment.