Skip to content

Commit

Permalink
chore: bump dependencies (#8149)
Browse files Browse the repository at this point in the history
Co-authored-by: Scott Morrison <[email protected]>
  • Loading branch information
kim-em and kim-em committed Nov 3, 2023
1 parent 2e15c5a commit 7d18b6d
Show file tree
Hide file tree
Showing 2 changed files with 13 additions and 15 deletions.
8 changes: 3 additions & 5 deletions Mathlib/Logic/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -356,11 +356,9 @@ theorem Or.imp3 (had : a → d) (hbe : b → e) (hcf : c → f) : a ∨ b ∨ c

#align or_imp_distrib or_imp

theorem or_iff_not_imp_left : a ∨ b ↔ ¬a → b := Decidable.or_iff_not_imp_left
#align or_iff_not_imp_left or_iff_not_imp_left

theorem or_iff_not_imp_right : a ∨ b ↔ ¬b → a := Decidable.or_iff_not_imp_right
#align or_iff_not_imp_right or_iff_not_imp_right
export Classical (or_iff_not_imp_left or_iff_not_imp_right)
#align or_iff_not_imp_left Classical.or_iff_not_imp_left
#align or_iff_not_imp_right Classical.or_iff_not_imp_right

theorem not_or_of_imp : (a → b) → ¬a ∨ b := Decidable.not_or_of_imp
#align not_or_of_imp not_or_of_imp
Expand Down
20 changes: 10 additions & 10 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,27 +4,19 @@
[{"git":
{"url": "https://github.com/leanprover/std4",
"subDir?": null,
"rev": "795918af0b01cd79aea67f828f215cca71699eca",
"rev": "9bfbd2a12ee9cf2e159a8a6b4d1ef6c149728f66",
"opts": {},
"name": "std",
"inputRev?": "main",
"inherited": false}},
{"git":
{"url": "https://github.com/leanprover-community/quote4",
"subDir?": null,
"rev": "a387c0eb611857e2460cf97a8e861c944286e6b2",
"rev": "396201245bf244f9d78e9007a02dd1c388193d27",
"opts": {},
"name": "Qq",
"inputRev?": "master",
"inherited": false}},
{"git":
{"url": "https://github.com/leanprover-community/aesop",
"subDir?": null,
"rev": "c9dbd09c1e02b66d09384076f7e0090d3df300d5",
"opts": {},
"name": "aesop",
"inputRev?": "master",
"inherited": false}},
{"git":
{"url": "https://github.com/leanprover/lean4-cli",
"subDir?": null,
Expand All @@ -40,5 +32,13 @@
"opts": {},
"name": "proofwidgets",
"inputRev?": "v0.0.21",
"inherited": false}},
{"git":
{"url": "https://github.com/leanprover-community/aesop",
"subDir?": null,
"rev": "cb87803274405db79ec578fc07c4730c093efb90",
"opts": {},
"name": "aesop",
"inputRev?": "master",
"inherited": false}}],
"name": "mathlib"}

0 comments on commit 7d18b6d

Please sign in to comment.