Skip to content

Commit

Permalink
bump to nightly-2023-09-27-06
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Sep 27, 2023
1 parent 61f91ae commit b3e015b
Show file tree
Hide file tree
Showing 5 changed files with 11 additions and 11 deletions.
2 changes: 1 addition & 1 deletion Mathbin/Data/Polynomial/Degree/Definitions.lean
Expand Up @@ -270,7 +270,7 @@ theorem degree_ne_of_natDegree_ne {n : ℕ} : p.natDegree ≠ n → degree p ≠

#print Polynomial.natDegree_le_iff_degree_le /-
theorem natDegree_le_iff_degree_le {n : ℕ} : natDegree p ≤ n ↔ degree p ≤ n :=
WithBot.unbot'_bot_le_iff
WithBot.unbot'_le_iff
#align polynomial.nat_degree_le_iff_degree_le Polynomial.natDegree_le_iff_degree_le
-/

Expand Down
2 changes: 1 addition & 1 deletion Mathbin/Order/GaloisConnection.lean
Expand Up @@ -1176,7 +1176,7 @@ coercion form a Galois insertion. -/
def WithBot.giUnbot'Bot [Preorder α] [OrderBot α] :
GaloisInsertion (WithBot.unbot' ⊥) (coe : α → WithBot α)
where
gc a b := WithBot.unbot'_bot_le_iff
gc a b := WithBot.unbot'_le_iff
le_l_u a := le_rfl
choice o ho := o.unbot' ⊥
choice_eq _ _ := rfl
Expand Down
6 changes: 3 additions & 3 deletions Mathbin/Order/WithBot.lean
Expand Up @@ -480,10 +480,10 @@ theorem le_coe_unbot' [Preorder α] : ∀ (a : WithBot α) (b : α), a ≤ a.unb
#align with_bot.le_coe_unbot' WithBot.le_coe_unbot'
-/

#print WithBot.unbot'_bot_le_iff /-
theorem unbot'_bot_le_iff [LE α] [OrderBot α] {a : WithBot α} {b : α} : a.unbot' ⊥ ≤ b ↔ a ≤ b := by
#print WithBot.unbot'_le_iff /-
theorem unbot'_le_iff [LE α] [OrderBot α] {a : WithBot α} {b : α} : a.unbot' ⊥ ≤ b ↔ a ≤ b := by
cases a <;> simp [none_eq_bot, some_eq_coe]
#align with_bot.unbot'_bot_le_iff WithBot.unbot'_bot_le_iff
#align with_bot.unbot'_bot_le_iff WithBot.unbot'_le_iff
-/

#print WithBot.unbot'_lt_iff /-
Expand Down
8 changes: 4 additions & 4 deletions lake-manifest.json
Expand Up @@ -4,18 +4,18 @@
[{"git":
{"url": "https://github.com/leanprover-community/lean3port.git",
"subDir?": null,
"rev": "1ce0a5a3986b4c41d2282f72802fc3776d8b8381",
"rev": "758cb0e8c273df825524e578128e3e94e0c639d3",
"opts": {},
"name": "lean3port",
"inputRev?": "1ce0a5a3986b4c41d2282f72802fc3776d8b8381",
"inputRev?": "758cb0e8c273df825524e578128e3e94e0c639d3",
"inherited": false}},
{"git":
{"url": "https://github.com/leanprover-community/mathlib4.git",
"subDir?": null,
"rev": "6f7f5f38aeade5fd16b2d96674a055b3a850e736",
"rev": "0fd376a2a6771146b41dfd81b6726431ebc5f2c4",
"opts": {},
"name": "mathlib",
"inputRev?": "6f7f5f38aeade5fd16b2d96674a055b3a850e736",
"inputRev?": "0fd376a2a6771146b41dfd81b6726431ebc5f2c4",
"inherited": true}},
{"git":
{"url": "https://github.com/mhuisi/lean4-cli.git",
Expand Down
4 changes: 2 additions & 2 deletions lakefile.lean
Expand Up @@ -4,7 +4,7 @@ open Lake DSL System
-- Usually the `tag` will be of the form `nightly-2021-11-22`.
-- If you would like to use an artifact from a PR build,
-- it will be of the form `pr-branchname-sha`.
def tag : String := "nightly-2023-09-26-06"
def tag : String := "nightly-2023-09-27-06"
def releaseRepo : String := "leanprover-community/mathport"
def oleanTarName : String := "mathlib3-binport.tar.gz"

Expand Down Expand Up @@ -38,7 +38,7 @@ target fetchOleans (_pkg) : Unit := do
untarReleaseArtifact releaseRepo tag oleanTarName libDir
return .nil

require lean3port from git "https://github.com/leanprover-community/lean3port.git"@"1ce0a5a3986b4c41d2282f72802fc3776d8b8381"
require lean3port from git "https://github.com/leanprover-community/lean3port.git"@"758cb0e8c273df825524e578128e3e94e0c639d3"

@[default_target]
lean_lib Mathbin where
Expand Down

0 comments on commit b3e015b

Please sign in to comment.