Update mathlib

This commit is contained in:
Stefan Kebekus 2024-10-31 07:37:54 +01:00
parent 279dcd32b9
commit 449de2e42a
2 changed files with 4 additions and 4 deletions

View File

@ -24,7 +24,7 @@ lemma logsinBound : ∀ x ∈ (Set.Icc 0 1), ‖(log ∘ sin) x‖ ≤ ‖log ((
exact zero_lt_two exact zero_lt_two
apply (Set.mem_Icc.1 hx).1 apply (Set.mem_Icc.1 hx).1
simp simp
apply mul_le_one apply mul_le_one
rw [div_le_one pi_pos] rw [div_le_one pi_pos]
exact two_le_pi exact two_le_pi
exact (Set.mem_Icc.1 hx).1 exact (Set.mem_Icc.1 hx).1

View File

@ -5,7 +5,7 @@
"type": "git", "type": "git",
"subDir": null, "subDir": null,
"scope": "leanprover-community", "scope": "leanprover-community",
"rev": "dc72dcdb8e97b3c56bd70f06f043ed2dee3258e6", "rev": "500a529408399c44d7e1649577e3c98697f95aa4",
"name": "batteries", "name": "batteries",
"manifestFile": "lake-manifest.json", "manifestFile": "lake-manifest.json",
"inputRev": "main", "inputRev": "main",
@ -55,7 +55,7 @@
"type": "git", "type": "git",
"subDir": null, "subDir": null,
"scope": "leanprover-community", "scope": "leanprover-community",
"rev": "0ea83a676d288220ba227808568cbb80fe43ace0", "rev": "c1970bea80ac3357a6a991a6d00d12e7435c12c7",
"name": "importGraph", "name": "importGraph",
"manifestFile": "lake-manifest.json", "manifestFile": "lake-manifest.json",
"inputRev": "main", "inputRev": "main",
@ -75,7 +75,7 @@
"type": "git", "type": "git",
"subDir": null, "subDir": null,
"scope": "", "scope": "",
"rev": "893b3a846645d48ac45143ec02149cc551acd99d", "rev": "d9273054fe5aee13954cca827d9bbfe7a01bde67",
"name": "mathlib", "name": "mathlib",
"manifestFile": "lake-manifest.json", "manifestFile": "lake-manifest.json",
"inputRev": null, "inputRev": null,