Skip to content

Commit

Permalink
Update Mathlib/NumberTheory/NumberField/FinitePlaces.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Michael Stoll <[email protected]>
  • Loading branch information
fbarroero and MichaelStollBayreuth authored Dec 3, 2024
1 parent bea3cb8 commit 5b8d18a
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/NumberTheory/NumberField/FinitePlaces.lean
Original file line number Diff line number Diff line change
Expand Up @@ -151,7 +151,7 @@ instance : MonoidWithZeroHomClass (FinitePlace K) K ℝ where
map_zero w := w.1.map_zero

instance : NonnegHomClass (FinitePlace K) K ℝ where
apply_nonneg w _ := w.1.nonneg _
apply_nonneg w := w.1.nonneg

@[simp]
theorem apply (v : HeightOneSpectrum (𝓞 K)) (x : K) : mk v x = ‖embedding v x‖ := rfl
Expand Down

0 comments on commit 5b8d18a

Please sign in to comment.