Skip to content

Commit 069873c

Browse files
committed
feat: tweaks to roundtrip with new CI releases
1 parent 7ea701f commit 069873c

File tree

4 files changed

+6
-6
lines changed

4 files changed

+6
-6
lines changed

Diff for: Lean4Packages/leanbin/lakefile.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
11
import Lake
22
open Lake DSL System
33

4-
def tag : String := "pr-CI-ac6084d" -- "nightly-2021-11-11"
4+
def tag : String := "nightly-2021-11-17"
55
def releaseRepo : String := "leanprover-community/mathport"
66
def tarName : String := "lean3-binport.tar.gz"
77

@@ -34,6 +34,6 @@ package leanbin (dir) {
3434
defaultFacet := PackageFacet.oleans
3535
dependencies := #[{
3636
name := "mathlib",
37-
src := Source.git "https://github.com/dselsam/mathlib4.git" "5366ff9252f9001fc10e610795efd259fd4b8dc6"
37+
src := Source.git "https://github.com/leanprover-community/mathlib4.git" "64f9c43eb9a75fb4c5989ac711623d06e9696e60"
3838
}]
3939
}

Diff for: Lean4Packages/leanbin/lean-toolchain

+1-1
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:nightly-2021-10-28
1+
leanprover/lean4:nightly-2021-11-07

Diff for: Lean4Packages/mathbin/lakefile.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
11
import Lake
22
open Lake DSL System
33

4-
def tag : String := "pr-CI-ac6084d" -- "nightly-2021-11-11"
4+
def tag : String := "nightly-2021-11-17"
55
def releaseRepo : String := "leanprover-community/mathport"
66
def tarName : String := "mathlib3-binport.tar.gz"
77

@@ -34,7 +34,7 @@ package mathbin (dir) {
3434
defaultFacet := PackageFacet.oleans
3535
dependencies := #[{
3636
name := "leanbin",
37-
src := Source.git "https://github.com/dselsam/mathport.git" "master",
37+
src := Source.git "https://github.com/leanprover-community/mathport.git" "master",
3838
dir := "Lean4Packages/leanbin"
3939
}]
4040
}

Diff for: Lean4Packages/mathbin/lean-toolchain

+1-1
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:nightly-2021-10-28
1+
leanprover/lean4:nightly-2021-11-07

0 commit comments

Comments
 (0)