Skip to content

Commit

Permalink
chore: bump to 2022-12-23 (#1191)
Browse files Browse the repository at this point in the history
  • Loading branch information
gebner committed Dec 23, 2022
1 parent 101a430 commit 08e8d37
Show file tree
Hide file tree
Showing 3 changed files with 6 additions and 6 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Data/Int/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -275,7 +275,7 @@ theorem sign_coe_nat_of_nonzero {n : ℕ} (hn : n ≠ 0) : Int.sign n = 1 := sig
#align int.to_nat_add_nat Int.toNat_add_nat
#align int.pred_to_nat Int.pred_toNat
#align int.to_nat_sub_to_nat_neg Int.toNat_sub_toNat_neg
#align int.to_nat_add_to_nat_neg_eq_nat_abs Int.toNat_add_toNat_neg_eq_nat_abs
#align int.to_nat_add_to_nat_neg_eq_nat_abs Int.toNat_add_toNat_neg_eq_natAbs
#align int.mem_to_nat' Int.mem_toNat'
#align int.toNat_neg_nat Int.toNat_neg_nat

Expand Down
8 changes: 4 additions & 4 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -10,13 +10,13 @@
{"git":
{"url": "https://github.com/leanprover/lake",
"subDir?": null,
"rev": "235383015cdcb0082777b0347b84dba01843c79c",
"rev": "d0b530530f14dde97a547b03abf87eee06360d60",
"name": "lake",
"inputRev?": "master"}},
{"git":
{"url": "https://github.com/leanprover/doc-gen4",
"subDir?": null,
"rev": "f221bbdcffe6a17bb310f0e9ee10767812b03e13",
"rev": "bdf803b1002786b87da7b8db8d2746c0002a715f",
"name": "doc-gen4",
"inputRev?": "main"}},
{"git":
Expand All @@ -40,7 +40,7 @@
{"git":
{"url": "https://github.com/hargonix/LeanInk",
"subDir?": null,
"rev": "9f3101452135964ac9107ec8e9910bfd14022bbc",
"rev": "2447df5cc6e48eb965c3c3fba87e46d353b5e9f1",
"name": "leanInk",
"inputRev?": "doc-gen"}},
{"git":
Expand All @@ -52,6 +52,6 @@
{"git":
{"url": "https://github.com/leanprover/std4",
"subDir?": null,
"rev": "2ace3a9803a96fd765d588b2a95fb6fafaf05bb3",
"rev": "a109889bf299f0d086f93a228e4c152f40ff5b0d",
"name": "std",
"inputRev?": "main"}}]}
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:nightly-2022-12-22
leanprover/lean4:nightly-2022-12-23

0 comments on commit 08e8d37

Please sign in to comment.