Update mathlib

This commit is contained in:
Stefan Kebekus 2024-11-29 09:55:22 +01:00
parent e20dcdbd19
commit eec4cd1ffa
3 changed files with 6 additions and 6 deletions

View File

@ -94,9 +94,9 @@ lemma int₀
let ρ := ‖a‖⁻¹ let ρ := ‖a‖⁻¹
have hρ : 1 < ρ := by have hρ : 1 < ρ := by
apply one_lt_inv_iff.mpr apply one_lt_inv_iff.mpr
constructor constructor
· exact norm_pos_iff'.mpr h₁a · exact norm_pos_iff.mpr h₁a
· exact mem_ball_zero_iff.mp ha · exact mem_ball_zero_iff.mp ha
let F := fun z ↦ log ‖1 - z * a‖ let F := fun z ↦ log ‖1 - z * a‖
@ -114,7 +114,7 @@ lemma int₀
_ < ρ * ‖a‖ := by _ < ρ * ‖a‖ := by
apply (mul_lt_mul_right _).2 apply (mul_lt_mul_right _).2
exact mem_ball_zero_iff.mp hx exact mem_ball_zero_iff.mp hx
exact norm_pos_iff'.mpr h₁a exact norm_pos_iff.mpr h₁a
_ = 1 := by _ = 1 := by
dsimp [ρ] dsimp [ρ]
apply inv_mul_cancel₀ apply inv_mul_cancel₀

View File

@ -5,7 +5,7 @@
"type": "git", "type": "git",
"subDir": null, "subDir": null,
"scope": "leanprover-community", "scope": "leanprover-community",
"rev": "44e2d2e643fd2618b01f9a0592d7dcbd3ffa22de", "rev": "c933dd9b00271d869e22b802a015092d1e8e454a",
"name": "batteries", "name": "batteries",
"manifestFile": "lake-manifest.json", "manifestFile": "lake-manifest.json",
"inputRev": "main", "inputRev": "main",
@ -85,7 +85,7 @@
"type": "git", "type": "git",
"subDir": null, "subDir": null,
"scope": "", "scope": "",
"rev": "b96544419e0739c6aefecfc4ee368400a77266ce", "rev": "ab780650a6c8db2942d137b91ede7c94c47a4950",
"name": "mathlib", "name": "mathlib",
"manifestFile": "lake-manifest.json", "manifestFile": "lake-manifest.json",
"inputRev": null, "inputRev": null,

View File

@ -1 +1 @@
leanprover/lean4:v4.14.0-rc2 leanprover/lean4:v4.14.0-rc3