Skip to content

Commit

Permalink
bump to nightly-2024-01-28-06
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Jan 28, 2024
1 parent 5704388 commit fe4dd9a
Show file tree
Hide file tree
Showing 4 changed files with 10 additions and 10 deletions.
6 changes: 3 additions & 3 deletions Mathbin/Data/Nat/Parity.lean
Expand Up @@ -313,14 +313,14 @@ theorem even_mul_succ_self (n : ℕ) : Even (n * (n + 1)) :=
#align nat.even_mul_succ_self Nat.even_mul_succ_self
-/

#print Nat.even_mul_self_pred /-
theorem even_mul_self_pred (n : ℕ) : Even (n * (n - 1)) :=
#print Nat.even_mul_pred_self /-
theorem even_mul_pred_self (n : ℕ) : Even (n * (n - 1)) :=
by
cases n
· exact even_zero
· rw [mul_comm]
apply even_mul_succ_self
#align nat.even_mul_self_pred Nat.even_mul_self_pred
#align nat.even_mul_self_pred Nat.even_mul_pred_self
-/

#print Nat.two_mul_div_two_of_even /-
Expand Down
2 changes: 1 addition & 1 deletion Mathbin/RingTheory/Discriminant.lean
Expand Up @@ -229,7 +229,7 @@ theorem discr_powerBasis_eq_prod'' [IsSeparable K L] (e : Fin pb.dim ≃ (L →
by
rw [← AlgHom.card K L E, ← Fintype.card_fin pb.dim]
exact card_congr (Equiv.symm e)
have h₂ : 2 ∣ pb.dim * (pb.dim - 1) := even_iff_two_dvd.1 (Nat.even_mul_self_pred _)
have h₂ : 2 ∣ pb.dim * (pb.dim - 1) := even_iff_two_dvd.1 (Nat.even_mul_pred_self _)
have hne : ((2 : ℕ) : ℚ) ≠ 0 := by simp
have hle : 1 ≤ pb.dim :=
by
Expand Down
8 changes: 4 additions & 4 deletions lake-manifest.json
Expand Up @@ -58,19 +58,19 @@
{"url": "https://github.com/leanprover-community/mathlib4.git",
"type": "git",
"subDir": null,
"rev": "970a1ab2bfb8a7921fd05c872c630a0a83632bb8",
"rev": "62acecee993214f545acf44c171ee0e2a2fe4051",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": "970a1ab2bfb8a7921fd05c872c630a0a83632bb8",
"inputRev": "62acecee993214f545acf44c171ee0e2a2fe4051",
"inherited": true,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover-community/lean3port.git",
"type": "git",
"subDir": null,
"rev": "b1f6bf1e0388482dd12c4c9887d34e01aedb30f7",
"rev": "3b890e7719e32224564d4af64c69d2e725b421fb",
"name": "lean3port",
"manifestFile": "lake-manifest.json",
"inputRev": "b1f6bf1e0388482dd12c4c9887d34e01aedb30f7",
"inputRev": "3b890e7719e32224564d4af64c69d2e725b421fb",
"inherited": false,
"configFile": "lakefile.lean"}],
"name": "mathlib3port",
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-2024-01-27-06"
def tag : String := "nightly-2024-01-28-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"@"b1f6bf1e0388482dd12c4c9887d34e01aedb30f7"
require lean3port from git "https://github.com/leanprover-community/lean3port.git"@"3b890e7719e32224564d4af64c69d2e725b421fb"

@[default_target]
lean_lib Mathbin where
Expand Down

0 comments on commit fe4dd9a

Please sign in to comment.