Update mathlib

This commit is contained in:
Stefan Kebekus 2024-11-11 08:46:26 +01:00
parent 6d403874e2
commit f3e951884f
3 changed files with 21 additions and 11 deletions

View File

@ -31,7 +31,7 @@ theorem CauchyRiemann₃ : (DifferentiableAt f z)
have ContinuousLinearMap.comp_lineDeriv : ∀ w : , ∀ l : →L[] , lineDeriv (l ∘ f) z w = l ((fderiv f z) w) := by
intro w l
rw [DifferentiableAt.lineDeriv_eq_fderiv]
rw [fderiv.comp]
rw [fderiv_comp]
simp
fun_prop
exact h.restrictScalars

View File

@ -5,7 +5,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "500a529408399c44d7e1649577e3c98697f95aa4",
"rev": "325d06c3ef6bcb16c43c4ac6614976731ce6a63e",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
@ -15,7 +15,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "1357f4f49450abb9dfd4783e38219f4ce84f9785",
"rev": "303b23fbcea94ac4f96e590c1cad6618fd4f5f41",
"name": "Qq",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
@ -25,7 +25,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "9ac12945862fa39eab7795c2f79bb9aa0c8e332c",
"rev": "5dfdc66e0d503631527ad90c1b5d7815c86a8662",
"name": "aesop",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
@ -35,17 +35,17 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "baa65c6339a56bd22b7292aa4511c54b3cc7a6af",
"rev": "1383e72b40dd62a566896a6e348ffe868801b172",
"name": "proofwidgets",
"manifestFile": "lake-manifest.json",
"inputRev": "v0.0.43",
"inputRev": "v0.0.46",
"inherited": true,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover/lean4-cli",
"type": "git",
"subDir": null,
"scope": "leanprover",
"rev": "2cf1030dc2ae6b3632c84a09350b675ef3e347d0",
"rev": "726b3c9ad13acca724d4651f14afc4804a7b0e4d",
"name": "Cli",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
@ -55,7 +55,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "c1970bea80ac3357a6a991a6d00d12e7435c12c7",
"rev": "ac7b989cbf99169509433124ae484318e953d201",
"name": "importGraph",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
@ -65,17 +65,27 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "7bedaed1ef024add1e171cc17706b012a9a37802",
"rev": "86d0d0584f5cd165353e2f8a30c455cd0e168ac2",
"name": "LeanSearchClient",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inherited": true,
"configFile": "lakefile.toml"},
{"url": "https://github.com/leanprover-community/plausible",
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "42dc02bdbc5d0c2f395718462a76c3d87318f7fa",
"name": "plausible",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inherited": true,
"configFile": "lakefile.toml"},
{"url": "https://github.com/leanprover-community/mathlib4.git",
"type": "git",
"subDir": null,
"scope": "",
"rev": "d9273054fe5aee13954cca827d9bbfe7a01bde67",
"rev": "b8570f16d4170663edb8a12b8eae9f0d84e96ab4",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,

View File

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