Skip to content

Commit

Permalink
chore(number_theory/number_field/basic): fix a name (#16943)
Browse files Browse the repository at this point in the history
This lemma is in the `ring_of_integers` namespace, so the name was redundant.
  • Loading branch information
riccardobrasca committed Oct 13, 2022
1 parent 5147123 commit 2976108
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/number_theory/number_field/basic.lean
Expand Up @@ -102,7 +102,7 @@ integral_closure.is_integrally_closed_of_finite_extension ℚ
lemma is_integral_coe (x : 𝓞 K) : is_integral ℤ (x : K) :=
x.2

lemma map_mem_ring_of_integers {F L : Type*} [field L] [char_zero K] [char_zero L]
lemma map_mem {F L : Type*} [field L] [char_zero K] [char_zero L]
[alg_hom_class F ℚ K L] (f : F) (x : 𝓞 K) : f x ∈ 𝓞 L :=
(mem_ring_of_integers _ _).2 $ map_is_integral_int f $ ring_of_integers.is_integral_coe x

Expand Down

0 comments on commit 2976108

Please sign in to comment.