Skip to content

Commit

Permalink
Merge branch 'nightly-testing' of github.com:leanprover-community/mat…
Browse files Browse the repository at this point in the history
…hlib4 into nightly-testing
  • Loading branch information
kim-em committed Aug 28, 2024
2 parents 7a1ec97 + 2b343f2 commit 6c31c06
Show file tree
Hide file tree
Showing 2 changed files with 6 additions and 2 deletions.
3 changes: 3 additions & 0 deletions Mathlib/Analysis/SpecialFunctions/Log/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -275,6 +275,9 @@ theorem log_le_sub_one_of_pos {x : ℝ} (hx : 0 < x) : log x ≤ x - 1 := by
convert add_one_le_exp (log x)
rw [exp_log hx]

lemma one_sub_inv_le_log_of_pos (hx : 0 < x) : 1 - x⁻¹ ≤ log x := by
simpa [add_comm] using log_le_sub_one_of_pos (inv_pos.2 hx)

/-- Bound for `|log x * x|` in the interval `(0, 1]`. -/
theorem abs_log_mul_self_lt (x : ℝ) (h1 : 0 < x) (h2 : x ≤ 1) : |log x * x| < 1 := by
have : 0 < 1 / x := by simpa only [one_div, inv_pos] using h1
Expand Down
5 changes: 3 additions & 2 deletions Mathlib/RingTheory/Valuation/AlgebraInstances.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,3 @@
#exit
/-
Copyright (c) 2024 María Inés de Frutos-Fernández, Filippo A. E. Nuccio. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Expand Down Expand Up @@ -33,7 +32,7 @@ variable {K : Type*} [Field K] (v : Valuation K ℤₘ₀) (L : Type*) [Field L]
namespace ValuationSubring

-- Implementation note : this instance was automatic in Lean3
instance smul : SMul v.valuationSubring (integralClosure v.valuationSubring L) := Algebra.toSMul
instance : Algebra v.valuationSubring L := Algebra.ofSubring v.valuationSubring.toSubring

theorem algebraMap_injective : Injective (algebraMap v.valuationSubring L) :=
(NoZeroSMulDivisors.algebraMap_injective K L).comp (IsFractionRing.injective _ _)
Expand All @@ -51,6 +50,8 @@ theorem isIntegral_of_mem_ringOfIntegers' {x : (integralClosure v.valuationSubri

variable (E : Type _) [Field E] [Algebra K E] [Algebra L E] [IsScalarTower K L E]

-- Imprementation note: this instance was not needed until 28-08-2024

This comment has been minimized.

Copy link
@mattrobball

mattrobball Aug 28, 2024

Collaborator

Both of these are re-declarations with the keys for the type ValuationSubring as opposed to the previous Subring.

instance : IsScalarTower v.valuationSubring L E := Subring.instIsScalarTowerSubtypeMem _
/-- Given an algebra between two field extensions `L` and `E` of a field `K` with a valuation `v`,
create an algebra between their two rings of integers. -/
instance algebra :
Expand Down

0 comments on commit 6c31c06

Please sign in to comment.