Zulip Chat Archive

Stream: nightly-testing

Topic: Mathlib status updates


github mathlib4 bot (Mar 15 2024 at 09:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 15 2024 at 10:02):

The importGraph package will need updating.

github mathlib4 bot (Mar 15 2024 at 10:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 15 2024 at 10:17):

Okay, there is a lot more fallout from https://github.com/leanprover/lean4/pull/3675.

Kim Morrison (Mar 15 2024 at 10:18):

Some of this is that auxiliary lemmas generated by simp have changed names.

Kim Morrison (Mar 15 2024 at 10:18):

Try replace foo._eq_1 with foo.eq_1; this fixes a lot of it. (Also try omitting it from the simp set: this often seems to work.)

Kim Morrison (Mar 15 2024 at 10:20):

  • There is a not-obviously related problem in Mathlib.Data.Nat.Bitwise.

github mathlib4 bot (Mar 15 2024 at 10:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 15 2024 at 10:33):

  • Failure in Mathlib.Data.Rel, where it seems like attribute [eqns flip_def] flip is no longer working.
  • Mathlib.Control.Fold is affected by the same issue.
  • Mathlib.Data.DFinsupp.WellFounded too.

Finding a minimal example of this problem with @[eqns] seems like a priority: whether the fix belongs in Mathlib.Tactic.Eqns or needs to go upstream. Pinging @Eric Wieser as the @[eqns] expert. :-)

Kim Morrison (Mar 15 2024 at 10:41):

I'm done for the day. Suggestion for anyone who wants to work on this:

  • Claim either of the bullet points above with a :hammer_and_wrench: and try to work out what has happened!
  • There are more errors in the build, so just running lake build and seeing what you encounter is useful.
  • There are enough problems that it is helpful if you encounter an error that you can't immediately fix to:
    • Add -- FIXME nightly-testing
    • Sorry the broken proof
    • Post a bullet point here for someone to claim.

github mathlib4 bot (Mar 15 2024 at 11:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 15 2024 at 13:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 15 2024 at 15:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 15 2024 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 16 2024 at 01:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 16 2024 at 10:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Mar 16 2024 at 12:02):

This is fun - we have a theorem Asymptotics.IsLittleO.def but lean doesn't allow calling things def anymore

github mathlib4 bot (Mar 16 2024 at 12:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 16 2024 at 12:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 16 2024 at 12:33):

Yes, we have quite a few of these. I've been renaming def to def'... Ideas?

Ruben Van de Velde (Mar 16 2024 at 12:35):

The first one I encountered already had a def', so I used definition

github mathlib4 bot (Mar 16 2024 at 12:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 16 2024 at 15:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kevin Buzzard (Mar 16 2024 at 16:23):

I only recently discovered that definition was not a keyword! I had always imagined that def was short for it.

Kyle Miller (Mar 16 2024 at 17:00):

Lean 3 had definition as a keyword! Lean 4 cleaned up some synonyms.

Eric Wieser (Mar 16 2024 at 17:20):

We can just use «def», right?

Kyle Miller (Mar 16 2024 at 18:41):

There's a change to the equation lemma generator, and now .def is reserved

github mathlib4 bot (Mar 16 2024 at 18:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 16 2024 at 21:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 16 2024 at 23:03):

/poll What to do with .def being reserved?

Kyle Miller (Mar 16 2024 at 23:57):

What does option «def» mean? Isn't that equivalent to def?

github mathlib4 bot (Mar 17 2024 at 00:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kyle Miller (Mar 17 2024 at 01:00):

For Asymptotics.IsLittleO.def, that isn't the definition of Asymptotics.IsLittleO, so why is it called def?

Are there other cases where Lean's auto-generated def isn't the def lemma that we wanted?

github mathlib4 bot (Mar 17 2024 at 03:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 17 2024 at 04:41):

Resuming work on this, just dealing with errors from lake build

Kim Morrison (Mar 17 2024 at 04:44):

Would unfold be good as an alternative for the automatically generated (and reserved) name?

Mario Carneiro (Mar 17 2024 at 04:46):

might be good to set up some basic test for this by querying the import Mathlib environment and seeing how popular various choices are

Mario Carneiro (Mar 17 2024 at 04:48):

my gut feeling is that foo.unfold will have fewer hits than foo.def

Mario Carneiro (Mar 17 2024 at 04:48):

what exactly is it being reserved for?

Mario Carneiro (Mar 17 2024 at 04:49):

Aren't unfolding theorems already called foo.eq_<n>?

github mathlib4 bot (Mar 17 2024 at 04:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 17 2024 at 04:58):

I've created #11437 with the adaptations so far for nightly-2024-3-16. Let's work on that in preference to nightly-testing, so we can try to get this done without having to deal with subsequent changes as nightly-testing automatically advances.

Kim Morrison (Mar 17 2024 at 05:02):

@Mario Carneiro, e.g.:

#print IsSeparator
-- def CategoryTheory.IsSeparator.{v₁, u₁} : {C : Type u₁} → [inst : Category.{v₁, u₁} C] → C → Prop :=
--   fun {C} [Category.{v₁, u₁} C] G ↦ IsSeparating {G}

#print CategoryTheory.IsSeparator.def
-- theorem CategoryTheory.IsSeparator.def.{v₁, u₁} : ∀ {C : Type u₁} [inst : Category.{v₁, u₁} C] (G : C),
--   IsSeparator G = IsSeparating {G} :=
-- fun {C} [Category.{v₁, u₁} C] G ↦ Eq.refl (IsSeparator G)

while the manually created theorem which currently needs renaming is

theorem IsSeparator.def' {G : C} :
    IsSeparator G   X Y : C (f g : X  Y), ( h : G  X, h  f = h  g)  f = g :=
  (isSeparator_def _).1

Mario Carneiro (Mar 17 2024 at 05:04):

Also, is there a reason these theorems can't be like foo._def? Isn't the leading underscore supposed to mean "reserved for the system"?

Mario Carneiro (Mar 17 2024 at 05:04):

i.e. we already solved this problem

github mathlib4 bot (Mar 17 2024 at 09:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 17 2024 at 11:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 17 2024 at 12:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 17 2024 at 16:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 17 2024 at 22:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 17 2024 at 22:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 17 2024 at 23:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 17 2024 at 23:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 18 2024 at 00:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 18 2024 at 01:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 18 2024 at 07:35):

Hmm... it succeeded earlier today, but the bot didn't post.

Kim Morrison (Mar 18 2024 at 07:40):

https://github.com/leanprover-community/mathlib4/actions/runs/8321208093/job/22767110964

Kim Morrison (Mar 18 2024 at 07:43):

#11469

Ruben Van de Velde (Mar 18 2024 at 07:48):

Should we rename the defs on master already or do we expect that core will allow them again?

Kim Morrison (Mar 18 2024 at 07:49):

I think core will allow them again, but probably not until next week.

Kim Morrison (Mar 18 2024 at 07:49):

Probably that means it is best to rename with a note for now, unfortunately, and then rename back later. :-(

github mathlib4 bot (Mar 18 2024 at 09:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Mar 18 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 18 2024 at 11:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 18 2024 at 12:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 18 2024 at 13:09):

Wow, this failed at "verify lake exe graph works". I guess it's good we added that to CI!

github mathlib4 bot (Mar 18 2024 at 13:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 18 2024 at 14:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 18 2024 at 15:07):

Needs a shake!

github mathlib4 bot (Mar 18 2024 at 16:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Thomas Murrills (Mar 18 2024 at 17:45):

We shook too hard! :shaking_face:

Thomas Murrills (Mar 18 2024 at 17:53):

Should Mathlib.Tactic.Relation.Rfl be in Mathlib.Tactic.Common? It doesn’t import any theory files, but also doesn’t define any tactic syntax itself.

Thomas Murrills (Mar 18 2024 at 17:58):

I put it there for now; I’ll record here that if we don’t want it there, the import should be moved to Mathlib.CategoryTheory.Category.Basic.

github mathlib4 bot (Mar 18 2024 at 19:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 18 2024 at 21:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 18 2024 at 23:09):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Mar 18 2024 at 23:51):

This then leaves us with a question:

  • #11437 (the adaptation PR for nightly-2024-03-16) is still open
  • nightly-testing now contains further changes (not compatible with nightly-2024-03-16), and builds against nightly-2024-03-18
  • Should we open a new PR from nightly-testing now, and have two such PRs in flight? Or just wait with these changes on nightly-testing (which will possibly break again with subsequent nightlies).

Kim Morrison (Mar 18 2024 at 23:53):

(Regarding my own priorities: I want to prioritize my work on adaptations towards getting nightly-testing working, as this is the critical step in enabling Lean CI to test against Mathlib, which in turn reduces the burden of subsequent adaptations. It's also the phase in which we learn what requests and bug reports need to be funnelled back to the FRO. But I'm hoping that to the extent possible the creation, review, and merging of the adaptation PRs to bump/v4.8.0 is shared.)

github mathlib4 bot (Mar 19 2024 at 01:21):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Johan Commelin (Mar 19 2024 at 04:32):

Scott Morrison opening a 2nd PR noe can't really hurt, right?

github mathlib4 bot (Mar 19 2024 at 04:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Yaël Dillies (Mar 19 2024 at 07:33):

Johan, wrong Scott!

Johan Commelin (Mar 19 2024 at 07:38):

Good catch! Anyway, Scott created the PR nonetheless :wink:

github mathlib4 bot (Mar 19 2024 at 10:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 19 2024 at 12:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Mar 19 2024 at 23:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 19 2024 at 23:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 20 2024 at 01:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 20 2024 at 03:02):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Mar 20 2024 at 18:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 20 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 01:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 04:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 06:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 10:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 18:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 22:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 21 2024 at 22:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 22 2024 at 00:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 22 2024 at 01:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 22 2024 at 02:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 22 2024 at 05:14):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Mar 22 2024 at 07:01):

#11579 is the PR to bump/v4.8.0 from this latest success.

Kim Morrison (Mar 22 2024 at 07:08):

Ah, most of the diff will disappear once #11576 (an Std bump) lands. It got stuck in CI.

github mathlib4 bot (Mar 22 2024 at 07:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 22 2024 at 08:05):

Scott Morrison said:

Ah, most of the diff will disappear once #11576 (an Std bump) lands. It got stuck in CI.

This should be trivial to review now.

github mathlib4 bot (Mar 22 2024 at 08:30):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Mar 22 2024 at 09:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 22 2024 at 09:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 22 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 22 2024 at 10:50):

Lots of new output from the new unused variables linter! These could all be backported to master.

Kevin Buzzard (Mar 22 2024 at 10:55):

Why did unused variables become a sin? I discovered that I use unused variables quite a lot in introductory teaching (e.g. teaching a proof of P -> (Q -> P) I do intro hP, intro hQ, exact hP and get a complaint that I didn't use hQ. I know! Who cares!)

Sébastien Gouëzel (Mar 22 2024 at 10:56):

If you know, just do intro _hQ so that your reader also knows.

Ruben Van de Velde (Mar 22 2024 at 10:58):

Generally in programming if you compute something that you don't need, either you can drop some unnecessary work in computing the thing, or you were meant to use it and forgot to. I guess neither applies as strongly in theorem proving

Ruben Van de Velde (Mar 22 2024 at 10:58):

I'll fix a few of the warnings now

Kim Morrison (Mar 22 2024 at 11:00):

(And an aside for those who are keeping track of these thing: the new unused variables linter is much faster, and I'm hoping there'll be a nontrivial change in total build time.)

Mario Carneiro (Mar 22 2024 at 11:06):

Ruben Van de Velde said:

Generally in programming if you compute something that you don't need, either you can drop some unnecessary work in computing the thing, or you were meant to use it and forgot to. I guess neither applies as strongly in theorem proving

The version of this that definitely does apply in theorem proving is that you made an unnecessary assumption and didn't use it, and probably you should drop it and strengthen the theorem

Mario Carneiro (Mar 22 2024 at 11:06):

Also unused have statements are an indication of unnecessary steps in a proof

Kim Morrison (Mar 22 2024 at 11:08):

(I really appreciate the unused have statements linter. I have found myself writing proofs recently where I saturate the context with plausible inputs for omega, and then clean up once omega says I'm done...)

Kevin Buzzard (Mar 22 2024 at 11:13):

I do this for exact? as well -- "what is likely to be useful? We have 0 < n, maybe I'll add n != 0" etc

Johan Commelin (Mar 22 2024 at 12:34):

Sounds like we need a saturate_context tactic

Ruben Van de Velde (Mar 22 2024 at 12:36):

#11583

github mathlib4 bot (Mar 22 2024 at 16:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Jireh Loreaux (Mar 22 2024 at 16:30):

Kevin, for teaching you could just add set_option linter.unusedVariables false at the top of the file, or even in the appropriate place in your lakefile (although I'm not sure exactly where that place is).

Damiano Testa (Mar 22 2024 at 17:24):

In the lakefile for my course, I have

package «mA4N1_2023» where
  -- add any package configuration options here
  moreServerArgs := #[ "-DautoImplicit=false" ]

so I imagine that an easy modification of this should work for unusedVariables.

github mathlib4 bot (Mar 22 2024 at 19:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Mar 22 2024 at 21:28):

#11594 has the rest of the unused variables

github mathlib4 bot (Mar 23 2024 at 00:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 23 2024 at 04:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 23 2024 at 07:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 23 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 23 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 23 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 23 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 23 2024 at 22:16):

Some upstreamed material needs removing, working on that now.

Kim Morrison (Mar 23 2024 at 22:23):

Unfortunately the upstreamed rw? is failing many of the tests in Mathlib. Will investigate.

Kim Morrison (Mar 23 2024 at 22:38):

These will require fixes upstream, and I've raised this with Joe.

For now I'm going to comment out some failing tests so we can keep moving... Expect regressions in rw? on nightly-testing!

Kim Morrison (Mar 23 2024 at 23:05):

Ah... and the changes to rw? in upstreaming have completely killed rw_search. Commented out the test suite for now, and will have to discuss with @Joe Hendrix on Monday.

Joe Hendrix (Mar 23 2024 at 23:58):

I'm traveling and so my ability to investigate is a bit limited, but there's an existing adaptation branch in lean-pr-testing-3719 that I think had working testing. Has that been merged in and found insufficient?

github mathlib4 bot (Mar 24 2024 at 00:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 24 2024 at 00:33):

Missed that one, thank you!

Kim Morrison (Mar 24 2024 at 00:41):

I've merged it, but still all the tests are failing.

Kim Morrison (Mar 24 2024 at 00:44):

Unfortunately I can't got back to lean#3719 itself, as it never had full-ci, so there's no macos toolchain.

github mathlib4 bot (Mar 24 2024 at 01:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 24 2024 at 02:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 24 2024 at 03:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 24 2024 at 10:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 24 2024 at 11:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 24 2024 at 12:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 24 2024 at 13:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 24 2024 at 15:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 24 2024 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 24 2024 at 21:11):

@Christian Merten, your changes from #11420 have caused breakages with the nightly. Is there any chance you would be able to checkout nightly-testing and see if you can see this fix quickly? I haven't looked yet past the error message.

Kim Morrison (Mar 24 2024 at 21:12):

(If you are able, feel free to just push changes direct to that branch.)

Kim Morrison (Mar 24 2024 at 21:13):

There was also a trivial-to-fix simp failure in EulerMascheroni, which I've just pushed a fix for.

Kim Morrison (Mar 24 2024 at 21:16):

Actually, @Christian Merten, it might be a trivial problem due to merge conflicgts.

Kim Morrison (Mar 24 2024 at 21:16):

Just checking out the master copy of MonCat/Limits into nightly-testing looks like it might work.

Kim Morrison (Mar 24 2024 at 21:17):

Scratch that, sorry.

Christian Merten (Mar 24 2024 at 21:17):

I think I have a fix, let me try.

github mathlib4 bot (Mar 24 2024 at 21:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Christian Merten (Mar 24 2024 at 21:25):

Worked for MonCat, just need to fix it for the rest.

github mathlib4 bot (Mar 24 2024 at 22:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 24 2024 at 22:31):

tests affected by unused variables or pretty printer changes

Kim Morrison (Mar 24 2024 at 22:35):

@Kyle Miller, there is a bad interaction between variable? and the new unused variables linter. For now I'm just commenting out the test in test/Variable.lean on nightly-testing: could I drop investigating that on you?

Joe Hendrix (Mar 24 2024 at 22:39):

Scott Morrison said:

I've merged it, but still all the tests are failing.

I am taking a look at resolving this today.

Kim Morrison (Mar 24 2024 at 22:41):

Thanks! Let me know if there's anything I can do to help.

I'm sorry, I didn't really anticipate when we first talked about upstreaming rw? that you might get caught up by rw_search failures ... :-(

github mathlib4 bot (Mar 24 2024 at 23:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Mar 26 2024 at 08:19):

Failures incoming from https://github.com/leanprover/lean4/pull/3767. :working_on_it:

github mathlib4 bot (Mar 26 2024 at 08:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 26 2024 at 11:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 26 2024 at 22:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 26 2024 at 22:42):

Sigh. This test failure (for rw_search) works locally for me. :-(

Kim Morrison (Mar 26 2024 at 22:44):

In CI it times out, locally it works with 200 heartbeats.

github mathlib4 bot (Mar 26 2024 at 22:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 27 2024 at 00:55):

This test looks like it is fixed in lean#3769, so should come good in a few hours.

github mathlib4 bot (Mar 27 2024 at 10:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 27 2024 at 11:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 27 2024 at 11:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 27 2024 at 11:54):

Okay, I'm out of time dealing with these rw? issues. This last one is my fault, a consequence of me messing with MVarId.refl and MVarId.applyRfl. I know what to do, but it may not happen until next week, so for now the failing test is just commented out.

github mathlib4 bot (Mar 27 2024 at 12:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 27 2024 at 21:53):

These failures are changes in the output of exact? on nightly-2024-03-27.

I think these changes are mostly for the worse, and we should try to remedy them.

Kim Morrison (Mar 27 2024 at 21:53):

@Joe Hendrix

Kim Morrison (Mar 27 2024 at 21:54):

Presumably these are changes in the order things come back from the DiscrTree in lean4#3769.

github mathlib4 bot (Mar 27 2024 at 22:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 27 2024 at 23:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Mar 27 2024 at 23:23):

Scott Morrison said:

These failures are changes in the output of exact? on nightly-2024-03-27.

I think these changes are mostly for the worse, and we should try to remedy them.

Oh, @Joe Hendrix, I forgot to mention this one when we just talked, but notice in that commit I had to double the heartbeat limit in test/observe.lean. This is one that Johan cares about a lot, as he often uses something close to this test file in Lean demo talks.

github mathlib4 bot (Mar 27 2024 at 23:47):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Mar 28 2024 at 06:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 28 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 28 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 28 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 28 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 28 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 29 2024 at 06:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 29 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 29 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 29 2024 at 12:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 29 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 29 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 30 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 30 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 30 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 30 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 30 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 30 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 31 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 31 2024 at 03:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 31 2024 at 10:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Mar 31 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 01 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 01 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 01 2024 at 12:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Joe Hendrix (Apr 01 2024 at 17:28):

Scott Morrison said:

These failures are changes in the output of exact? on nightly-2024-03-27.

I think these changes are mostly for the worse, and we should try to remedy them.

I have a PR lean4#3818 that appears to return results closer to the original order. There's some discussion there on the change. One downside is that with the revised order the rewrite_search test below fails:

/-
info: Try this: rw [← @add_assoc, @add_right_comm, @add_assoc, @add_add_add_comm, ← @add_assoc, @add_right_comm]
-/
#guard_msgs (drop info) in
example [AddCommMonoid α] {a b c d : α} : (a + b) + (c + d) = a + d + c + b := by
  rw_search

I've traced this test case and I think it's ok to break this test case. The edit distance heuristics don 't currently seem well suited to AC rewriting and so I think this is a pretty brittle test case. I haven't compared it with the original implementation though so maybe there's some heuristic that helps I am missing.

github mathlib4 bot (Apr 01 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 01 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 01 2024 at 22:48):

Quite a few things broken here. I will try to post a summary soon.

github mathlib4 bot (Apr 01 2024 at 23:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 02 2024 at 01:31):

Okay, I think we have a build (with sorries) incoming now. There appears to be a significant new performance problem, which we're going to have to track down.

github mathlib4 bot (Apr 02 2024 at 02:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 02 2024 at 03:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 02 2024 at 03:15):

Here are the current sorrys on nightly-testing. I would really appreciate help getting to the bottom of these. Some may just need a fix or work around, others may required a minimisation / identification of a regression in Lean.

I'll post each one separately so people can use emojis to claim and release items. I'll ping the authors of files, but please don't consider these as either demands, or exclusive locks. :-)

In any of these files, just search for FIXME nightly-testing to locate the problem.

Kim Morrison (Apr 02 2024 at 03:15):

  • Mathlib/AlgebraicGeometry/Pullbacks.lean: a type mismatch? @Andrew Yang?

Kim Morrison (Apr 02 2024 at 03:16):

  • Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean an @[ext] lemma no longer unifies. @Bhavik Mehta? @Markus Himmel?
  • Mathlib/CategoryTheory/Limits/Shapes/KernelPair.lean: similarly

Kim Morrison (Apr 02 2024 at 03:16):

  • Mathlib/CategoryTheory/Limits/Shapes/Pullbacks.lean: a convert that no longer goes through

Kim Morrison (Apr 02 2024 at 03:16):

  • Mathlib/CategoryTheory/Limits/Shapes/Products.lean: some proofs were previously done by aesop_cat in an autoparam, but now fail.

Kim Morrison (Apr 02 2024 at 03:16):

  • Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean: probably a broken simp

Kim Morrison (Apr 02 2024 at 03:16):

  • Mathlib/Data/Multiset/FinsetOps.lean: a proof that used to be rfl

Kim Morrison (Apr 02 2024 at 03:16):

  • Mathlib/Data/Polynomial/Basic.lean: an exact support_add that no longer works

Kim Morrison (Apr 02 2024 at 03:16):

  • test/notation3.lean: looks like some beta reductions are needed? @Mario Carneiro or @Kyle Miller?

Kim Morrison (Apr 02 2024 at 03:16):

  • test/Variable.lean: we're now getting an unused variable warning in variable?. @Kyle Miller?

Mario Carneiro (Apr 02 2024 at 03:17):

By the way, it would be good to summarize the upstream changes that are causing breakage in these threads

Mario Carneiro (Apr 02 2024 at 03:17):

(if you know what they are)

Kim Morrison (Apr 02 2024 at 03:17):

Yes: that's part of what we need to determine. For the problems above, I don't know yet.

Kim Morrison (Apr 02 2024 at 03:20):

There are also a lot of slow-downs requiring raising maxHeartbeats. There are all marked with Adaptation note: nightly-2024-04-01.

Hopefully these all have the same source, but again, I don't know yet what it is.

These problems occur in Algebra/Algebra/Operations, Algebra/Category/ModuleCat/ChangeOfRings, Algebra/Category/Ring/Limits, AlgebraicGeometry/GammaSpecAdjunction | Gluing | Spec, Combinatorics/SimpleGraph/Subgraph, Data/List/Intervals, FieldTheory/Extension | NormalClosure, LinearAlgebra/QuadraticForm/QuadraticModuleCat/Monoidal, Topology/ContinuousFunction/UniqueCFC, test/fun_prop2, and test/observe.

Kim Morrison (Apr 02 2024 at 03:25):

Oh, also rw_search is currently completely broken, but may be improved after https://github.com/leanprover/lean4/pull/3818. I haven't had a chance to test yet.

Kyle Miller (Apr 02 2024 at 03:25):

(AdjMatrix was pow_succ <-> pow_succ' in mathlib4#11451)

Kim Morrison (Apr 02 2024 at 03:26):

Great. I got quite a few of these, but apparently not all. :-)

Kim Morrison (Apr 02 2024 at 03:28):

The linter is also failing many times with synthInstance.maxHeartbeats problems; so I don't think we'll get a successful CI build until we sort that out.

Kim Morrison (Apr 02 2024 at 03:30):

The relevant nightly releases since we last had a build are:

I'm looking through these now for anything suspicious re: the above.

Kim Morrison (Apr 02 2024 at 03:32):

https://github.com/leanprover/lean4/pull/3807 landed during this period: it is meant to be a performance fix for isDefEq, but is so far the obvious suspect to slowdowns.

Kim Morrison (Apr 02 2024 at 03:34):

lean4#3816 is a possible cause for the unification failures in CategoryTheory.

Kim Morrison (Apr 02 2024 at 03:34):

Everything else in those nightlies looks pretty harmless to me.

Kyle Miller (Apr 02 2024 at 03:55):

test/notation3.lean was a good little puzzle — I completely forgot about the mathlib delaborator combinators

Mario Carneiro (Apr 02 2024 at 03:55):

what's breaking in them now?

Kyle Miller (Apr 02 2024 at 03:58):

It was just docs#Lean.PrettyPrinter.Delaborator.withBindingBodyUnusedName', but it took awhile to think to look at it.

Kyle Miller (Apr 02 2024 at 04:37):

@Mario Carneiro For variable?, do you know how to appease the unused variable linter here? It has unused_variables_ignore_fn, but I'm not sure that ever worked. Is there some hack we could use to cause the binders to be considered to be used?

Mario Carneiro (Apr 02 2024 at 04:37):

unused_variables_ignore_fn should be fixed on nightly

Mario Carneiro (Apr 02 2024 at 04:38):

IIRC the fix for that landed not long before the unused variables rewrite

Kyle Miller (Apr 02 2024 at 04:39):

Thanks, good to know. I think I found the problem, it's silly.

Kyle Miller (Apr 02 2024 at 04:40):

It had `Mathlib.Command.variable? instead of ``Mathlib.Command.Variable.variable?

Mario Carneiro (Apr 02 2024 at 04:40):

oops, where's our double backtick linter

github mathlib4 bot (Apr 02 2024 at 05:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 02 2024 at 05:55):

I am currently working on a minimisation of some of the timeouts.

Kyle Miller (Apr 02 2024 at 06:06):

Mathlib/CategoryTheory/Limits/Shapes/Pullbacks.lean looks like it could be from a change to the defeq algorithm? I had to insert a dsimp to get some types to unify.

github mathlib4 bot (Apr 02 2024 at 06:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 02 2024 at 09:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 02 2024 at 09:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 02 2024 at 09:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 02 2024 at 09:50):

Could someone (@Eric Wieser?) please update quote4 to run on nightly-2024-04-02? It has a <- ... that (foot-gun!) always lifts out of an if, and as of nightly-2024-04-02 this is an error.

Kim Morrison (Apr 02 2024 at 09:50):

The error is in Match.lean, in makeMatchCode.

Kim Morrison (Apr 02 2024 at 09:53):

For anyone who would like to continue working on nightly-testing, I've made the branch nightly-testing-2024-04-01-WIP before nightly-testing moved to nightly-2024-04-02. It should still be possible to work on that until quote4 is fixed. nightly-testing itself is not viable until then.

(Edit: nightly-testing is more or less working again, so this has become irrelevant.)

Kim Morrison (Apr 02 2024 at 09:56):

(Also pinging @Gabriel Ebner in case they are available to fix quote4 problems.)

Mario Carneiro (Apr 02 2024 at 10:50):

I have merge rights if you want to send a PR

Kim Morrison (Apr 02 2024 at 11:00):

I have merge rights too, I'm just not excited about debugging quote4. :-)

Eric Wieser (Apr 02 2024 at 11:00):

Which line is the error on?

Kim Morrison (Apr 02 2024 at 11:01):

114

Kim Morrison (Apr 02 2024 at 11:01):

sorry, the real error is 115

Kim Morrison (Apr 02 2024 at 11:01):

the <- is not allowed in that position anymore, because it will always lift outside the if

Eric Wieser (Apr 02 2024 at 11:04):

I don't think that linter really makes sense here; "inside the if" is at runtime, and outside the if is at generation time

Eric Wieser (Apr 02 2024 at 11:04):

That is, the $() should be protecting the <-

Eric Wieser (Apr 02 2024 at 11:05):

So in summary: this is an easy workaround in Qq (lifting the expression outside manually), but core should not be complaining here

Mario Carneiro (Apr 02 2024 at 11:08):

there is a TODO in the core PR about this

Mario Carneiro (Apr 02 2024 at 11:08):

the current workaround is to just lift it manually

Mario Carneiro (Apr 02 2024 at 11:10):

I remember finding this in mathport even before this PR because of `(do $(<- trExpr)) stuff

Mario Carneiro (Apr 02 2024 at 11:10):

which does something... very strange IIRC

Kim Morrison (Apr 02 2024 at 11:18):

@Eric Wieser, could you please push the workaround?

github mathlib4 bot (Apr 02 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 02 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 02 2024 at 18:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Eric Wieser (Apr 02 2024 at 20:06):

Mario Carneiro said:

I remember finding this in mathport even before this PR because of `(do $(<- trExpr)) stuff

Is there a tracking issue for this?

a mwe is:

import Lean
open Lean

def foo : MetaM (TSyntax ``Parser.Term.doSeq) := do `(Parser.Term.doSeq| pure 37)

-- fails
#check do `(do $( foo))

-- ok
#check do
  let mkDo x := `(do $x)
  mkDo ( foo)

Eric Wieser (Apr 02 2024 at 20:14):

Filed as lean4#3827

Eric Wieser (Apr 02 2024 at 20:27):

Scott Morrison said:

Eric Wieser, could you please push the workaround?

Pushed in https://github.com/leanprover-community/quote4/pull/41; can you check that branch works on the latest lean?

Kim Morrison (Apr 02 2024 at 22:42):

Checked and merged.

github mathlib4 bot (Apr 02 2024 at 23:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 03 2024 at 01:09):

Okay, we are making good progress. We are now down to:

Kim Morrison (Apr 03 2024 at 01:09):

  • AlgebraicGeometry/Pullbacks is failing in multiple places, almost surely because of the defeq abuse throughout AG interacting with the latest change to isDefEq.

Kim Morrison (Apr 03 2024 at 01:09):

  • the rw_search tests are all broken, but hopefully mostly fixed in lean4#3818, which will land tonight

Kim Morrison (Apr 03 2024 at 01:09):

  • there are still some slowdowns, but I've fixed the terrible ones. I'm not inclined to treat these as blockers.

Kim Morrison (Apr 03 2024 at 01:11):

Note that I'm now hoping that nightly-2024-04-04 can become v4.8.0-rc1, so deciding to leave these slowdowns in means that will be part of life for the next month.

Kim Morrison (Apr 03 2024 at 01:18):

@Andrew Yang, if you have any availability to look at def openCoverOfBase' in Mathlib/AlgebraicGeometry/Pullbacks.lean on the nightly-testing branch, that would be extremely helpful. I'm starting to look at it otherwise.

Kim Morrison (Apr 03 2024 at 01:32):

Ah, maybe have it sorted.

github mathlib4 bot (Apr 03 2024 at 02:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 03 2024 at 03:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 03 2024 at 04:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Andrew Yang (Apr 03 2024 at 04:51):

Scott Morrison said:

Andrew Yang, if you have any availability to look at def openCoverOfBase' in Mathlib/AlgebraicGeometry/Pullbacks.lean on the nightly-testing branch, that would be extremely helpful. I'm starting to look at it otherwise.

Is this sorted out?

Kim Morrison (Apr 03 2024 at 05:59):

Yes, it is, thank you!

github mathlib4 bot (Apr 03 2024 at 10:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 03 2024 at 11:43):

Getting closer.

Remaining issues are

  • rw_search completely broken, despite working on lean-pr-testing-3818 (and that having been merged)
  • needing to minimize at least one of the new slowdowns. I have partial progress on that locally, but will need to keep working on that tomorrow.

github mathlib4 bot (Apr 03 2024 at 13:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 03 2024 at 16:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 03 2024 at 19:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 03 2024 at 22:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 03 2024 at 22:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 04 2024 at 01:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 04 2024 at 03:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 04 2024 at 05:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Apr 04 2024 at 05:46):

Finally!

Kim Morrison (Apr 04 2024 at 05:47):

However, still working on minimization of the timeouts.

Kim Morrison (Apr 04 2024 at 05:47):

Nevertheless, I will put up a PR so others can review the changes so far, with the understanding that our intention is to fix the timeouts before v4.8.0-rc1 (unless we don't. :-)

github mathlib4 bot (Apr 04 2024 at 11:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 04 2024 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 04 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 04 2024 at 17:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 04 2024 at 19:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 04 2024 at 20:30):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 04 2024 at 22:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 01:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 04:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 05:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 05 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 10:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 12:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 19:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 21:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 05 2024 at 21:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 00:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 01:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 02:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kyle Miller (Apr 06 2024 at 02:35):

A norm_num "regression" is that this fails now:

import Mathlib.Tactic.NormNum.Basic

example (h : 4 = 2) : False := by
  norm_num at h

A fix is to make sure Mathlib.Tactic.NormNum is imported. (In particular, import Mathlib.Tactic.NormNum.Eq)

Kyle Miller (Apr 06 2024 at 02:37):

There are some shake errors I'm not sure how to handle correctly, and there's a simpNF linter error I'm not sure how to debug.

github mathlib4 bot (Apr 06 2024 at 03:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 03:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 04:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 10:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 12:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 15:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 18:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 06 2024 at 19:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Joe Hendrix (Apr 06 2024 at 21:32):

Kyle Miller said:

A norm_num "regression" is that this fails now:

import Mathlib.Tactic.NormNum.Basic

example (h : 4 = 2) : False := by
  norm_num at h

A fix is to make sure Mathlib.Tactic.NormNum is imported. (In particular, import Mathlib.Tactic.NormNum.Eq)

On norm_num implementation side, I've noticed that norm_num appears to be using the simplifer with simp lemmas, but not simprocs.

That's not surprising given the age of norm num and recent additions of simprocs, and norm num appears to have its own version of simprocs such as the one for equality solving this.

I think your approach of making sure import Mathlib.Tactic.NormNum.Eq is in scope is a good one. A larger fix would be to support Lean core simprocs so norm_num's use of simp matches the simp elaborator. I don't anticipate needing to remove any additional successor simplification lemmas though.

There's also the possibility of Mathlib adding @[simp] back to the two lemmas that had removed it (see below), however simp will resume its old behavior which leads to timeouts on even moderately large Nat literals. I wouldn't personally recommend this.

attribute [simp] Nat.succ.injEq Nat.succ_sub_succ_eq_sub

github mathlib4 bot (Apr 06 2024 at 22:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Notification Bot (Apr 06 2024 at 22:18):

7 messages were moved from this topic to #mathlib4 > norm_num vs simprocs by Eric Wieser.

Eric Wieser (Apr 06 2024 at 22:19):

I agree that ensuring import Mathlib.Tactic.NormNum.Eq is present is a totally reasonable fix

github mathlib4 bot (Apr 06 2024 at 23:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 01:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 06:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 08:16):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 07 2024 at 09:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 10:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 10:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 12:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 15:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 18:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 19:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 20:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 07 2024 at 23:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 08 2024 at 03:07):

Looks like it succeeded in CI, not sure why the bot didn't post.

github mathlib4 bot (Apr 08 2024 at 04:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 06:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 18:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 19:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 21:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 08 2024 at 22:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 08 2024 at 22:53):

It got as far as the counterexamples now, with what looks like an easy fix

github mathlib4 bot (Apr 09 2024 at 01:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 09 2024 at 07:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 09 2024 at 08:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Ruben Van de Velde (Apr 09 2024 at 08:22):

Going to look why the bot doesn't work

Ruben Van de Velde (Apr 09 2024 at 08:27):

Oh, "Update the nightly-testing-YYYY-MM-DD branch" is failing

github mathlib4 bot (Apr 09 2024 at 08:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Ruben Van de Velde (Apr 09 2024 at 09:06):

#11856 broke it

Ruben Van de Velde (Apr 09 2024 at 09:15):

(I'll try to debug a little)

github mathlib4 bot (Apr 09 2024 at 09:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 09 2024 at 10:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 09 2024 at 12:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 12 2024 at 13:26):

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-12 branch from nightly-testing, and then PR that to "bump/v4.8.0".

github mathlib4 bot (Apr 12 2024 at 16:50):

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-12 branch from nightly-testing, and then PR that to "bump/v4.8.0".

github mathlib4 bot (Apr 12 2024 at 19:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 12 2024 at 22:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 13 2024 at 00:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 13 2024 at 07:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 13 2024 at 11:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 13 2024 at 12:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 13 2024 at 15:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 13 2024 at 18:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 13 2024 at 21:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 14 2024 at 07:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 14 2024 at 10:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 14 2024 at 14:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 14 2024 at 16:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 14 2024 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 14 2024 at 21:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kyle Miller (Apr 15 2024 at 02:23):

Fixed, but depends on unmerged aesop#123.

Kyle Miller (Apr 15 2024 at 02:26):

There are a couple erws I had to include (marked them with adaptation notes). I don't understand exactly why, but they seem to have to do with List.map_pmap being applied in ways where pmap has to be unfolded.

Kyle Miller (Apr 15 2024 at 02:26):

Also, the lake-manifest had three copies of std4, and I pruned it.

github mathlib4 bot (Apr 15 2024 at 02:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kyle Miller (Apr 15 2024 at 02:30):

I'm very surprised that the changes to rcases/obtain (to make it so for Nat, you get 0 and n + 1 instead of Nat.zero and Nat.succ n') didn't have much fallout. It's possible that there are many uses of simp only [Nat.succ_eq_add_one, ...] that I didn't clean up.

github mathlib4 bot (Apr 15 2024 at 04:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 15 2024 at 06:00):

Aesop bump was required.

github mathlib4 bot (Apr 15 2024 at 07:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 15 2024 at 08:59):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 15 2024 at 08:59):

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-14 branch from nightly-testing, and then PR that to "bump/v4.8.0".

Kim Morrison (Apr 15 2024 at 09:50):

Well, we need to decide what to do with #11997 first. It still contains regressions from IsDefEq changes. I have a few local fixes that I will push to that branch (and thence to nightly-testing) soon, but far from all of them.

Kim Morrison (Apr 15 2024 at 09:50):

Any preferences from Mathlib maintainers how we handle this? Merge the regressions into bump/v4.8.0, to reduce the pain of keeping nightly-testing alive? Or not merge until we make further progress on these.

Kim Morrison (Apr 15 2024 at 09:52):

These regressions are blocking v4.8.0-rc1, so we do need to make progress here.

Enough of the timeouts reveal Mathlib over-using defeq that we can't just say "its lean4#3807's fault"...

Ruben Van de Velde (Apr 15 2024 at 10:02):

Unfortunately it's so big that it's pretty much unreviewable, and it seems we can't merge master into bump/v4.8.0 because master has already restored .def lemmas and bump/v4.8.0 doesn't support them.

How would you feel about this as a strategy to reduce the diff:

  • merge #12097 into bump/v4.8.0 so that it at least builds
  • I fix the conflicts on #11828 and #11829, we merge those into master, and cherry-pick them into bump/v4.8.0
  • review the remaining diff in #11997 to see if we can apply that treatment to any other changes

and then I think we really do need to merge #11997 and make sure any remaining problems have issues filed

Kim Morrison (Apr 15 2024 at 10:21):

Great!

Kim Morrison (Apr 15 2024 at 10:22):

I am looking at #12097 now, hopefully merging soon.

Kim Morrison (Apr 15 2024 at 10:23):

@Ruben Van de Velde, the two FIXMEs on #12097 are going to resolve themselves on nightly-testing, because they are explaining how the proofs will break again, right?

Kim Morrison (Apr 15 2024 at 10:28):

:merge:'d #12097 into bump/v4.8.0

Kim Morrison (Apr 15 2024 at 10:30):

And I've merged master and optimistically resolved conflicts on both #11828 and #11829.

Ruben Van de Velde (Apr 15 2024 at 10:38):

Kim Morrison said:

Ruben Van de Velde, the two FIXMEs on #12097 are going to resolve themselves on nightly-testing, because they are explaining how the proofs will break again, right?

Yes, exactly

Ruben Van de Velde (Apr 15 2024 at 10:38):

Thanks!

Kim Morrison (Apr 15 2024 at 11:05):

Okay, I see #11828 has been closed (not much diff left). I've :peace_sign:'d #11829, but may need to go to bed before CI is finished: feel free to merge as soon as it is good.

Kim Morrison (Apr 15 2024 at 11:08):

Also, once it lands on master if you want to cherry-pick it over to bump/v4.8.0 that would be great. Otherwise I'll resume tomorrow.

github mathlib4 bot (Apr 15 2024 at 11:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Eric Wieser (Apr 15 2024 at 12:41):

it seems we can't merge master into bump/v4.8.0 because master has already restored .def lemmas and bump/v4.8.0 doesn't support them.

What do you mean by this?

github mathlib4 bot (Apr 15 2024 at 12:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Eric Wieser (Apr 15 2024 at 12:43):

Also, how does this thread differ from #nightly-testing > Mathlib status updates (plural)?

github mathlib4 bot (Apr 15 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 15 2024 at 15:45):

Kim Morrison said:

Also, once it lands on master if you want to cherry-pick it over to bump/v4.8.0 that would be great. Otherwise I'll resume tomorrow.

#12158 for the cherry-pick; I can't push to the bump branch directly

Ruben Van de Velde (Apr 15 2024 at 15:47):

Eric Wieser said:

it seems we can't merge master into bump/v4.8.0 because master has already restored .def lemmas and bump/v4.8.0 doesn't support them.

What do you mean by this?

bump/v4.8.0 is currently on a nightly that doesn't allow definitions called Foo.def (e.g. IsRoot.def). We renamed those on master, but apparently we renamed them back as well

github mathlib4 bot (Apr 15 2024 at 18:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 15 2024 at 21:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 15 2024 at 21:54):

Eric Wieser said:

Also, how does this thread differ from #nightly-testing > Mathlib status updates (plural)?

There are two different bots, that apparently disagree on the name...

Kim Morrison (Apr 15 2024 at 21:55):

PR'd and bors'd in #12165.

Kim Morrison (Apr 15 2024 at 21:57):

Also, I've just merged the streams.

Kim Morrison (Apr 15 2024 at 21:58):

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Not sure what happened here, CI is marked as cancelled.

Kim Morrison (Apr 15 2024 at 22:00):

Kim Morrison said:

Also, once it lands on master if you want to cherry-pick it over to bump/v4.8.0 that would be great. Otherwise I'll resume tomorrow.

Okay, I've cherry-picked b8a0f589c3ef08ae093d7d1896142e5eb05e599a, which had been "chore: avoid id.def (adaptation for nightly-2024-03-27) #11829" onto bump/v4.8.0.

Kim Morrison (Apr 15 2024 at 22:03):

The diff for #11997 (the PR to bump/v4.8.0 bringing us to 04-07) is now slightly smaller, but still substantial: 270 files.

I need to take a break for about an hour, but will get back to this then. I think reducing / reviewing / approving the remaining diff is the main work at the moment for nightly-testing.

github mathlib4 bot (Apr 15 2024 at 22:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kyle Miller (Apr 15 2024 at 22:25):

Oops, I didn't know about the bump branch. I got nightly-testing building though, hopefully there's little accidental duplicated effort.

github mathlib4 bot (Apr 15 2024 at 22:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 15 2024 at 22:27):

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-14 branch from nightly-testing, and then PR that to "bump/v4.8.0".

github mathlib4 bot (Apr 16 2024 at 01:14):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 16 2024 at 01:14):

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-14 branch from nightly-testing, and then PR that to "bump/v4.8.0".

Joachim Breitner (Apr 16 2024 at 07:01):

Quite noisy bot…

BTW, have you considered doing only one master -> nightly-testing merge per day, maybe 12h after the tool chain bump?

More time to focus on getting it to work without bots interfering, less noise on the branch and here, at the cost of having a slightly worse time when a commit on master broke it and you need to find which one.

github mathlib4 bot (Apr 16 2024 at 07:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 16 2024 at 07:27):

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-14 branch from nightly-testing, and then PR that to "bump/v4.8.0".

Kim Morrison (Apr 16 2024 at 07:32):

Ah, the two bots are now interacting in a bad way. The success bot knows to not say anything if it was the last person to speak. The PR reminder bot gets it in the way, because it always speaks... Sad. Ideally the reminder bot would only post once.

Kim Morrison (Apr 16 2024 at 07:37):

Okay, I've just made #12176, which backports a bunch more changes to master. If someone is available to quickly review and merge that, that would be great. Once it lands on master we can cherry-pick it to bump/v4.8.0.

Kim Morrison (Apr 16 2024 at 07:39):

github mathlib4 bot said:

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-14 branch from nightly-testing, and then PR that to "bump/v4.8.0".

I guess I will just obey the bot, it is making a reasonable suggestion!

Kim Morrison (Apr 16 2024 at 07:43):

Hmm, I made a bump/nightly-2024-04-14 branch from nightly-testing, but it is completely unreviewable as a PR to bump/v4.8.0 until we are able to merge master to bump/v4.8.0 again, i.e. after getting #11997 in.

Markus Himmel (Apr 16 2024 at 07:45):

Kim Morrison said:

Okay, I've just made #12176, which backports a bunch more changes to master. If someone is available to quickly review and merge that, that would be great. Once it lands on master we can cherry-pick it to bump/v4.8.0.

Maybe I'm misunderstanding the diff that GitHub is showing me, but it seems to be that the PR is partially reverting some recent commits to mathlib.

Kim Morrison (Apr 16 2024 at 07:55):

Sorry, I completely botched it. Trying again now. :-(

Eric Wieser (Apr 16 2024 at 08:11):

Kim Morrison said:

Ah, the two bots are now interacting in a bad way. The success bot knows to not say anything if it was the last person to speak. The PR reminder bot gets it in the way, because it always speaks... Sad. Ideally the reminder bot would only post once.

Perhaps two threads is reasonable after all? One could be "Mathlib bump branch reminders" or something

Ruben Van de Velde (Apr 16 2024 at 08:33):

There was a simp? says failure in #12176, I just removed the says since it doesn't seem useful

Ruben Van de Velde (Apr 16 2024 at 08:35):

I had also started doing the same; I'll make a PR once this is in

Ruben Van de Velde (Apr 16 2024 at 09:31):

#12176 is green, if anyone can merge it

github mathlib4 bot (Apr 16 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 16 2024 at 10:52):

Kim Morrison said:

Sorry, I completely botched it. Trying again now. :-(

Okay, I've had another go at #12176. Could someone review it please?

Ruben Van de Velde (Apr 16 2024 at 11:05):

Oh, why? It was on the bors queue

Kim Morrison (Apr 16 2024 at 11:06):

Oops, sorry, I should have checked the comments. Not having a great day today, it seems. I backported more id.def --> id or _root_.id replacements as well.

Kim Morrison (Apr 16 2024 at 11:06):

I'll put it back on the queue.

github mathlib4 bot (Apr 16 2024 at 12:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 16 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 16 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 17 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 17 2024 at 02:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 17 2024 at 03:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 17 2024 at 03:29):

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-16 branch from nightly-testing, and then PR that to "bump/v4.8.0".

github mathlib4 bot (Apr 17 2024 at 04:35):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 17 2024 at 04:36):

:working_on_it:: it looks like it's time to create a new bump/nightly-2024-04-16 branch from nightly-testing, and then PR that to "bump/v4.8.0".

github mathlib4 bot (Apr 17 2024 at 08:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 17 2024 at 09:16):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 17 2024 at 13:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 17 2024 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 17 2024 at 18:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 17 2024 at 21:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 18 2024 at 00:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 18 2024 at 02:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 18 2024 at 10:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 18 2024 at 13:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 18 2024 at 16:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 18 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 18 2024 at 22:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 01:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 04:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 05:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 07:02):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 19 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 10:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 10:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 19 2024 at 12:00):

(It turns out we use a lot of autogenerated instance names)

github mathlib4 bot (Apr 19 2024 at 12:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 12:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 19 2024 at 13:26):

Oh, neat, rw? no longer inserts @ everywhere

github mathlib4 bot (Apr 19 2024 at 13:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 19 2024 at 14:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 20 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 20 2024 at 07:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 20 2024 at 09:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kyle Miller (Apr 20 2024 at 16:11):

Ruben Van de Velde said:

(It turns out we use a lot of autogenerated instance names)

I was really confused about how there were still instance names to fix, since I made sure to have a mathlib bump PR, but it turns out that there were still some old instance names hiding out inside of Init that didn't get updated until Lean's stage0 was updated.

github mathlib4 bot (Apr 21 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 21 2024 at 23:56):

Just needed a lake update after fixing Std.

github mathlib4 bot (Apr 22 2024 at 00:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 22 2024 at 00:55):

More fallout from lean4#3960.

Kim Morrison (Apr 22 2024 at 01:06):

@Mario Carneiro, I pushed an icky fix to UInt8.toChar in Mathlib/Data/UInt.lean on nightly-testing, to adapt to your lean4#3960. Would you mind taking a look and pushing a better proof if appropriate?

github mathlib4 bot (Apr 22 2024 at 01:35):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Apr 22 2024 at 10:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 22 2024 at 10:40):

First step is to merge the lean-pr-testing-3951 branches to Std/Aesop/Mathlib

Kim Morrison (Apr 22 2024 at 10:44):

@Mac Malone, lake update on nightly-testing is persistently duplicating entries in lake-manifest.json. Could you take a look?

Ruben Van de Velde (Apr 22 2024 at 10:44):

@Kim Morrison sorry, I already pushed fixes to the two errors in the log, but it seems like lean-pr-testing-3951 doesn't have code changes in mathlib?

Kim Morrison (Apr 22 2024 at 10:45):

I think all it has it changes to the lakefile, to use the lean-pr-testing-3951 branches in Std and Aesop

Kim Morrison (Apr 22 2024 at 10:45):

I've just merged those back into nightly-testing.

Ruben Van de Velde (Apr 22 2024 at 10:48):

Oh right, std and mathlib build in parallel, so seeing errors in mathlib doesn't prove that all of std works

Kim Morrison (Apr 22 2024 at 10:48):

Oh, crap! lean4#3951 didn't actually make it into this nightly...

Kim Morrison (Apr 22 2024 at 10:49):

It missed by just a bit.

Kim Morrison (Apr 22 2024 at 10:49):

hmm.

Kim Morrison (Apr 22 2024 at 10:49):

No big deal, I think I unwound it okay.

Kim Morrison (Apr 22 2024 at 10:52):

But there are real errors on nightly-testing, presumably because of the latest IsDefEq changes!

Ruben Van de Velde (Apr 22 2024 at 10:53):

I wonder if we should expect things like this to work

Error: ././././Mathlib/Order/CompleteLatticeIntervals.lean:253:38: error: invalid constructor ...⟩, expected type must be an inductive type
  ?m.31195 c'
Error: ././././Mathlib/Order/CompleteLatticeIntervals.lean:255:36: error: application type mismatch
  And.intro b.property
argument
  b.property
has type
  b  Iic a : Prop
but is expected to have type
  ?m.32594  ?m.32595 : Prop

Kim Morrison (Apr 22 2024 at 11:04):

Hmmm, I haven't worked out CompleteLatticeIntevals yet, but there are various problems with Lean no longer being able to infer a _...

Kim Morrison (Apr 22 2024 at 11:11):

Ah, got CompleteLatticeIntervals.

Kim Morrison (Apr 22 2024 at 11:11):

It just needs two (α := α).

Kim Morrison (Apr 22 2024 at 11:13):

Oh, curious, weird interaction of named arguments and dot notation, you can write f (x :=y).h and it is interpreted as (f (x := y)).h.

Kim Morrison (Apr 22 2024 at 11:42):

I am pausing for a bit. If anyone would like to pick up nightly-testing, there are currently errors in

  • Mathlib/Algebra/Module/LinearMap/Basic.lean
  • Mathlib/GroupTheory/CoprodI.lean
  • Mathlib/Order/RelSeries.lean

Kim Morrison (Apr 22 2024 at 11:43):

It seems Lean has got a bit worse at guessing some implicit arguments, but I don't yet understand any pattern in the regressions so far...

github mathlib4 bot (Apr 22 2024 at 11:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 22 2024 at 12:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 22 2024 at 13:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 22 2024 at 14:09):

Kim Morrison said:

It seems Lean has got a bit worse at guessing some implicit arguments, but I don't yet understand any pattern in the regressions so far...

I think these are going to count as bug reports for Lean, so perhaps for now there is not much need to keep pushing nightly-testing forward, but rather to create minimizations of the regressions that I've already pushed to nightly-testing.

Kim Morrison (Apr 22 2024 at 14:09):

It's late here, but these will be my plan tomorrow!

github mathlib4 bot (Apr 23 2024 at 05:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 05:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 06:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 07:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 09:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 10:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 12:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 18:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 23 2024 at 18:58):

aesop is failing cc @Kyle Miller

Error: ././.lake/packages/aesop/././Aesop/Util/Basic.lean:367:7: error: invalid field 'isEmpty', the environment does not contain 'Lean.MessageData.isEmpty'

Kyle Miller (Apr 23 2024 at 19:44):

@Joachim Breitner removed MessageData.isEmpty in lean4#3951

Damiano Testa (Apr 23 2024 at 19:46):

Oh, I think that the have vs let linter also uses it.

Joachim Breitner (Apr 23 2024 at 20:14):

There should be lean-pr-testing-3951 branches around, though

github mathlib4 bot (Apr 23 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 23 2024 at 22:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 23 2024 at 22:26):

I've just undone some changes on nightly-testing that were needed to cope with lean4#3965, as we're hoping that lean4#3977 arriving tonight will obviate the need for them. nightly-testing will remain broken in the meantime, however.

Kim Morrison (Apr 23 2024 at 22:29):

Joachim Breitner said:

There should be lean-pr-testing-3951 branches around, though

Merged into aesop's nightly-testing, and bumped Mathlib's nightly-testing

github mathlib4 bot (Apr 23 2024 at 22:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 00:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 03:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 04:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 06:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 06:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 09:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 24 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 25 2024 at 03:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 25 2024 at 06:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 25 2024 at 07:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 25 2024 at 07:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 25 2024 at 08:02):

Waiting for someone to fix Std, I guess

github mathlib4 bot (Apr 25 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 25 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 25 2024 at 15:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 25 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 26 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 26 2024 at 12:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 26 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 26 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 26 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 06:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 09:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 10:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 11:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 27 2024 at 11:49):

A short update: lots of stuff is bad on nightly-testing still: the recent changes to IsDefEq in lean4#3965 and lean4#3977 have being playing tug-of-war with Mathlib, and there are still lots of slow-downs. Leo still has one more fix in the works that hasn't hit the lean4 repo. Being extremely optimistic, this will fix everything.

Pessimistically, we have a ways to go and need to do more minimization of the issues on nightly-testing.

If anyone wants to have a look for either Adaptation note: 2024-04-23 or FIXME: nightly-testing on the nightly-testing branch, and at any of those occurrences, try to minimize what's going on, that would be amazing. This is my plan tomorrow/Monday...

github mathlib4 bot (Apr 27 2024 at 11:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 12:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 27 2024 at 13:15):

I'll take a look now if I can get anywhere

github mathlib4 bot (Apr 27 2024 at 13:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 13:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 14:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 27 2024 at 14:12):

I opened #12466 to backport clear defeq abuse fixes; feel free to review or push similar fixes to it

github mathlib4 bot (Apr 27 2024 at 14:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 27 2024 at 14:19):

Stepping away for a bit

github mathlib4 bot (Apr 27 2024 at 14:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 16:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 17:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 19:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 27 2024 at 19:18):

I'll apply @Kevin Buzzard's changed from #12469 to nightly-testing

github mathlib4 bot (Apr 27 2024 at 19:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 19:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 19:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 20:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 27 2024 at 20:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 27 2024 at 20:12):

Okay, mathlib builds. Thanks @Kevin Buzzard for the clue!

Kevin Buzzard (Apr 27 2024 at 20:15):

You can thank the gods of chance! Or the guy who asked the community to look at GammaSpecAdjunction :-)

Ruben Van de Velde (Apr 27 2024 at 20:15):

:dice:

github mathlib4 bot (Apr 27 2024 at 20:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Apr 27 2024 at 20:48):

Linter issues and some unused imports if someone wants to look at them

github mathlib4 bot (Apr 27 2024 at 22:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 28 2024 at 00:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 28 2024 at 01:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Apr 28 2024 at 05:55):

This "success" still contains some sorrys, and many "adaptation note"s about significant slowdowns! We're not quite there yet. But it's progress!

github mathlib4 bot (Apr 28 2024 at 06:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 28 2024 at 06:34):

I've intentionally borked nightly-testing for the next ~2-3 hours, by starting to compile it against lean4#4008.

github mathlib4 bot (Apr 28 2024 at 07:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 28 2024 at 07:13):

@Ruben Van de Velde, I saw on nightly-testing in Mathlib/AlgebraicGeometry/FunctionField.lean you added

-- Adaptation note: 2024-04-23

but with no further text. Could you make sure that adaptation notes include some explanation of what changed, so that it's not necessary to look at the git history to understand what happened?

Kim Morrison (Apr 28 2024 at 07:18):

Similarly in AlgebraicGeometry/Properties and MeasureTheory/Covering/Differentation

github mathlib4 bot (Apr 28 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Michael Stoll (Apr 28 2024 at 10:21):

It looks like the new option is not visible in (some files in) Mathlib?

github mathlib4 bot (Apr 28 2024 at 10:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 28 2024 at 10:59):

Michael Stoll said:

It looks like the new option is not visible in (some files in) Mathlib?

Should be momentarily: I was pushing to nightly-testing use a local overriden toolchain.

github mathlib4 bot (Apr 28 2024 at 12:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Michael Stoll (Apr 28 2024 at 13:10):

Looks like rw [Ne.def, ...] causes a problem here? (In Mathlib.Data.Nat.Factors: replicate_subperm_factors_iff, which is pretty recent... @Ruben Van de Velde )

Ruben Van de Velde (Apr 28 2024 at 13:10):

Please replace by rw [Ne, ...

Michael Stoll (Apr 28 2024 at 13:18):

This seems to be working. Can I push to this branch?

Michael Stoll (Apr 28 2024 at 13:23):

Mathlib.CategoryTheory.Iso has a problem as well, but the only message I see is

error: external command `/home/mstoll/.elan/toolchains/leanprover--lean4---nightly-2024-04-28/bin/lean` exited with code 139

Michael Stoll (Apr 28 2024 at 13:27):

Michael Stoll said:

This seems to be working. Can I push to this branch?

Or should somebody make a PR to Mathlib fixing this? (It seems to be the only Ne.def in Mathlib.)

Ruben Van de Velde (Apr 28 2024 at 13:29):

Go ahead and push to nightly-testing

Michael Stoll (Apr 28 2024 at 13:33):

Done. Should I also make a PR to Mathlib? (Once the build finishes...)

Ruben Van de Velde (Apr 28 2024 at 13:39):

You can, but it's not really needed

Michael Stoll (Apr 28 2024 at 13:40):

Then I won't.

github mathlib4 bot (Apr 28 2024 at 13:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Michael Stoll (Apr 28 2024 at 13:55):

Michael Stoll said:

Mathlib.CategoryTheory.Iso has a problem as well, but the only message I see is

error: external command `/home/mstoll/.elan/toolchains/leanprover--lean4---nightly-2024-04-28/bin/lean` exited with code 139

The strange thing is that when looking at this file in VSCode, it compiles without problems.

Michael Stoll (Apr 28 2024 at 14:07):

I've had a look at Mathlib.NumberTheory.RamificationInertia (the file I was experimenting with in #12412). Replacing two _s by explicit arguments makes the two declarations that had become very slow fairly fast. (I had already done that in #12412.)

I see that most of the slow Subsingleton instances are gone (with one exception), but Module, AddCommMonoid and AddMonoidHomClass are still often slow.

Michael Stoll (Apr 28 2024 at 14:08):

Overall, it looks like typeclass inference only takes 50% of the time it took before lean4#4003.

Michael Stoll (Apr 28 2024 at 14:09):

Michael Stoll said:

exited with code 139

What is the meaning of this error code?

github mathlib4 bot (Apr 28 2024 at 14:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Michael Stoll (Apr 28 2024 at 14:35):

Michael Stoll said:

Michael Stoll said:

exited with code 139

What is the meaning of this error code?

Adding the lines

set_option profiler true
set_option profiler.threshold 1

near the beginning of the file makes lake build Mathlib.CategoryTheory.Iso succeed (but, of course, noisy), whereas leaving out set_option profiler.threshold 1 still produces the error. :shrug:

Michael Stoll (Apr 28 2024 at 14:39):

It complies with the threshold set to 9, but not with 10.

Michael Stoll (Apr 28 2024 at 14:40):

(deleted)

Michael Stoll (Apr 28 2024 at 15:06):

When I put #exit before line 67

attribute [reassoc (attr := simp)] Iso.hom_inv_id Iso.inv_hom_id

it builds, but when I put it after, it doesn't. So the problem seems to be with that line.

There is a note (lines 279-287)

-- FIXME putting @[reassoc] on the `hom_inv_id` above somehow unfolds `inv`
-- This happens even if we make `inv` irreducible!
-- I don't understand how this is happening: it is likely a bug.

-- attribute [reassoc] hom_inv_id inv_hom_id
-- #print hom_inv_id_assoc
--   theorem CategoryTheory.IsIso.hom_inv_id_assoc {X Y : C} (f : X ⟶ Y) [I : IsIso f]
--     {Z : C} (h : X ⟶ Z),
--     f ≫ Classical.choose (_ : Exists fun inv ↦ f ≫ inv = 𝟙 X ∧ inv ≫ f = 𝟙 Y) ≫ h = h := ...

which may indicate that there have been problems with reassoc before. I'm out of my depth here.

github mathlib4 bot (Apr 28 2024 at 16:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 28 2024 at 21:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 28 2024 at 22:03):

Leo has just added some further flags for disabling some of the IsDefEq changes made recently. They seem to be effective in dealing with slow-downs.

My plan:

  • Install these flags (today even, before the nightly is released, using a local elan override set, which means nightly-testing won't work for others until about +10 hours from now)
  • Hope that Mathlib is happy with in the short term keeping these flags in the problematic places (~30), even on master
  • Continue minimizing the examples where these flags are necessary, with the hope that we can continue to work on IsDefEq.

It's going to be a bit messy in the short term, but I think we're already going to see some big speedups overall. (e.g. @Michael Stoll's noticing what a big effect lean4#4003 has already had).

github mathlib4 bot (Apr 28 2024 at 22:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 28 2024 at 23:10):

Michael Stoll said:

Michael Stoll said:

Michael Stoll said:

exited with code 139

What is the meaning of this error code?

Adding the lines

set_option profiler true
set_option profiler.threshold 1

near the beginning of the file makes lake build Mathlib.CategoryTheory.Iso succeed (but, of course, noisy), whereas leaving out set_option profiler.threshold 1 still produces the error. :shrug:

These errors are fallout from lean4#4006. Fix in the works.

github mathlib4 bot (Apr 28 2024 at 23:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 29 2024 at 01:11):

@Michael Stoll, thanks for your recent help on nightly-testing.

Also, though, a request about writing adaptation notes: it's really helpful if they can be understood without reading the git history.

You wrote:

-- Adaptation note: 2024-04-28
-- replacing the `_` by `P` makes it fast (compare #12412)
@[simp]
theorem Quotient.algebraMap_quotient_of_ramificationIdx_neZero (x : R) :
    algebraMap (R  p) (S  P) (Ideal.Quotient.mk p x) = Ideal.Quotient.mk P (f x) := rfl

but notice here there is no _ after the edit, and several Ps. I'm guessing that it is the P in the RHS, but this is not as obvious as it could be.

Kim Morrison (Apr 29 2024 at 01:13):

(I've updated this note.)

Kim Morrison (Apr 29 2024 at 01:14):

Separately: there is no linkifier in VSCode, so writing https://github.com/leanprover-community/mathlib4/pull/12412 in a comment is much more useful than writing #12412.

github mathlib4 bot (Apr 29 2024 at 01:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 01:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 01:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 03:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 06:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Michael Stoll (Apr 29 2024 at 06:42):

Kim Morrison said:

Separately: there is no linkifier in VSCode, so writing https://github.com/leanprover-community/mathlib4/pull/12412 in a comment is much more useful than writing #12412.

@Kim Morrison Thanks for the tips; I'm doing this for the first time...

Kim Morrison (Apr 29 2024 at 06:43):

(As above, very much appreciated.)

Johan Commelin (Apr 29 2024 at 06:50):

Should we have #adaptation_note that complains

  • If there is a spelling mistake in adaptation_note (atm grep will not find Adapation notes)
  • If there is no version number?
  • If there is no date?
  • If there is no free-form comment...

Johan Commelin (Apr 29 2024 at 06:51):

I'm mostly worried about the first bullet point.

Kim Morrison (Apr 29 2024 at 06:58):

Seems reasonable. Want to implement it? :-)

Johan Commelin (Apr 29 2024 at 06:59):

I'll put it on my Hilbert ~hotel~ todo list

Kim Morrison (Apr 29 2024 at 06:59):

I think we need a technical debt list of lists maintained somewhere, and this can be a bullet point there.

Michael Rothgang (Apr 29 2024 at 07:23):

Kim Morrison said:

I think we need a technical debt list of lists maintained somewhere, and this can be a bullet point there.

Making this list on github is on my TODO list - I can pinky promise to do this by end of June. I've noted this item for it :-)

Kim Morrison (Apr 29 2024 at 08:14):

Gah, lean4#4021 failed, and didn't make it into the nightly, so nightly-testing is probably borked for another day. :-(

github mathlib4 bot (Apr 29 2024 at 08:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 10:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 13:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 18:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 29 2024 at 21:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 30 2024 at 00:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 30 2024 at 00:37):

Despite all the red crosses, we are actually close to converging here.

Kim Morrison (Apr 30 2024 at 00:37):

Unfortunately the "exit code 139" crash that appeared in lean4#4006 has not been resolved, but we at least know how to suppress it (lean4#4021), and we're working on diagnosing the underlying problem. (We discovered one bug in lean4#4028, but that doesn't seem to be the source.)

Kim Morrison (Apr 30 2024 at 00:37):

When nightly-2024-04-30 lands tonight, I think nightly-testing should come green again.

Kim Morrison (Apr 30 2024 at 00:37):

There are quite a few uses of the new backwards compatibility flags on nightly-testing, and my current intention is that we will merge these with master, and deal with them on an ongoing basis.

Kim Morrison (Apr 30 2024 at 00:37):

  • There are currently 5 files that require a set_option backward.isDefEq.lazyProjDelta false in to avoid a timeout. This flag locally reverts the changes to isDefEq from lean4#3965.
  • There are currently 19 files that requies a set_option backward.isDefEq.lazyWhnfCore false in to avoid a timeout. (lean4#4023 is a minimization of one of these, and Leo is actively looking at this.) This flag locally reverts the changes to isDefEq from lean4#4004.
  • There are two files (Mathlib.AlgebraicGeometry.Spec (a known offender with deep defeq abuse) and Mathlib.Geometry.Manifold.VectorBundle (an otherwise nice show case of @Heather Macbeth and @Floris van Doorn's work) which now have new timeouts (i.e. we set maxHeartbeats higher).
    • In Spec, lazyWhnfCore helps, but even with that it requires 800,000 heartbeats (i.e. 4x the limit).
    • In VectorBundle the backwards compatibility flags don't make much difference, but it's also not much over the limit.
  • There are 34 files that require a set_option backward.synthInstance.canonInstances false in to avoid a timeout. I haven't looked at this at all yet, but am not too worried. This flag locally reverts the changes to typeclass search from lean4#4003, prompted by the issue raised in lean4#3996. This change will hopefully give a big speedup overall, so these flags are small cost. I am really hoping that "the community" will be keen to look into these flags and find ways to remove them.

Kim Morrison (Apr 30 2024 at 00:37):

I would like to get feedback on merging these backwards compatibility flags into master. I think it is the right approach, but some +1s would be great.

Kim Morrison (Apr 30 2024 at 00:37):

Finally, at this point we have a long period (2 months) of divergence between nightly-testing and master, and I'm pretty worried about bad merges polluting nightly-testing. I'm going to make a new PR from nightly-testing to bump/v4.8.0 shortly, and I would appreciate careful eyes looking at that diff. Hopefully we can merge that even tonight! After that I think I'll open a PR from bump/v4.8.0 to master (even before v4.8.0-rc1 is out), so we can also get some eyes on that.

github mathlib4 bot (Apr 30 2024 at 01:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Damiano Testa (Apr 30 2024 at 01:32):

Kim, in case it is helpful, the no_lost_declarations script on nightly-testing reports

  • - def add.add := True
  • - def backwardWeight := 1
  • - def buildDiscrTree : IO (DiscrTreeCache (Name × Bool × Nat)) :=
  • - def cachePath : IO FilePath :=
  • + def compute_rfl? (n : SearchNode) : MetaM SearchNode := do
  • - def compute_rfl? (n : SearchNode) : MetaM SearchNode := withMCtx n.mctx do
  • + def cons (a : α) (v : Vector3 α n) : Vector3 α (n + 1) := fun i => by
  • - def cons (a : α) (v : Vector3 α n) : Vector3 α (succ n) := fun i => by
  • + def consElim {C : Vector3 α (n + 1) → Sort u} (H : ∀ (a : α) (t : Vector3 α n), C (a :: t))
  • - def consElim {C : Vector3 α (succ n) → Sort u} (H : ∀ (a : α) (t : Vector3 α n), C (a :: t))
  • - def discrTreeConfig : WhnfCoreConfig := {}
  • - def foldlM {α : Type} {m} [Monad m] (f : α → Expr → m α) (x : α) (e : Expr) : m α :=
  • - def Foo.foo := True
  • - def forwardWeight := 2
  • + def head (v : Vector3 α (n + 1)) : α :=
  • - def head (v : Vector3 α (succ n)) : α :=
  • - def iffOfEq (mvarId : MVarId) : MetaM MVarId := do
  • + def insert (a : α) (v : Vector3 α n) (i : Fin2 (n + 1)) : Vector3 α (n + 1) := fun j =>
  • - def insert (a : α) (v : Vector3 α n) (i : Fin2 (succ n)) : Vector3 α (succ n) := fun j =>
  • - def localHypotheses (except : List FVarId := []) : MetaM (Array (Expr × Bool × Nat)) := do
  • - def processLemma (name : Name) (constInfo : ConstantInfo) :
  • - def proofIrrelHeq (mvarId : MVarId) : MetaM Bool :=
  • - def propext (mvarId : MVarId) : MetaM MVarId := do
  • - def RewriteResult.by? (r : RewriteResult) : Option Expr :=
  • - def RewriteResult.computeRfl (r : RewriteResult) : MetaM RewriteResult := do
  • - def RewriteResult.ppResult (r : RewriteResult) : MetaM String :=
  • - def RewriteResult.prepare_ppResult (r : RewriteResult) : MetaM RewriteResult := do
  • - def rewritesCore (hyps : Array (Expr × Bool × Nat))
  • - def rewritesDedup (hyps : Array (Expr × Bool × Nat))
  • - def rewrites (hyps : Array (Expr × Bool × Nat))
  • - def _root_.Lean.MVarId.liftReflToEq (mvarId : MVarId) : MetaM MVarId := do
  • - def roots : Array FilePath :=
  • + def roots : Array FilePath := #["Mathlib.lean"]
  • - def solveByElim (goals : List MVarId) (depth : Nat := 6) : MetaM PUnit := do
  • - def subsingletonElim (mvarId : MVarId) : MetaM Bool :=
  • + def tail (v : Vector3 α (n + 1)) : Vector3 α n := fun i => v (fs i)
  • - def tail (v : Vector3 α (succ n)) : Vector3 α n := fun i => v (fs i)
  • + def testConst : Nat := 4
  • + def toChar (n : UInt8) : Char := ⟨n.toUInt32, .inl (n.1.2.trans (by decide))⟩
  • - def toChar (n : UInt8) : Char := ⟨n.toUInt32, toChar_aux n.1 n.1.2⟩
  • - def traverseChildren [Applicative M] (f : Expr → M Expr) : Expr → M Expr
  • - def withBindingBody' (n : Name) (x : Expr → m α) : m α := do
  • - def zero : Nat := 0
  • - inductive SideConditions
  • - instance : AddCommGroup (Completion α) :=
  • + instance : CoeTC (M →+[R] M₃) (M →ₗ[R] M₃) :=
  • - instance : CompleteSpace ℝ := by
  • - instance : Denumerable ℚ := by
  • - instance : EuclideanDomain R[X] :=
  • - instance : HasQuotient R (Ideal R) :=
  • + instance instAddCommGroup : AddCommGroup (Completion α) :=
  • - instance instCoeTCLinearMap : CoeTC (M →+[R] M₃) (M →ₗ[R] M₃) :=
  • + instance instDecidableEq [DecidableEq α] : DecidableEq (Booleanisation α) :=
  • - instance instDecidableEq [DecidableEq α] : DecidableEq (Booleanisation α) := Sum.instDecidableEqSum
  • + instance instDenumerable : Denumerable ℚ := by
  • + instance instEuclideanDomain : EuclideanDomain R[X] :=
  • + instance instHasQuotient : HasQuotient R (Ideal R) :=
  • + instance instIsScalarTowerOfSMul [SMul M N] [∀ i, IsScalarTower M N (α i)] :
  • + instance instIsScalarTowerOfSMul [SMul M N] [IsScalarTower M N α] : IsScalarTower M N (Option α) :=
  • + instance instIsScalarTowerOfSMul [SMul R S] : IsScalarTower R S PUnit :=
  • + instance instMulProd {M N} [Mul M] [Mul N] : Mul (M × N) := ⟨fun p q ↦ ⟨p.1 * q.1, p.2 * q.2⟩⟩
  • - instance {M N} [Mul M] [Mul N] : Mul (M × N) := ⟨fun p q ↦ ⟨p.1 * q.1, p.2 * q.2⟩⟩
  • + instance Real.instCompleteSpace : CompleteSpace ℝ := by
  • + instance : SmallCategory (HomAsType α) := inferInstanceAs <| SmallCategory (ShrinkHoms _)
  • - instance : SmallCategory (HomAsType α) := ShrinkHoms.instCategoryShrinkHoms.{0} _
  • - instance [SMul M N] [∀ i, IsScalarTower M N (α i)] : IsScalarTower M N (Σi, α i) :=
  • - instance [SMul M N] [IsScalarTower M N α] : IsScalarTower M N (Option α) :=
  • - instance [SMul R S] : IsScalarTower R S PUnit :=
  • + instance {β : Type*} {C : β → Type*} [∀ b, TopologicalSpace (C b)]
  • + lemma harmonic_eq_sum_Icc {n : ℕ} : harmonic n = ∑ i in Finset.Icc 1 n, (↑i)⁻¹ := by
  • - lemma harmonic_eq_sum_Icc {n : ℕ} : harmonic n = ∑ i in Finset.Icc 1 n, (↑i)⁻¹ := by
  • + lemma one_lt_succ_succ (n : ℕ) : 1 < n.succ.succ := succ_lt_succ <| succ_pos n
  • - lemma pred_eq_sub_one (n : ℕ) : pred n = n - 1 := rfl
  • - lemma prime_of_prime (n : ℕ) : Prime n ↔ Nat.Prime n := by
  • + lemma rec_add_one {C : ℕ → Sort*} (h0 : C 0) (h : ∀ n, C n → C (n + 1)) (n : ℕ) :
  • + lemma stdSimplex_fin_two :
  • - lemma stdSimplex_fin_two : stdSimplex 𝕜 (Fin 2) = [Pi.single 0 1 -[𝕜] Pi.single 1 1] := by
  • - structure RewriteResult where
  • + theorem add_one_pos (n : ℕ) : 0 < n + 1 := succ_pos n
  • + theorem and_or_imp {a b c : Prop} : a ∧ b ∨ (a → c) ↔ a → b ∨ c := Decidable.and_or_imp
  • + theorem antidiagonalTuple_zero_succ (n : ℕ) : antidiagonalTuple 0 (n + 1) = [] :=
  • - theorem antidiagonalTuple_zero_succ (n : ℕ) : antidiagonalTuple 0 n.succ = [] :=
  • + theorem append_insert (a : α) (t : Vector3 α m) (v : Vector3 α n) (i : Fin2 (n + 1))
  • - theorem append_insert (a : α) (t : Vector3 α m) (v : Vector3 α n) (i : Fin2 (succ n))
  • + theorem bagInter_consecutive (n m l : Nat) :
  • - theorem bagInter_consecutive (n m l : Nat) : @List.bagInter ℕ instBEq (Ico n m) (Ico m l) = [] :=
  • - theorem beq_comm {α} [BEq α] [LawfulBEq α] {a b : α} : (a == b) = (b == a) :=
  • - theorem beq_eq_decide_eq {α} [BEq α] [LawfulBEq α] [DecidableEq α]
  • - theorem cast_add [AddMonoidWithOne R] (m n : ℕ) : ((m + n : ℕ) : R) = m + n := by
  • + theorem cast_add_one_ne_zero (n : ℕ) : (n + 1 : R) ≠ 0 :=
  • - theorem cast_add_one_ne_zero (n : ℕ) : (n + 1 : R) ≠ 0 := by
  • + theorem cast_add {R : Type*} [AddMonoidWithOne R] (m n : ℕ) : ((m + n : ℕ) : R) = m + n := by
  • - theorem coe_iff_coe : ∀ {a b : Bool}, (a ↔ b) ↔ a = b := by decide
  • - theorem cond_decide {α} (p : Prop) [Decidable p] (t e : α) :
  • - theorem cond_eq_ite {α} (b : Bool) (t e : α) : cond b t e = if b then t else e := by
  • - theorem cond_not {α} (b : Bool) (t e : α) : cond (!b) t e = cond b e t := by cases b <;> rfl
  • - theorem cond_self.{u} {α : Type u} (b : Bool) (a : α) : cond b a a = a := by cases b <;> rfl
  • + theorem cons_head_tail (v : Vector3 α (n + 1)) : (head v :: tail v) = v :=
  • - theorem cons_head_tail (v : Vector3 α (succ n)) : (head v :: tail v) = v :=
  • - theorem decide_and (p q : Prop) [Decidable p] [Decidable q] : decide (p ∧ q) = (p && q) := by
  • - theorem decide_coe (b : Bool) {h} : @decide b h = b := by
  • - theorem decide_or (p q : Prop) [Decidable p] [Decidable q] : decide (p ∨ q) = (p || q) := by
  • - theorem default_bool : default = false :=
  • - theorem dist.def (n m : ℕ) : dist n m = n - m + (m - n) :=
  • + theorem eval_of (n : ℕ) (x : M) : eval I M n (of I M x) = mkQ (I ^ n • (⊤ : Submodule R M)) x :=
  • - theorem eval_of (n : ℕ) (x : M) : eval I M n (of I M x) = mkQ _ x :=
  • + theorem Fintype.card_exp_univ_card_eq [Fintype α] [Fintype β] :
  • + theorem foo (n : Nat) : makeSingleton n = [0] := by
  • - theorem getD_cons_succ : getD (x :: xs) (n + 1) d = getD xs n d :=
  • - theorem getD_cons_zero : getD (x :: xs) 0 d = x :=
  • - theorem getD_nil : getD [] n d = d :=
  • + theorem homOfLE_refl {x : X} (h : x ≤ x) : h.hom = 𝟙 x :=
  • - theorem homOfLE_refl {x : X} : (le_refl x).hom = 𝟙 x :=
  • - theorem imp_and_neg_imp_iff (p q : Prop) : (p → q) ∧ (¬p → q) ↔ q := by
  • + theorem imp_and_neg_imp_iff (p q : Prop) : (p → q) ∧ (¬p → q) ↔ q := by simp
  • + theorem imp_iff_right_iff {a b : Prop} : (a → b ↔ b) ↔ a ∨ b := Decidable.imp_iff_right_iff
  • + theorem index_exists {j : ℕ} (h : j < n) : ∃ i : ℕ, j < c.sizeUpTo (i + 1) ∧ i < c.length := by
  • - theorem index_exists {j : ℕ} (h : j < n) : ∃ i : ℕ, j < c.sizeUpTo i.succ ∧ i < c.length := by
  • + theorem insert_fs (a : α) (b : α) (v : Vector3 α n) (i : Fin2 (n + 1)) :
  • - theorem insert_fs (a : α) (b : α) (v : Vector3 α n) (i : Fin2 (succ n)) :
  • + theorem isEmpty_exists_isempty_fun : (∃ (_ : α), IsEmpty β) ↔ Nonempty α ∧ IsEmpty β := by
  • - theorem isEmpty_fun : IsEmpty (α → β) ↔ Nonempty α ∧ IsEmpty β := by
  • + theorem isEmpty_fun : IsEmpty (α → β) ↔ Nonempty α ∧ IsEmpty β := by simp
  • - theorem ite_eq_false_distrib (c : Prop) [Decidable c] (a b : Bool) :
  • - theorem ite_eq_true_distrib (c : Prop) [Decidable c] (a b : Bool) :
  • + theorem length_split_fst_le (l : List α) : length (split l).1 ≤ length l :=
  • + theorem length_split_snd_le (l : List α) : length (split l).2 ≤ length l :=

Damiano Testa (Apr 30 2024 at 01:32):

  • + theorem measure_fundamentalFrontier (hs : IsFundamentalDomain G s μ) :
  • - theorem measure_fundamentalFrontier : μ (fundamentalFrontier G s) = 0 := by
  • - theorem Ne.def {α : Sort u} (a b : α) : (a ≠ b) = ¬ (a = b) := rfl
  • - theorem not_eq_not : ∀ {a b : Bool}, ¬a = !b ↔ a = b := by decide
  • + theorem not_implies_eq : (¬ (p → q)) = (p ∧ ¬ q) := propext Classical.not_imp
  • - theorem not_implies_eq : (¬ (p → q)) = (p ∧ ¬ q) := propext not_imp
  • - theorem not_not_eq : ∀ {a b : Bool}, ¬(!a) = b ↔ a = b := by decide
  • + theorem nthLe_congr {l : List α} {n p : ℕ} {h : n < length l} (hnp : n = p) :
  • - theorem ofPowerSeries_X_pow {R} [CommSemiring R] (n : ℕ) :
  • + theorem ofPowerSeries_X_pow {R} [Semiring R] (n : ℕ) :
  • + theorem one_def : (1 : 𝒜 ᵍ⊗[R] ℬ) = 1 ᵍ⊗ₜ 1 := rfl
  • + theorem single_pow (a : Γ) (n : ℕ) (r : R) : single a r ^ n = single (n • a) (r ^ n) := by
  • - theorem succ_one : succ (1 : Ordinal) = 2 := by
  • + theorem succ_one : succ (1 : Ordinal) = 2 := by congr; simp only [Nat.unaryCast, zero_add]
  • - theorem toChar_aux (n : Nat) (h : n < size) : Nat.isValidChar (UInt32.ofNat n).1 := by

  • 53 added declarations
  • 89 removed declarations
  • 0 paired declarations

github mathlib4 bot (Apr 30 2024 at 01:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 30 2024 at 01:35):

That is both too much and too little to be helpful. :-)

Kim Morrison (Apr 30 2024 at 01:35):

Can it list differences by file?

Kim Morrison (Apr 30 2024 at 01:35):

And show namespaces?

Damiano Testa (Apr 30 2024 at 01:36):

I can easily make it print file names, but the tool was designed to help with moves, so it does not do it out-of-the-box.

Damiano Testa (Apr 30 2024 at 01:36):

Namespaces is trickier, since one of the features is that it runs with possibly corrupt files, so does not use oleans.

Damiano Testa (Apr 30 2024 at 01:37):

I can try to implement a text-based namespace, but it would be buggy (though likely usually helpful).

Damiano Testa (Apr 30 2024 at 01:37):

Again, that is not currently implemented, though.

Damiano Testa (Apr 30 2024 at 01:39):

In any case, it is quite late now and I am going to bed, so either one of these features will have to wait! :smile:

Kim Morrison (Apr 30 2024 at 01:45):

Okay, namespaces are not essential if filenames are available.

Kim Morrison (Apr 30 2024 at 01:49):

One important question here is if we need to write comments along with the set_option backward.isDefEq.lazyWhnfCore false in options, or if they are self-explanatory enough??

Kim Morrison (Apr 30 2024 at 01:49):

Maybe a tracking issue, one for each such flag, is best.

Kim Morrison (Apr 30 2024 at 01:49):

Currently all the canonInstance flags have a paragraph, but the other two don't.

Damiano Testa (Apr 30 2024 at 02:10):

Here is a first attempt at putting filenames: it is not polished, but might contain all the right information

First_batch

Damiano Testa (Apr 30 2024 at 02:10):

Second_batch

Damiano Testa (Apr 30 2024 at 02:11):

(now I am really going to bed!)

github mathlib4 bot (Apr 30 2024 at 02:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 30 2024 at 02:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 30 2024 at 06:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Michael Stoll (Apr 30 2024 at 09:06):

Kim Morrison said:

I would like to get feedback on merging these backwards compatibility flags into master. I think it is the right approach, but some +1s would be great.

I think it would be very good to get some of the new things to be usable with Mathlib soon (in particular, the fix for apply? and lena4#4003), so I am very much in favor of this.

The need for the backward compatibility flag on instance synthesis probably points to some problems with the design of our type classes in some areas, so this may actually be helpful in getting to the bottom of these problems.

github mathlib4 bot (Apr 30 2024 at 11:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 30 2024 at 11:22):

Woah, lean4checker failure.

Kim Morrison (Apr 30 2024 at 11:23):

Oh, lake has changed where it pipes its output. @Mac Malone

Error: The command 'lake exe lean4checker Lean4CheckerTests.AddFalse' did not produce the expected error.
Expected:
uncaught exception: (kernel) declaration type mismatch, 'false' has type
  Prop
but it is expected to have type
  False
Got:
[?/?] Computing build jobs
[1/5] Building Lean4Checker.Lean
[2/5] Building Main
[3/5] Compiling Main
[4/5] Compiling Lean4Checker.Lean
[5/5] Linking lean4checker
uncaught exception: (kernel) declaration type mismatch, 'false' has type
  Prop
but it is expected to have type
  False

Kim Morrison (Apr 30 2024 at 11:27):

Not saying this needs to be changed if it is intentional.

Kim Morrison (Apr 30 2024 at 11:28):

Oh, weird, and running it locally produces:

% ./test.sh
Error: The command 'lake -q exe lean4checker Lean4CheckerTests.AddFalse' did not produce the expected error.
Expected:
uncaught exception: (kernel) declaration type mismatch, 'false' has type
  Prop
but it is expected to have type
  False
Got:






uncaught exception: (kernel) declaration type mismatch, 'false' has type
  Prop
but it is expected to have type

Kim Morrison (Apr 30 2024 at 11:29):

That is looking like something to fix.

Floris van Doorn (Apr 30 2024 at 12:14):

@Kim Morrison I managed to minimize the timeout in vector bundle to this almost-mathlib free mwe:

import Mathlib.Logic.Basic

def MyExists := @Exists

lemma foo {α : Type _} {P : α  Prop} : ( x, P x)  MyExists P :=
  .rfl

example (x : ) :
   (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x), True := by
  simp only [foo]

This example gets exponentially slow depending on the number of hypotheses h you add. I think it has to do a congr-lemma in Mathlib.

Kim Morrison (Apr 30 2024 at 12:15):

Fascinating, thank you!

Kim Morrison (Apr 30 2024 at 12:16):

It ... doesn't look much like a vector bundle anymore.

Kim Morrison (Apr 30 2024 at 12:16):

What does the iterated existential correspond to originally?

Floris van Doorn (Apr 30 2024 at 12:16):

I can confirm that on Mathlib master this is linear in the number of hypotheses h.
It were iterated unions, and all the time was spent on simp only [mem_iUnion]

Kim Morrison (Apr 30 2024 at 12:17):

Awesome, okay, is it okay if I keep minimizing and get it off Mathlib entirely?

Floris van Doorn (Apr 30 2024 at 12:17):

Yes, please do!

Floris van Doorn (Apr 30 2024 at 12:19):

The declaration smoothFiberwiseLinear was already slow on Mathlib master, with a large amount of the time spent on the simp only's. So maybe there is more speedup to be gained there...

Kim Morrison (Apr 30 2024 at 12:32):

import Lean

section Mathlib.Logic.Basic

@[congr]
theorem exists_prop_congr {p p' : Prop} {q q' : p  Prop} (hq :  h, q h  q' h) (hp : p  p') :
    Exists q   h : p', q' (hp.2 h) := sorry

@[congr]
theorem exists_prop_congr' {p p' : Prop} {q q' : p  Prop} (hq :  h, q h  q' h) (hp : p  p') :
    Exists q =  h : p', q' (hp.2 h) := sorry

end Mathlib.Logic.Basic

def MyExists := @Exists

theorem foo {α : Type _} {P : α  Prop} : ( x, P x)  MyExists P :=
  .rfl

-- This takes under 1000 on `v4.7.0`, and is linear in the depth of the existential.
-- On `master` it is exponential!
set_option maxHeartbeats 10000 in
example (x : ) :
   (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x), True := by
  simp only [foo]
  sorry

is Mathlib free. It requires both of the congr lemmas to cause the bad behaviour.

Kim Morrison (Apr 30 2024 at 12:33):

Two things to do, I guess: find out what in lean is changing this to exponential behaviour, and see if we can get rid of one or both of these lemmas in Mathlib!

Floris van Doorn (Apr 30 2024 at 12:34):

With one congr lemma I also get exponential behavior:

@[congr]
theorem exists_prop_congr {p p' : Prop} {q q' : p  Prop} (hq :  h, q h  q' h) (hp : p  p') :
    Exists q   h : p', q' (hp.2 h) := sorry

set_option profiler true
example (x : Nat) :
   (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x), True := by
  simp only

Floris van Doorn (Apr 30 2024 at 12:35):

(I couldn't resist myself from also minimizing it a bit further myself :-) )

Kyle Miller (Apr 30 2024 at 12:38):

That seems like it's not a good congr lemma. Every time it's applied, simp will need to deal with the hp.2 h terms that accumulate.

Floris van Doorn (Apr 30 2024 at 12:39):

Maybe. We can try to see how much breaks in Mathlib if we only congr on q while leaving p constant. It seems useful to be able to simp both...

Kim Morrison (Apr 30 2024 at 12:40):

Half way through mathlib, no breakage so far.

Kim Morrison (Apr 30 2024 at 12:40):

I think just removing would be great, if nothing breaks.

Floris van Doorn (Apr 30 2024 at 12:40):

Does simp actually simplify proofs of propositions? Is that useful?

Kyle Miller (Apr 30 2024 at 12:40):

Oh right, hp.2 h is a proof, so it won't touch that.

Yaël Dillies (Apr 30 2024 at 12:40):

Yes, eg Acc

Floris van Doorn (Apr 30 2024 at 12:42):

@Kim Morrison I think that the congr lemma that made the vector bundle declaration slow is Set.iUnion_congr_Prop.

github mathlib4 bot (Apr 30 2024 at 12:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Matthew Ballard (Apr 30 2024 at 12:56):

Is this the change to docs#Lean.Meta.Simp.simpArrow ?

Matthew Ballard (Apr 30 2024 at 12:56):

Tracing debug crashes my editor

Matthew Ballard (Apr 30 2024 at 13:55):

Kim Morrison said:

  • There are currently 19 files that requies a set_option backward.isDefEq.lazyWhnfCore false in to avoid a timeout. (lean4#4023 is a minimization of one of these, and Leo is actively looking at this.) This flag locally reverts the changes to isDefEq from lean4#4004.

You can make lean#4023 instantaneous by specifying the submodule of the RHS. If not, Lean guesses correctly that it should try Submodule.localized' S p f M' but the metavariable appearing in its place is not assignable (depth?). This remains true even if you specify the ring for the submodule.

Do we want to make this adaptation for nightly-testing or wait until the something arrives for lean#4023?

Kim Morrison (Apr 30 2024 at 14:04):

Leo also discovered that making any of Membership.mem, Submodule.op, or ... one other, I forget, irreducible makes it instantaneous.

In v4.8.0-rc1 we will have much more flexibility to control reducibility (e.g. locally, in scopes, in later files), and hopefully we can use that flexibility to make a lot more things irreducible!

Kim Morrison (Apr 30 2024 at 14:04):

I'm inclined to postpone fixes for individual lazyWhnfCore options until after this all hits master.

Kim Morrison (Apr 30 2024 at 14:04):

(People will enjoy cleaning them up!)

Matthew Ballard (Apr 30 2024 at 14:05):

Performance on master is also quite bad. It just don't trip any limits

Kim Morrison (Apr 30 2024 at 14:07):

I hope that the workflow:

  • try making something irreducible
  • patch downstream problems by use a local attribute
  • (possibly merge in the meantime, and then later)
  • work out the missing lemmas to add to avoid needing local semireducibility
  • converge on making things irreducible immediately after the initial API setup

will be quite productive

Matthew Ballard (Apr 30 2024 at 14:10):

There is no option to trace metavariable creation with their individual contexts right?

Matthew Ballard (Apr 30 2024 at 14:10):

I get the creeping feeling that mathlib has an anti-pattern and this is an example

Floris van Doorn (Apr 30 2024 at 14:11):

I was also investigating another maxheartbeats in the manifold library, and I just made #12552 that makes LocalInvariantProp a structure, which means that many manifold-predicates can only be unfolded a few steps. This improves performance a bit, and flagged some defeq-abuses.

Patrick Massot (Apr 30 2024 at 14:19):

Do I understand correctly that we are going back to the way Lean 3 worked here?

github mathlib4 bot (Apr 30 2024 at 15:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Matthew Ballard (Apr 30 2024 at 16:44):

I still can't believe this universe issue.

Matthew Ballard (Apr 30 2024 at 16:45):

But it allows the removal of some backward.isDefEq.lazyWhnfCore flags

Matthew Ballard (Apr 30 2024 at 16:49):

Kim Morrison said:

* In Spec, lazyWhnfCore helps, but even with that it requires 800,000 heartbeats (i.e. 4x the limit).

Gone

Matthew Ballard (Apr 30 2024 at 16:53):

And the universe signature did not change.

Matthew Ballard (Apr 30 2024 at 17:26):

#12557

Matthew Ballard (Apr 30 2024 at 17:53):

Other than universe issues (which is also a case of this in a way), every regression I've poked at follows the same pattern:

  • there is some implicit variable that Lean needs to fill in
  • Lean tries to assign the correct thing but the metavariable is unassignable
  • Lean soldiers on, with much effort, with the metavariable in place hoping something else will work
  • filling in the implicit variable explicitly makes the declaration lightning quick

Matthew Ballard (Apr 30 2024 at 17:54):

In lean#4023, making those things irreducible only returns performance to ~master-level which is still orders of magnitude slower than filling the implicit explicitly

github mathlib4 bot (Apr 30 2024 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Michael Stoll (Apr 30 2024 at 19:47):

Does it make sense to try to fix the problem in Mathlib.Data.Rat.Defs?

Ruben Van de Velde (Apr 30 2024 at 21:12):

Matthew Ballard said:

#12557

This is ready for bors if anyone's around :)

github mathlib4 bot (Apr 30 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Apr 30 2024 at 23:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Apr 30 2024 at 23:30):

I've just merged master into bump/v4.8.0 again. I'm not super confident I got all the merge conflicts correct. I'm building locally now but will be away from the computer for a bit soon.

github mathlib4 bot (May 01 2024 at 00:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 01 2024 at 03:28):

#12567 just removes one of the two congr lemmas in the mwe, since it is unused and seems safest to have out of the way. I'll separately report the linear --> exponential change in behaviour.

github mathlib4 bot (May 01 2024 at 04:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 01 2024 at 05:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (May 01 2024 at 05:43):

Floris van Doorn said:

With one congr lemma I also get exponential behavior:

@[congr]
theorem exists_prop_congr {p p' : Prop} {q q' : p  Prop} (hq :  h, q h  q' h) (hp : p  p') :
    Exists q   h : p', q' (hp.2 h) := sorry

set_option profiler true
example (x : Nat) :
   (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x)
      (h : x = x), True := by
  simp only

A git bisect reveals this change in behaviour originates in lean4#3972, which changed how simp caching works.

Johan Commelin (May 01 2024 at 05:49):

I'm really excited to find out the total speed up compared to 2 weeks ago (say).

Kim Morrison (May 01 2024 at 05:52):

Yes, we are about to run !bench. I'm pretty terrified it is going to be disappointing. Local builds feel slow to me, but we have zero hard data right now. This is something we need to get much better at going forward. Every nightly-testing-YYYY-MM-DD (note that these are not actually created every day, only on green days) is already sent to the speedcenter, but we have no systematic way of looking at the results.

Kim Morrison (May 01 2024 at 05:54):

I think the two major things remaining are:

  • I'm looking through #12548 for anything that looks like a bad merge. I'd really appreciate if someone else can as well.
  • We need to run !bench...

Johan Commelin (May 01 2024 at 05:55):

Well, we have

  • change to CharP.CharOne instance
  • changes to convert/congr!, subsingleton stuff
  • explicit universes
  • change to TC synthesis algorithm to stop retrying stuff

Altogether this must have a noticeable impact, I hope!

Kim Morrison (May 01 2024 at 05:56):

Some of these have happened on master already, so won't be "credited" in the !bench results.

Kim Morrison (May 01 2024 at 05:56):

But yes, we can compare master two weeks ago.

github mathlib4 bot (May 01 2024 at 06:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (May 01 2024 at 06:49):

I will try to make some more time to review the pr today, but might only be tonight

github mathlib4 bot (May 01 2024 at 09:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 01 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 01 2024 at 11:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 01 2024 at 12:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 01 2024 at 12:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 01 2024 at 12:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 01 2024 at 12:24):

git is failing with a 128 on lake build cache. Not sure what could be wrong there!

github mathlib4 bot (May 01 2024 at 12:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 01 2024 at 15:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 01 2024 at 18:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 01 2024 at 21:08):

@Floris van Doorn, Leo has modified the simp cache in https://github.com/leanprover/lean4/pull/4044 and fixed the exponential behaviour.

github mathlib4 bot (May 01 2024 at 21:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 02 2024 at 01:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 02 2024 at 02:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 02 2024 at 03:25):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 02 2024 at 10:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 02 2024 at 15:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 02 2024 at 18:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 02 2024 at 21:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 03 2024 at 00:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 03 2024 at 04:04):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 03 2024 at 10:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 03 2024 at 13:51):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 03 2024 at 16:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 03 2024 at 19:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 04 2024 at 10:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 04 2024 at 12:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 04 2024 at 21:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 05 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 05 2024 at 03:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (May 05 2024 at 06:02):

error: ././././Mathlib/Order/Heyting/Hom.lean:191:2-191:11: failed to set reducibility status, BoundedLatticeHomClass.toBiheytingHomClass is not a definition
use set_option allowUnsafeReducibility true to override reducibility status validation

github mathlib4 bot (May 05 2024 at 06:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 05 2024 at 12:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 05 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 05 2024 at 18:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (May 05 2024 at 19:00):

I'm just removing any reducible attributes on theorems, I hope that's right

github mathlib4 bot (May 05 2024 at 19:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 05 2024 at 20:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 05 2024 at 22:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 01:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 05:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (May 06 2024 at 05:36):

@Ruben Van de Velde, I've backported most of your changes in #12691.

Ruben Van de Velde (May 06 2024 at 05:38):

I'm not sure if I should review my own changes:)

Kim Morrison (May 06 2024 at 05:38):

Okay, I guess. :-)

Kim Morrison (May 06 2024 at 05:52):

nb: incoming lean#4037 tonight will require lean-pr-testing-4037 merged into nightly-testing.

github mathlib4 bot (May 06 2024 at 06:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 07:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 06 2024 at 10:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 11:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 12:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 13:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 16:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 19:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 22:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 06 2024 at 23:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 07 2024 at 09:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (May 07 2024 at 09:34):

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

More batteries fallout cc @Mario Carneiro

github mathlib4 bot (May 07 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 07 2024 at 12:11):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 09 2024 at 08:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 09 2024 at 09:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 10 2024 at 09:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 10 2024 at 09:51):

The batteries bump hadn't arrived in time, but is in now.

github mathlib4 bot (May 10 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 10 2024 at 15:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 10 2024 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 10 2024 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 11 2024 at 03:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 11 2024 at 06:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 11 2024 at 09:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 11 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 11 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 11 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 11 2024 at 18:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 11 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 12 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 12 2024 at 03:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 12 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 12 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 12 2024 at 18:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 12 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 12 2024 at 23:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 12 2024 at 23:41):

Needs lean-pr-testing-4061 merged in.

github mathlib4 bot (May 13 2024 at 00:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 13 2024 at 00:52):

Needed a type annotation on an ambiguous numeral on an incoming change from master.

github mathlib4 bot (May 13 2024 at 01:51):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 14 2024 at 01:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 14 2024 at 03:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 14 2024 at 06:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 14 2024 at 10:07):

@Joachim Breitner, I've successfully removed the unseal Nat.modCores from nightly-testing, thanks!

Kim Morrison (May 14 2024 at 10:15):

I'm fixing a few proofs in nightly-testing to avoid needing to unseal things as much. I'll backport to master in a bit.

github mathlib4 bot (May 14 2024 at 11:07):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 14 2024 at 13:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 14 2024 at 19:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 14 2024 at 22:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 14 2024 at 23:39):

Deprecations in dot notation that aren't visible on master. Backported as #12920

github mathlib4 bot (May 15 2024 at 00:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 16 2024 at 10:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 16 2024 at 13:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 16 2024 at 16:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 16 2024 at 19:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 16 2024 at 22:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 17 2024 at 00:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 17 2024 at 01:27):

#12969 backports some changes to EllipticDivisibilitySequence

github mathlib4 bot (May 17 2024 at 02:33):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 17 2024 at 06:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 17 2024 at 10:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 17 2024 at 13:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 17 2024 at 16:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 17 2024 at 18:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 17 2024 at 22:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 18 2024 at 01:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 18 2024 at 07:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 18 2024 at 09:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 18 2024 at 10:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 18 2024 at 12:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 18 2024 at 15:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 18 2024 at 19:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 18 2024 at 21:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 19 2024 at 01:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 19 2024 at 03:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 19 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 19 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 19 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 19 2024 at 23:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 20 2024 at 00:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 20 2024 at 00:35):

#13045 has some backport deprecation warning fixes

github mathlib4 bot (May 20 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 20 2024 at 01:02):

#13046 contains further backports. There are still a few more changes, which look more regression-y, on nightly-testing. I'll make a PR out of these soon.

github mathlib4 bot (May 20 2024 at 02:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 20 2024 at 05:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 20 2024 at 05:19):

Just the noisy output detector correctly complaining about unwanted output from Lake, which will be fixed tonight in lean#4220.

github mathlib4 bot (May 20 2024 at 06:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 20 2024 at 11:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 20 2024 at 11:33):

Updated the noisy CI filter for the new lake output, hopefully okay now.

github mathlib4 bot (May 20 2024 at 11:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 20 2024 at 12:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 21 2024 at 10:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 21 2024 at 10:49):

Just required merging existing fixes on lean-pr-testing-4231, PR shortly.

Kim Morrison (May 21 2024 at 10:50):

Btw --- if anyone wants to check out the new lake build output, it is available now on nightly-testing.

github mathlib4 bot (May 21 2024 at 10:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 21 2024 at 10:50):

Wouldn't hurt to have a few people take a look, as the new lake build output is going to arrive on rc2 (hopefully <24 hours?), and hasn't been tested a whole lot.

Kim Morrison (May 21 2024 at 10:53):

Oops, Cache was broken by the Lake.crlf2lf --> String.crlfToLf (undeprecated!) rename.

Kim Morrison (May 21 2024 at 10:56):

And needed to merge lean-pr-testing-4224 as well.

But our system is working nicely at the moment: lots of Lean PRs are using the nightly-with-mathlib tag as their base, and so we end up with Mathlib patches all ready to go, rather than having to diagnose the breakage. :-) :-)

github mathlib4 bot (May 21 2024 at 11:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 21 2024 at 13:54):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 23 2024 at 10:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 23 2024 at 10:35):

Ah, this is fallout from @Yuyang Zhao's lean#4188. I should have asked for a mathlib build before merging, by mistake.

@Yuyang Zhao, do you have a fix on hand?

Kim Morrison (May 23 2024 at 10:40):

Okay, think I have it sorted out.

Mauricio Collares (May 23 2024 at 10:41):

Whoops, sorry! I forgot to check here and just pushed what I think is a fix.

Mauricio Collares (May 23 2024 at 10:41):

Feel free to force push your fix

Kim Morrison (May 23 2024 at 11:08):

No worries, I left for dinner. I'll merge and see what happens.

Kim Morrison (May 23 2024 at 11:09):

All good. One of your fixes was better than mine. I just replaced a lemma name, you replaced the whole proof!

github mathlib4 bot (May 23 2024 at 12:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 23 2024 at 12:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 23 2024 at 13:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 23 2024 at 13:52):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 24 2024 at 07:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 24 2024 at 09:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 24 2024 at 11:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 24 2024 at 11:16):

Just a deprecation.

github mathlib4 bot (May 24 2024 at 12:16):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 24 2024 at 16:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 24 2024 at 19:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 24 2024 at 22:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 25 2024 at 01:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 25 2024 at 01:34):

Just some deprecations, backported on #13192.

github mathlib4 bot (May 25 2024 at 02:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 25 2024 at 04:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 25 2024 at 09:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 25 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 25 2024 at 13:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 25 2024 at 16:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 25 2024 at 22:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 26 2024 at 01:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 26 2024 at 04:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 26 2024 at 10:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 26 2024 at 12:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 26 2024 at 12:25):

@Jannis Limperg, there was a problem here in Aesop caused by your https://github.com/leanprover-community/aesop/commit/1bbc601de6ff7b69fee3c028069879e830baa0e8.

The problem is that we have removed Lean.Expr.findM? (recently added), because we decided it was too dangerous to allow potential side-effecting monadic calculations while using a pointer based cache.

Your recent addition of hasSorry relied on findM?.

Kim Morrison (May 26 2024 at 12:25):

For now I've simply reverted this commit on nightly-testing, but obviously we still need a solution here.

Kim Morrison (May 26 2024 at 12:25):

Can I pass the baton to you to think about how to achieve this without findM??

Kim Morrison (May 26 2024 at 12:26):

We did consider the possibility of keeping findM? but with prominent warnings that you have to be really careful about side effects... This can still be on the table.

github mathlib4 bot (May 26 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Jannis Limperg (May 26 2024 at 12:54):

Kim Morrison said:

Can I pass the baton to you to think about how to achieve this without findM??

I see a few options:

  • Work around it in Aesop by moving the monadic computation into a loop around find?. The code is not at all performance-critical, so this is fine.
  • Provide an unsafe findM? as you suggest.
  • Rename findM? to unsafeFindM? or another suitably scary name and possibly add a safe variant findM? without the pointer-based cache.

The last one would be my favourite.

Jannis Limperg (May 26 2024 at 12:56):

Actually, the workaround in Aesop is even easier than that. I just need to get the mctx and then use it for pure lookups in find?.

Kim Morrison (May 26 2024 at 13:46):

Let's do that. The decision to remove findM? was in part motivated by the hope that in most use cases, if there were no side effects probably it could actually be made pure.

github mathlib4 bot (May 26 2024 at 15:03):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 26 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 26 2024 at 19:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 26 2024 at 22:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 27 2024 at 01:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 27 2024 at 04:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 27 2024 at 07:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 27 2024 at 11:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 27 2024 at 11:34):

The problem here is that lake build is saying:

% lake build
 [544/4549] Replayed Mathlib.Data.Set.Basic
info: ././././Mathlib/Data/Set/Basic.lean:2646:0: 0
Build completed successfully.

and this is failing the noisy output check.

@Mac Malone, do you know why Lake would be telling us that it replayed something here?

Sebastian Ullrich (May 27 2024 at 11:55):

Is that not correct? https://github.com/leanprover-community/mathlib4/blob/nightly-testing/Mathlib/Data/Set/Basic.lean#L2646

Ruben Van de Velde (May 27 2024 at 12:00):

Yeah, that was my attempt to debug

Ruben Van de Velde (May 27 2024 at 12:00):

Before it was failing with

error: ././././Mathlib/Order/Circular.lean:6:0: failed to read file '././.lake/build/lib/Mathlib/Data/Set/Basic.olean', invalid header

Ruben Van de Velde (May 27 2024 at 12:01):

Hold on, didn't we recently start uploading to the cache when the build was interrupted?

Jannis Limperg (May 27 2024 at 12:06):

Kim Morrison said:

Let's do that. The decision to remove findM? was in part motivated by the hope that in most use cases, if there were no side effects probably it could actually be made pure.

Done and Aesop's nightly-testing is up to date again.

github mathlib4 bot (May 27 2024 at 13:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 27 2024 at 16:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 27 2024 at 19:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 27 2024 at 21:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 28 2024 at 01:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 28 2024 at 03:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 28 2024 at 06:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 28 2024 at 09:24):

A change on master (norm_iteratedFDeriv_fourierPowSMulRight) now requires a set_option maxSynthPendingDepth 2 in.

github mathlib4 bot (May 28 2024 at 11:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 28 2024 at 12:24):

Just a deprecation warning following a change on master. These will stop shortly when Mathlib means to v4.9.0-rc1.

github mathlib4 bot (May 28 2024 at 13:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 28 2024 at 16:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 28 2024 at 19:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 28 2024 at 22:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 29 2024 at 01:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 29 2024 at 04:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 29 2024 at 08:43):

Changes on master that relied on well-founded defs being semireducible.

github mathlib4 bot (May 29 2024 at 09:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (May 29 2024 at 09:31):

:up: probably more of the same in Mathlib/RingTheory/Polynomial/Chebyshev.lean (not looking right now)

github mathlib4 bot (May 29 2024 at 11:11):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 29 2024 at 17:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 29 2024 at 19:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 29 2024 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 30 2024 at 07:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 30 2024 at 10:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 30 2024 at 11:06):

Some synthPendingDepth issues with @Jireh Loreaux's changes to StoneWeierstrauss. Seems straightforward: we can remove some shortcut instances at the price of increasing synthPendingDepth.

github mathlib4 bot (May 30 2024 at 11:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Jireh Loreaux (May 30 2024 at 14:21):

@Kim Morrison can you explain further? I thought we couldn't increase synthPendingDepth?

github mathlib4 bot (May 30 2024 at 15:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 30 2024 at 18:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 30 2024 at 21:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 31 2024 at 03:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (May 31 2024 at 06:06):

Jireh Loreaux said:

Kim Morrison can you explain further? I thought we couldn't increase synthPendingDepth?

I think the consensus now is that it is fine to locally increase it to 2, and that this is preferable to aging appreciate instances.

Kim Morrison (May 31 2024 at 06:08):

Moreover, we should try to build Mathlib with it globally at 2 again, and if we can get it to build check the benchmark. (When we previously tried this it was too slow.) If we can avoid they performance penalty there is no reason not to increase it globally.

Kim Morrison (May 31 2024 at 08:08):

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Just some upstreamed lemmas about Fin.

github mathlib4 bot (May 31 2024 at 08:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 31 2024 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (May 31 2024 at 11:25):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (May 31 2024 at 15:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 01 2024 at 04:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 01 2024 at 07:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 01 2024 at 07:25):

File deleted on master (Mathlib/Data/BitVec/Lemmas) had local changes on nightly-testing, so wasn't deleted correctly.

github mathlib4 bot (Jun 01 2024 at 08:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 01 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 01 2024 at 11:48):

A shake was required, and I've also bumped dependencies.

github mathlib4 bot (Jun 01 2024 at 12:52):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 02 2024 at 10:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 02 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 03 2024 at 00:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 03 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 03 2024 at 11:52):

Appears to have just need lean-pr-testing-4314 merged. About to hope back on a plane. :-)

Ruben Van de Velde (Jun 03 2024 at 12:08):

I'll try that

github mathlib4 bot (Jun 03 2024 at 12:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Jun 03 2024 at 12:10):

Oh, you did

github mathlib4 bot (Jun 03 2024 at 13:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 03 2024 at 13:57):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Jun 03 2024 at 23:26):

Thanks!

github mathlib4 bot (Jun 04 2024 at 00:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 04 2024 at 00:52):

Just needs a shake again, after merging master->bump/v4.9.0->nightly-testing

github mathlib4 bot (Jun 04 2024 at 01:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 04 2024 at 10:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 04 2024 at 21:32):

Fallout from lean4#4321. There's no adaptation branch, but I'll fix this up soon.

Kim Morrison (Jun 04 2024 at 21:42):

Oof, this encountered an unpleasant any_goals simp [...] proof which was actually meant to be a swap · simp [...].

github mathlib4 bot (Jun 04 2024 at 22:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 04 2024 at 22:41):

Interesting! @Joachim Breitner's lean4#4177 has changed the behaviour of simp so when given an invalid theorem is generates an error but continues. This has changed the behaviour of norm_num to do the same, so we need to update the relevant norm_num test.

github mathlib4 bot (Jun 04 2024 at 22:56):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 05 2024 at 09:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 05 2024 at 09:29):

nightly-testing is badly broken today:

- Mathlib.Data.List.EditDistance.Estimator
- Mathlib.Data.Seq.Parallel
- Mathlib.CategoryTheory.Limits.HasLimits
- Mathlib.GroupTheory.Perm.Support
- Mathlib.Data.QPF.Multivariate.Constructions.Fix
- Mathlib.Combinatorics.Hall.Finite
- Mathlib.Combinatorics.SimpleGraph.Triangle.Counting
- Mathlib.SetTheory.Ordinal.FixedPointApproximants
- Mathlib.ModelTheory.Semantics
- Mathlib.GroupTheory.Solvable
- Mathlib.Data.Nat.Factorization.Root
- Mathlib.Topology.UniformSpace.UniformEmbedding
- Mathlib.LinearAlgebra.Basis

So far I don't even have a guess what has caused it. lean#4352 seems to be the only plausible suspect amongst the changes in this nightly.

Kim Morrison (Jun 05 2024 at 09:30):

Unfortunately it wasn't tested separately.

Ruben Van de Velde (Jun 05 2024 at 09:31):

Did you fix error: ././././Mathlib/Init/Core.lean:152:27: Declaration IsLawfulSingleton not found. already?

Kim Morrison (Jun 05 2024 at 09:31):

Yes, sorry, just pushed some easy changes.

Kim Morrison (Jun 05 2024 at 09:32):

(the various upstreams and renames)

Kim Morrison (Jun 05 2024 at 09:32):

I'm compiling lean#4352 locally to see if I can reproduce nightly-testing's troubles there. Probably it won't be possible to test separately because too many other things changed.

Kim Morrison (Jun 05 2024 at 09:38):

Yeah, it was lean#4352. I suspect this will require minimization and possibly some revisions at the Lean end, but I am jet-lagged and need to sleep!

github mathlib4 bot (Jun 05 2024 at 09:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Jun 05 2024 at 10:13):

I pushed a few workarounds with adaptation notes; not yet all of the files you listed

github mathlib4 bot (Jun 05 2024 at 10:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 05 2024 at 21:05):

Ruben Van de Velde said:

I pushed a few workarounds with adaptation notes; not yet all of the files you listed

Do you have a sense whether the workaround are reasonable? (i.e. previously the proofs were abusive in some way) Or if they likely indicate that we will need to go back and change lean#4352? I'll look later today.

Ruben Van de Velde (Jun 05 2024 at 21:11):

The ones I pushed were a bit disappointing, but probably not unreasonable. I guess it will depend on how many more of those are coming

github mathlib4 bot (Jun 05 2024 at 21:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 05 2024 at 23:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 06 2024 at 00:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 06 2024 at 00:18):

Nearly all fixed (there will be many backported changes to master; I'll prepare these soon).

Kim Morrison (Jun 06 2024 at 00:19):

The one remaining error is in Mathlib/Algebra/Lie/CartanExists.lean, where a simp_rw [coe_toEnd_pow] is no longer firing. Haven't quite worked this one out yet, so if any Lie theory enthusiasts (@Johan Commelin?) want to jump in that would be great. (Hopefully oleans available already?)

github mathlib4 bot (Jun 06 2024 at 00:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 06 2024 at 02:26):

Kim Morrison said:

The one remaining error is in Mathlib/Algebra/Lie/CartanExists.lean, where a simp_rw [coe_toEnd_pow] is no longer firing. Haven't quite worked this one out yet, so if any Lie theory enthusiasts (Johan Commelin?) want to jump in that would be great. (Hopefully oleans available already?)

Okay, sorted this one. Hopefully all working again.

github mathlib4 bot (Jun 06 2024 at 02:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 06 2024 at 02:56):

Some incoming problems from master.

github mathlib4 bot (Jun 06 2024 at 03:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 06 2024 at 04:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 06 2024 at 10:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 06 2024 at 11:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 06 2024 at 13:03):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 07 2024 at 10:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 08 2024 at 05:33):

Needs patches merged from lean-pr-testing-4370

github mathlib4 bot (Jun 08 2024 at 06:40):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 11 2024 at 10:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 11 2024 at 10:36):

I've merged patches for lean#4408 and lean#4385 that I prepared earlier.

github mathlib4 bot (Jun 11 2024 at 11:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 11 2024 at 16:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 11 2024 at 19:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 11 2024 at 22:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 12 2024 at 01:16):

Trying out the fix proposed at https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/v4.2E9.2E0-rc1.20discussion/near/444127287, but it is a bit voodoo so far.

github mathlib4 bot (Jun 12 2024 at 02:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 12 2024 at 04:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 12 2024 at 06:17):

Hopefully should come good again now that we are using @llllvvuu's batteries#838.

llllvvuu (Jun 12 2024 at 06:32):

We might have to address those linter warnings as well: #13754

(I might have awakened the linter by fixing a bug - my bad)

Kim Morrison (Jun 12 2024 at 06:35):

@llllvvuu, yes if you could send that to master that would be great. Ping me again and I'll merge!

llllvvuu (Jun 12 2024 at 06:40):

@Kim Morrison done

github mathlib4 bot (Jun 12 2024 at 07:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 12 2024 at 10:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 12 2024 at 13:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 12 2024 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 12 2024 at 18:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 12 2024 at 23:13):

Hopefully just needs lean-pr-testing-4421 merged in.

Kim Morrison (Jun 12 2024 at 23:36):

Also requires quite a few (positive!) fixes for lean4#4430.

github mathlib4 bot (Jun 13 2024 at 00:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 13 2024 at 00:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 13 2024 at 01:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 13 2024 at 01:59):

Ugh, my fault, after merging lean-pr-testing-4421 we were pointing to an old copy of Batteries.

github mathlib4 bot (Jun 13 2024 at 04:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 13 2024 at 04:45):

Failure in norm_num now from the universe permutation change: lean4#4408

Kim Morrison (Jun 13 2024 at 04:46):

Fix is easy enough, happily.

github mathlib4 bot (Jun 13 2024 at 05:02):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Jun 13 2024 at 05:04):

Hurrah! It's been a while. :-)

github mathlib4 bot (Jun 13 2024 at 06:49):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 14 2024 at 06:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 14 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 14 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 14 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 14 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 15 2024 at 06:50):

Hmm, I seem to have run into trouble here, with lake getting stuck.

@Mac Malone?

On the nightly-testing branch of Mathlib, I see:

% lake build
warning: manifest out of date: git url of dependency 'Cli' changed; use `lake update Cli` to update it
warning: manifest out of date: git revision of dependency 'Cli' changed; use `lake update Cli` to update it
 [?/?] Computing build jobs^C

with lake just hanging at that step.

I don't see anything wrong with Cli (and I'm pretty sure nothing has changed):

% lake update Cli
warning: ././.lake/packages/proofwidgets/lakefile.lean:22:20: warning: `Lake.inputFile` has been deprecated
warning: ././.lake/packages/proofwidgets/lakefile.lean:76:36: warning: `Lake.inputFile` has been deprecated
warning: Cli: ignoring missing dependency manifest '././.lake/packages/Cli/lake-manifest.json'
info: mathlib: running post-update hooks

doesn't result in any change to lake-manifest.json, and lake build hangs in the same manner.

I've tried the usual things of lake clean, and rm -rf .lake, to no avail.

Kim Morrison (Jun 15 2024 at 06:51):

(The warning about Lake.inputFile from ProofWidgets has been present for about a week: @Wojciech Nawrocki knows about it and is looking into it, so I think it is unrelated to today's problem.)

Kim Morrison (Jun 15 2024 at 09:36):

(Fully appreciating it is the weekend...) This is apparently completely blocking work on nightly-testing, so @Mac Malone I'd appreciate your help here on Monday! :-)

Mac Malone (Jun 15 2024 at 09:41):

Kim Morrison said:

warning: Cli: ignoring missing dependency manifest '././.lake/packages/Cli/lake-manifest.json'

This sticks out to me as odd as Cli has a lake-manifest.json . Does the file in question really not exist?

Kim Morrison (Jun 15 2024 at 09:42):

Yes, the file is missing.

Mac Malone (Jun 15 2024 at 09:43):

Well that's a problem. What does a rm -rf .lake and lake update Cli -v produce?

Kim Morrison (Jun 15 2024 at 09:44):

lean4-cli main is at a11566029bd9ec4f68a65394e8c3ff1af74c1a29, but git log in .lake/packages/Cli reports 39229f3630d734af7d9cfb5937ddc6b41d3aa6aa.

Kim Morrison (Jun 15 2024 at 09:44):

% rm -rf .lake
% lake update Cli -v
info: batteries: cloning https://github.com/leanprover-community/batteries to '././.lake/packages/batteries'
trace: .> git clone https://github.com/leanprover-community/batteries ././.lake/packages/batteries
trace: stderr:
Cloning into '././.lake/packages/batteries'...
trace: ././.lake/packages/batteries> git checkout --detach 8d2100637a91776707ca22636ae8aa04dd5c1e8d
trace: stderr:
HEAD is now at 8d21006 chore: bump to nightly-2024-06-15
info: Qq: cloning https://github.com/leanprover-community/quote4 to '././.lake/packages/Qq'
trace: .> git clone https://github.com/leanprover-community/quote4 ././.lake/packages/Qq
trace: stderr:
Cloning into '././.lake/packages/Qq'...
trace: ././.lake/packages/Qq> git checkout --detach 44f57616b0d9b8f9e5606f2c58d01df54840eba7
trace: stderr:
HEAD is now at 44f5761 bump toolchain
info: aesop: cloning https://github.com/leanprover-community/aesop to '././.lake/packages/aesop'
trace: .> git clone https://github.com/leanprover-community/aesop ././.lake/packages/aesop
trace: stderr:
Cloning into '././.lake/packages/aesop'...
trace: ././.lake/packages/aesop> git checkout --detach f744aab6fc4e06553464e6ae66730a3b14b8e615
trace: stderr:
HEAD is now at f744aab merge master, bump toolchain
info: proofwidgets: cloning https://github.com/leanprover-community/ProofWidgets4 to '././.lake/packages/proofwidgets'
trace: .> git clone https://github.com/leanprover-community/ProofWidgets4 ././.lake/packages/proofwidgets
trace: stderr:
Cloning into '././.lake/packages/proofwidgets'...
trace: ././.lake/packages/proofwidgets> git checkout --detach e6b6247c61280c77ade6bbf0bc3c66a44fe2e0c5
trace: stderr:
HEAD is now at e6b6247 Merge pull request #56 from leanprover-community/batteries
warning: ././.lake/packages/proofwidgets/lakefile.lean:22:20: warning: `Lake.inputFile` has been deprecated
warning: ././.lake/packages/proofwidgets/lakefile.lean:76:36: warning: `Lake.inputFile` has been deprecated
info: Cli: cloning https://github.com/mhuisi/lean4-cli to '././.lake/packages/Cli'
trace: .> git clone https://github.com/mhuisi/lean4-cli ././.lake/packages/Cli
trace: stderr:
Cloning into '././.lake/packages/Cli'...
trace: ././.lake/packages/Cli> git checkout --detach 39229f3630d734af7d9cfb5937ddc6b41d3aa6aa
trace: stderr:
HEAD is now at 39229f3 doc: adjust README for move to leanprover
warning: Cli: ignoring missing dependency manifest '././.lake/packages/Cli/lake-manifest.json'
info: importGraph: cloning https://github.com/leanprover-community/import-graph.git to '././.lake/packages/importGraph'
trace: .> git clone https://github.com/leanprover-community/import-graph.git ././.lake/packages/importGraph
trace: stderr:
Cloning into '././.lake/packages/importGraph'...
trace: ././.lake/packages/importGraph> git checkout --detach 7983e959f8f4a79313215720de3ef1eca2d6d474
trace: stderr:
HEAD is now at 7983e95 Merge pull request #12 from leanprover-community/bump_to_v4.9.0-rc1
info: mathlib: running post-update hooks

Kim Morrison (Jun 15 2024 at 09:46):

ah, for some reason we are getting 39229f3630d734af7d9cfb5937ddc6b41d3aa6aa from the nightly branch of lean4-cli, rather than the latest 10d88b52fa8d717fa8e29af3abf0c3a2bf175497.

Kim Morrison (Jun 15 2024 at 09:49):

Oh, is this because it is a transitive dependency via import-graph?

Kim Morrison (Jun 15 2024 at 09:51):

I bumped that at https://github.com/leanprover-community/import-graph/pull/13

Kim Morrison (Jun 15 2024 at 09:54):

I can not work out why lake is puling 39229f for lean4-cli.

Mac Malone (Jun 15 2024 at 09:54):

@Kim Morrison It appears to be getting it from batteries. I don't know why, though. This is something I specifically tested against, but something appears to be going wrong here for some reason.

Kim Morrison (Jun 15 2024 at 09:55):

What? But Batteries doesn't have any dependencies!

Mac Malone (Jun 15 2024 at 09:56):

What do you mean? https://github.com/leanprover-community/batteries/blob/main/lake-manifest.json

Mac Malone (Jun 15 2024 at 09:56):

(from doc-gen4)

Kim Morrison (Jun 15 2024 at 09:56):

Ugh... someone has committed in doc mode. I thought we didn't do this.

Patrick Massot (Jun 15 2024 at 09:57):

https://github.com/leanprover-community/batteries/blob/main/lakefile.lean#L21-L22

Kim Morrison (Jun 15 2024 at 09:57):

(meta if delenda est)

Mac Malone (Jun 15 2024 at 09:57):

I did that a while back as it is needed to figure out the doc-gen4 that is compatible with batteries.

Kim Morrison (Jun 15 2024 at 09:57):

Haha, @Mac Malone committed the lake-manifest.

Kim Morrison (Jun 15 2024 at 09:58):

We really need to get rid of that.

Kim Morrison (Jun 15 2024 at 09:58):

Batteries is not meant to have dependencies

Kim Morrison (Jun 15 2024 at 09:58):

If someone or something wants to run doc-gen4 on Batteries, they turn it on privately, and must not pollute everyone else's setup.

Kim Morrison (Jun 15 2024 at 09:59):

Do you know a reason why I can't commit the correct lake-manifest.json for Batteries without all this doc-gen stuff?

Mac Malone (Jun 15 2024 at 10:00):

However, I think I realized the test case I overlooked. It so happens that my test case tested the resolution order without dependency package manifests. Relooking at the code, I believe it breaks in the presence of them. I will fix this monday.

A quick fix is to move the CLI dependency to the top of the require block in mathlib.

Kim Morrison (Jun 15 2024 at 10:00):

I'm committing an empty lake-manifest to Batteries

Mac Malone (Jun 15 2024 at 10:02):

That can break things in a different way (and will likely be undone soon).

Kim Morrison (Jun 15 2024 at 10:03):

Okay, that gets rid of the warning about Cli, but the underlying problem remains:

% lake build
info: batteries: cloning https://github.com/leanprover-community/batteries to '././.lake/packages/batteries'
info: Qq: cloning https://github.com/leanprover-community/quote4 to '././.lake/packages/Qq'
info: aesop: cloning https://github.com/leanprover-community/aesop to '././.lake/packages/aesop'
info: proofwidgets: cloning https://github.com/leanprover-community/ProofWidgets4 to '././.lake/packages/proofwidgets'
warning: ././.lake/packages/proofwidgets/lakefile.lean:22:20: warning: `Lake.inputFile` has been deprecated
warning: ././.lake/packages/proofwidgets/lakefile.lean:76:36: warning: `Lake.inputFile` has been deprecated
info: importGraph: cloning https://github.com/leanprover-community/import-graph.git to '././.lake/packages/importGraph'
info: Cli: cloning https://github.com/leanprover/lean4-cli to '././.lake/packages/Cli'
 [?/?] Computing build jobs

Kim Morrison (Jun 15 2024 at 10:03):

Mac Malone said:

That can break things in a different way (and will likely be undone soon).

How can it break things? And why would it be undone?

Mac Malone (Jun 15 2024 at 10:04):

(Part of the require overhaul that I working on merging was unconditionally adding conditional dependencies to the manifest.)

Kim Morrison (Jun 15 2024 at 10:04):

Hmm, okay. We'll deal with that when we get there. Hopefully that is only a small window until lake install anyway. :-)

Kim Morrison (Jun 15 2024 at 10:05):

And in any case it seems that this problem is orthogonal to the actual blocker.

Mac Malone (Jun 15 2024 at 10:05):

The current problem is a bug in the resolution refactor (lean4#4371) that results in a change in the package resolution order that I had not intended (and I had tried to test to avoid).

Kim Morrison (Jun 15 2024 at 10:07):

(Sorry, "current problem" means getting stuck at "Computing build jobs"?)

Mac Malone (Jun 15 2024 at 10:08):

No, the CLI one.

I am not sure what would cause Lake to hang.

Mac Malone (Jun 15 2024 at 10:09):

I had hope the fixing the CLI bug would fix it but sadly apparently not.

Mac Malone (Jun 15 2024 at 10:14):

@Kim Morrison does lake build -v give any more info?

Kim Morrison (Jun 15 2024 at 10:18):

Unfortunately not.

Kim Morrison (Jun 15 2024 at 10:18):

Do you want to see if you can repro? It's just the nightly-testing branch of Mathlib.

Mac Malone (Jun 15 2024 at 10:21):

Sure. What was the last nightly that was known to not have this issue?

Mac Malone (Jun 15 2024 at 10:22):

Does running lake exe cache get work on machine? (It does on mine.)

Kim Morrison (Jun 15 2024 at 10:22):

Hmm, the tag nightly-testing-2024-06-12 definitely works, but there will be more in between.

Kim Morrison (Jun 15 2024 at 10:23):

lake exe cache get runs, but finds nothing.

Kim Morrison (Jun 15 2024 at 10:24):

Ahha!

Mac Malone (Jun 15 2024 at 10:24):

Its proofwidgets (run lake build proofwidgets to see)

Kim Morrison (Jun 15 2024 at 10:24):

Batteries.Lean.Name has been deleted

Kim Morrison (Jun 15 2024 at 10:24):

and removing all the import Batteries.Lean.Name lines causes lake build to not get stuck!

Mac Malone (Jun 15 2024 at 10:25):

Oh, so does any library depending on batteries break?

Kim Morrison (Jun 15 2024 at 10:25):

If you import that missing file?

Kim Morrison (Jun 15 2024 at 10:26):

That deletion was intentional

Kim Morrison (Jun 15 2024 at 10:26):

But lake shouldn't freeze because you import a file from another package that doesn't exist!

Mac Malone (Jun 15 2024 at 10:27):

I don't think it is freezing -- I think proofwidgets is being rebuilt.

Mac Malone (Jun 15 2024 at 10:27):

And since mathlib is using the old proofwidgets v0.0.36 which is not integrated with the new build monitor, no info is dispalyed.

Kim Morrison (Jun 15 2024 at 10:29):

Oh, hmm. I think I did leave it in this state for >1 hour this afternoon... but it's possible.

github mathlib4 bot (Jun 15 2024 at 10:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Mac Malone (Jun 15 2024 at 10:31):

I tried lake build <pkg> on mathlib's indiviual dependencies and the only that hangs is proofwidgets, hence my conjecture.

Kim Morrison (Jun 15 2024 at 10:31):

Well, having deleted these bad imports, I guess I am unstuck.

Kim Morrison (Jun 15 2024 at 10:31):

Hopefully I can leave it to you to work out any lake fixes warranted. :-)

Kim Morrison (Jun 15 2024 at 10:31):

And hopefully Wojciech will let us bump ProofWidgets soon. :-)

Mac Malone (Jun 15 2024 at 10:33):

Note that import graph also has the bad battiries import.

github mathlib4 bot (Jun 15 2024 at 11:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 15 2024 at 15:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 15 2024 at 19:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 15 2024 at 22:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 16 2024 at 00:11):

Tidying up some Name API had broken import-graph, so I had to update its nightly-testing branch and move Mathlib's nightly-testing to that.

github mathlib4 bot (Jun 16 2024 at 01:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 16 2024 at 01:47):

Should come good after #13855.

github mathlib4 bot (Jun 16 2024 at 02:40):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 16 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 16 2024 at 12:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 16 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 16 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 16 2024 at 23:10):

Again, merging lean-pr-testing-4400.

github mathlib4 bot (Jun 16 2024 at 23:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 16 2024 at 23:46):

Transient network error?

github mathlib4 bot (Jun 17 2024 at 01:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 17 2024 at 02:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 17 2024 at 08:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 17 2024 at 09:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 17 2024 at 10:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 17 2024 at 11:05):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 18 2024 at 01:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 18 2024 at 03:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 18 2024 at 07:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 18 2024 at 08:54):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Jun 18 2024 at 09:35):

I'm just fixing up for nightly-2024-07-18 now. There are some breakages, and I'm not entirely sure what Lean change caused them. Either lean#4481 or lean#4434 potentially?

Kim Morrison (Jun 18 2024 at 09:36):

The breakages are in Mathlib.Data.Matrix.PEquiv and Mathlib.Data.Finsupp.Basic.

Kim Morrison (Jun 18 2024 at 09:36):

I'm done with Mathlib for the day, so if anyone wanted to investigate that would be lovely, and otherwise I'll look more tomorrow.

github mathlib4 bot (Jun 18 2024 at 09:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 18 2024 at 13:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 18 2024 at 15:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 18 2024 at 18:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 18 2024 at 21:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 19 2024 at 10:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 19 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 19 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 19 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 19 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 19 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 20 2024 at 02:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 20 2024 at 02:29):

Kim Morrison said:

The breakages are in Mathlib.Data.Matrix.PEquiv and Mathlib.Data.Finsupp.Basic.

I've fixed this, but I'm confused what has gone wrong. It is a few instances where dsimp will no longer use a lemma, and we need to rw instead. I can't work out which underlying Lean change must be responsible.

Kim Morrison (Jun 20 2024 at 02:29):

For now I've worked around and left #adaptation_notes for someone in the future. :-)

Kim Morrison (Jun 20 2024 at 02:48):

Quite a few more changes needed downstream. I just added Pi.one_apply to simp sets freely to solve problems...

github mathlib4 bot (Jun 20 2024 at 03:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 20 2024 at 03:25):

Just a shake

github mathlib4 bot (Jun 20 2024 at 03:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 20 2024 at 03:44):

Oh dear, still many linter failures.

github mathlib4 bot (Jun 20 2024 at 04:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 20 2024 at 04:41):

Transient?

github mathlib4 bot (Jun 20 2024 at 05:35):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 21 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 21 2024 at 10:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 21 2024 at 11:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 21 2024 at 12:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 21 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 21 2024 at 18:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 21 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 22 2024 at 00:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 22 2024 at 09:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 22 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 22 2024 at 10:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 22 2024 at 12:02):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 22 2024 at 15:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 22 2024 at 18:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 22 2024 at 21:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 23 2024 at 00:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 23 2024 at 01:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 23 2024 at 10:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 23 2024 at 12:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 23 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 23 2024 at 18:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 23 2024 at 23:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 24 2024 at 00:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 24 2024 at 01:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 24 2024 at 01:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 24 2024 at 02:56):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Jun 24 2024 at 09:35):

Just merged branch#lean-pr-testing-4493, hopefully this is enough for today's update.

github mathlib4 bot (Jun 24 2024 at 10:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 24 2024 at 11:01):

Needed to fix some tests, now that the bodies of examples can not affect the universe levels appearing in the type signature.

github mathlib4 bot (Jun 24 2024 at 11:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 24 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 24 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 24 2024 at 18:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 24 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 25 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 25 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 25 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 25 2024 at 10:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 25 2024 at 10:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 25 2024 at 11:57):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 26 2024 at 00:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 26 2024 at 02:23):

The underlying failure here is that Batteries has made a Mathlib breaking change, and these land on nightly-testing first.

I'm trying to get the "automatically bump Batteries in Mathlib" automation going still, latest attempt at #14142

github mathlib4 bot (Jun 26 2024 at 03:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 26 2024 at 03:45):

and now #14143 ...

github mathlib4 bot (Jun 26 2024 at 06:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 26 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 26 2024 at 09:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 26 2024 at 10:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 26 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 26 2024 at 15:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 26 2024 at 18:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 27 2024 at 00:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 27 2024 at 03:27):

The problem now is that Aesop's nightly-testing branch need to have master branch merged into it!

Kim Morrison (Jun 27 2024 at 03:27):

(and bump the toolchain and Batteries)

Kim Morrison (Jun 27 2024 at 03:34):

Also required some universe reorderings due to different behaviour on nightly.

github mathlib4 bot (Jun 27 2024 at 04:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 27 2024 at 04:59):

Just some simp? says that no longer say spurious lemmas!

github mathlib4 bot (Jun 27 2024 at 05:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 27 2024 at 05:33):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 27 2024 at 10:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 27 2024 at 11:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 27 2024 at 13:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 27 2024 at 16:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 27 2024 at 19:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 27 2024 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 28 2024 at 01:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 29 2024 at 16:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jun 29 2024 at 17:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jun 30 2024 at 08:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jun 30 2024 at 08:44):

This was the unusedTactic linter successfully identifying an eta_reduce that had become unnecessary on nightly-testing. Nice!

github mathlib4 bot (Jun 30 2024 at 08:57):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 01 2024 at 10:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 01 2024 at 12:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 01 2024 at 12:24):

Needed a shake.

github mathlib4 bot (Jul 01 2024 at 13:42):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 03 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 03 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 03 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 03 2024 at 18:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 04 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 04 2024 at 02:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 04 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 04 2024 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 04 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 05 2024 at 00:09):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Jul 08 2024 at 17:14):

Sigh, the bot is down and not reporting that nightly-testing is currently failing. :-(

Ruben Van de Velde (Jul 08 2024 at 17:39):

It is?

Ruben Van de Velde (Jul 08 2024 at 17:39):

https://github.com/leanprover-community/mathlib4/commits/nightly-testing/ looks green

Kim Morrison (Jul 08 2024 at 17:46):

Oops, my mistake!

github mathlib4 bot (Jul 08 2024 at 19:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 08 2024 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 08 2024 at 22:03):

There's nothing to be done until lean4#4680 lands tonight.

github mathlib4 bot (Jul 09 2024 at 00:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kyle Miller (Jul 09 2024 at 03:44):

This commit has batteries fixes for lean4#4543, and this commit has mathlib fixes.

These don't build on their own, but they're cherry-pickable.

Kyle Miller (Jul 09 2024 at 03:48):

Done, updated nightly-testing for batteries and mathlib

github mathlib4 bot (Jul 09 2024 at 03:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 06:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 09 2024 at 14:04):

Can someone help me here? I don't know how to cherry-pick the commit Kyle links to above

https://github.com/leanprover-community/batteries/commit/b1ae464adce816f24439b5830bda7a39c8381f9a

because I can't even find the commit anywhere...

Kim Morrison (Jul 09 2024 at 14:06):

Scratch that, Kyle has already done it.

Kim Morrison (Jul 09 2024 at 14:08):

@Mac Malone can you help me here? nightly-testing is consistently getting stuck at ⣿ [?/?] Computing build jobs, despite rm -rf .lake.

Kim Morrison (Jul 09 2024 at 14:08):

We're at f268021ae5575623c2737370dcf251e0010f0122

Kim Morrison (Jul 09 2024 at 14:09):

I'm unable to do anything on nightly-testing for now.

Mac Malone (Jul 09 2024 at 14:10):

@Kim Morrison Is this mathlib or batteries nightly-testing that is stuck?

Kim Morrison (Jul 09 2024 at 14:11):

Mathlib

Kim Morrison (Jul 09 2024 at 16:35):

Okay, we're running again. A file had been deleted in Batteries; removing the import causes lake to not hang. Mac is investigating.

github mathlib4 bot (Jul 09 2024 at 16:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 18:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 19:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 20:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 09 2024 at 22:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 09 2024 at 22:42):

Oof, problems in import-graph.

github mathlib4 bot (Jul 09 2024 at 23:47):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 10 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 10 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 10 2024 at 14:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 10 2024 at 16:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 10 2024 at 17:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 10 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 10 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 10 2024 at 22:13):

Gah, I keep doing this: I merged lean-pr-testing-4678, but forgot that this changed the Batteries dependency to the lean-pr-testing-4678 branch, and hence got a slightly out of sync Batteries.

github mathlib4 bot (Jul 10 2024 at 23:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kyle Miller (Jul 11 2024 at 00:49):

There's a simp "lhs simplifies" error for mathlib's docs#List.getLast?_append_cons

It's almost provable by the core simp lemma docs#List.getLast?_append, but it would be able to fully prove it if docs#List.getLast?_cons were a simp lemma too. It's in terms of getLastD though. Maybe this would be better, with some lemmas for handling Option.or expressions.

@[simp] theorem getLast?_cons' {a : α} {l : List α} :
    (a :: l).getLast? = l.getLast?.or (some a) := by
  cases l <;> rfl

Kim Morrison (Jul 11 2024 at 00:58):

Why not just (a :: l).getLast? = l.getLast?.getD a?

I would prefer that all the D functions unfold via simp to ? function followed by Option.getD.

Kim Morrison (Jul 11 2024 at 00:59):

It's clear that more thought it still required about List.getLastD, and I'll make sure to look at it soon.

Kyle Miller (Jul 11 2024 at 01:00):

Right now I'm seeing if mathlib builds without this simp lemma and I'll leave an adaptation note

Kyle Miller (Jul 11 2024 at 01:01):

Kim Morrison said:

Why not just (a :: l).getLast? = l.getLast?.getD a?

The lemma List.getLast?_append is in terms of Option.or, so I thought that it would be more convenient sticking with that sublanguage, but :shrug:

github mathlib4 bot (Jul 11 2024 at 02:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 11 2024 at 02:15):

Just needs a shake.

github mathlib4 bot (Jul 11 2024 at 03:10):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 11 2024 at 03:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 11 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 11 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 11 2024 at 13:34):

Builds and shakes locally, hopefully it will come green shortly.

github mathlib4 bot (Jul 11 2024 at 14:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 11 2024 at 19:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 11 2024 at 22:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 12 2024 at 07:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 12 2024 at 13:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 12 2024 at 13:30):

I'm afk for a few days, but this failure looks relatively fixable. The explicitness of pullback.fst/snd was just changed on master, but there were existing changes in nightly-testing and the automatic merge did the wrong thing.

Kim Morrison (Jul 12 2024 at 13:30):

Just taking a look at the errors and seeing if the current code in master works now may suffice.

github mathlib4 bot (Jul 12 2024 at 16:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 12 2024 at 19:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 12 2024 at 22:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 13 2024 at 01:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 13 2024 at 04:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 13 2024 at 07:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 13 2024 at 10:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 13 2024 at 13:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 13 2024 at 16:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 13 2024 at 19:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 13 2024 at 22:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 14 2024 at 00:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 14 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 14 2024 at 06:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 14 2024 at 09:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 14 2024 at 12:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 14 2024 at 16:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 14 2024 at 19:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 14 2024 at 22:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 15 2024 at 01:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 15 2024 at 03:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 15 2024 at 06:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 15 2024 at 09:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 15 2024 at 13:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 15 2024 at 16:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 15 2024 at 18:37):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Jul 15 2024 at 21:06):

Just merged master in bump/v4.11.0 and then that into nightly-testing, in preparation for making the next adaptation PR.

Kim Morrison (Jul 15 2024 at 21:06):

Both stages had quite a few (~10ish) merge conflicts, so presumably I've made a mistake somewhere and they will show up in a nightly-testing failure shortly. :-)

Kim Morrison (Jul 15 2024 at 21:07):

(Notice also that Lean's nightly releases have been in hiatus since the 12th, so when that resumes soon we'll have a bit of catching up to do.)

github mathlib4 bot (Jul 15 2024 at 22:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 15 2024 at 22:35):

Merging #14778 (after I fix it ...) should solve this.

github mathlib4 bot (Jul 15 2024 at 22:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 15 2024 at 23:11):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 16 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 16 2024 at 00:53):

Sigh...

Kim Morrison (Jul 16 2024 at 00:56):

A missing import, I'm not quite sure how that ended up missing. I guess lots has been hitting master today.

github mathlib4 bot (Jul 16 2024 at 01:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 16 2024 at 02:31):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 16 2024 at 11:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 16 2024 at 13:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 16 2024 at 15:02):

A failure from incoming changes from master. Opened lean#4758 to request a more actionable error message when we need @[ext (iff := false)].

github mathlib4 bot (Jul 16 2024 at 16:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 16 2024 at 16:54):

Just a shake --update.

github mathlib4 bot (Jul 16 2024 at 17:07):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 17 2024 at 10:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 17 2024 at 12:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 17 2024 at 13:24):

Just the upstreaming of TransGen replacing Lean's TC, it seems.

github mathlib4 bot (Jul 17 2024 at 14:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 17 2024 at 14:58):

Needed a shake.

Kim Morrison (Jul 17 2024 at 15:01):

hmm, and then some tactic import fixes.

github mathlib4 bot (Jul 17 2024 at 16:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 17 2024 at 16:22):

Just some ext_iff cleanup.

github mathlib4 bot (Jul 17 2024 at 16:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 17 2024 at 19:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 17 2024 at 19:50):

Fixed, bad merge when preparing #14846.

github mathlib4 bot (Jul 17 2024 at 20:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 18 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 18 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 18 2024 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 18 2024 at 17:18):

Hmm, not sure about the remaining errors. Something has changed in elaboration, going to look for relevant merged PRs!

Kim Morrison (Jul 18 2024 at 17:21):

lean#4722 seems the most likely candidate, and it wasn't tested against Mathlib.

@Kyle Miller, would you have a moment to look at nightly-testing and see if the errors are likely because of lean#4722?

Kim Morrison (Jul 18 2024 at 17:22):

Failures, all of the form "failed to elaborate eliminator, motive is not type correct", are in:

- Mathlib.MeasureTheory.Constructions.Pi
- Mathlib.RingTheory.ClassGroup
- Mathlib.MeasureTheory.Function.SimpleFuncDenseLp

Kim Morrison (Jul 18 2024 at 17:22):

Ah, solution seems to just be to remove some elab_as_elim attributes.

Kim Morrison (Jul 18 2024 at 17:23):

That fixes the latter two.

Kyle Miller (Jul 18 2024 at 17:23):

That's fascinating that these used to work despite having type incorrect motives

Kim Morrison (Jul 18 2024 at 17:23):

(Have to run for a moment.)

Kyle Miller (Jul 18 2024 at 17:24):

You can also add (motive := _) to turn off elab_as_elim. Maybe they're normally ok — it's not an indictment of the theorem, but the use

Kim Morrison (Jul 18 2024 at 17:29):

Okay, looks good now, thanks.

Kim Morrison (Jul 18 2024 at 18:02):

Backported removal of the two elab_as_elims as #14876.

Kyle Miller (Jul 18 2024 at 18:08):

Why are we removing those? They look fine as elab_as_elim at first glance.

Kyle Miller (Jul 18 2024 at 18:22):

For example, in MeasureTheory.Constructions.Pi you add an explicit motive argument:

theorem pi_of_empty {α : Type*} [Fintype α] [IsEmpty α] {β : α  Type*}
    {m :  a, MeasurableSpace (β a)} (μ :  a : α, Measure (β a)) (x :  a, β a := isEmptyElim) :
    Measure.pi μ = dirac x := by
  haveI :  a, SigmaFinite (μ a) := isEmptyElim
  refine pi_eq fun s _ => ?_
  rw [Fintype.prod_empty, dirac_apply_of_mem]
  exact isEmptyElim (p := _) (α := α) -- added `(p := _)` here

Kyle Miller (Jul 18 2024 at 18:42):

I'm fixing the motive problems right now and I'll push to nightly-testing

Kyle Miller (Jul 18 2024 at 18:49):

It seems that there's an issue with lean4#4722, which is that it's checking type correctness of the motive too early. I've left adaptation notes in nightly-testing for now.

github mathlib4 bot (Jul 18 2024 at 19:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 18 2024 at 22:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 19 2024 at 00:20):

Just long lines.

github mathlib4 bot (Jul 19 2024 at 00:43):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 19 2024 at 03:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 19 2024 at 06:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 19 2024 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 19 2024 at 10:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 19 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 19 2024 at 12:47):

Looks like #14850 didn't merge cleanly into nightly-testing, there are a bunch of imports to update.

github mathlib4 bot (Jul 19 2024 at 13:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 19 2024 at 17:16):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 19 2024 at 22:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 19 2024 at 22:37):

(I'm going to be afk for 48 hours.)

github mathlib4 bot (Jul 19 2024 at 23:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 20 2024 at 00:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 09:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 09:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 10:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 12:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 20 2024 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 09:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 10:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 12:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 12:37):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 21 2024 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 19:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 21 2024 at 21:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 21 2024 at 23:06):

Looks like just incoming changes from master.

Kim Morrison (Jul 21 2024 at 23:07):

Hopefully will come good shortly; builds locally.

github mathlib4 bot (Jul 21 2024 at 23:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 22 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 22 2024 at 11:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 22 2024 at 22:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 22 2024 at 23:18):

Failing because of LazyList deprecation in Batteries.

github mathlib4 bot (Jul 23 2024 at 01:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 23 2024 at 04:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 23 2024 at 06:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 23 2024 at 06:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 23 2024 at 11:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 23 2024 at 12:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 23 2024 at 13:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kyle Miller (Jul 23 2024 at 16:43):

Kim Morrison said:

lean#4722 seems the most likely candidate, and it wasn't tested against Mathlib.

I do know better than to change the elaborator without doing a full test against mathlib... but adding error detection seemed innocuous :face_with_diagonal_mouth:

Here's a postmortem: it turns out that the cases of elab_as_elim that broke were all using a set of features of the elabAsElim elaborator that individually had bugs but which together sort of canceled out. Adding the motive typechecking caused it to rightfully fail in one of the broken intermediate states. This is all fixed in lean4#4800, and I've eliminated the elab_as_elim adaptation notes.

The trigger was having an under-applied eliminator that had an explicitly supplied argument that was necessary for elaborating the type of an eliminator target, where that target was not supplied. It turned out that another adaptation fix we could have used was to remove such arguments, since they counterintuitively hindered elaboration!

github mathlib4 bot (Jul 23 2024 at 16:51):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 23 2024 at 21:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 23 2024 at 23:24):

Looks like it just needed an ext lemma in Scheme fixes, because of an incoming change from master.

github mathlib4 bot (Jul 23 2024 at 23:42):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 24 2024 at 19:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 24 2024 at 22:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 24 2024 at 23:46):

Just incoming changes from master interacting with changes to ext lemmas.

github mathlib4 bot (Jul 24 2024 at 23:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 24 2024 at 23:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 25 2024 at 00:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 25 2024 at 17:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 25 2024 at 19:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 25 2024 at 20:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 25 2024 at 20:59):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 25 2024 at 21:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 25 2024 at 22:25):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Jul 25 2024 at 22:35):

#15145 will result in this bot including commit SHAs in the messages.

github mathlib4 bot (Jul 25 2024 at 23:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 26 2024 at 00:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 26 2024 at 03:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 26 2024 at 04:03):

Needed an import tweak after changes on master.

github mathlib4 bot (Jul 26 2024 at 05:06):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 26 2024 at 08:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 26 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 26 2024 at 11:14):

Adjustments needed for upstreaming and new List lemmas

github mathlib4 bot (Jul 26 2024 at 11:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 26 2024 at 12:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 26 2024 at 13:06):

Some linting; new simp lemmas in core.

github mathlib4 bot (Jul 26 2024 at 14:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 26 2024 at 15:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 26 2024 at 19:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 26 2024 at 21:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 27 2024 at 00:52):

Just needed a shake, I think.

Kim Morrison (Jul 27 2024 at 00:53):

It would be nice to have a bot that could automate running shake --fix (perhaps falling back to shake --update if a subsequent lake build fails?)

github mathlib4 bot (Jul 27 2024 at 01:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 27 2024 at 05:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 27 2024 at 07:30):

More shaking required!

github mathlib4 bot (Jul 27 2024 at 08:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 27 2024 at 09:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 27 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kyle Miller (Jul 27 2024 at 17:38):

For the next nightly, here are a few fixes: https://github.com/leanprover-community/mathlib4/compare/nightly-testing...lean-pr-testing-4817

github mathlib4 bot (Jul 27 2024 at 18:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 27 2024 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 28 2024 at 00:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 28 2024 at 01:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 28 2024 at 03:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 28 2024 at 22:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 28 2024 at 22:09):

Incoming changes from master interacting with changes to ext

github mathlib4 bot (Jul 28 2024 at 22:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 29 2024 at 09:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Jul 29 2024 at 09:48):

Looks like bump/v4.11.0 needs a shake and a merge from master

Kim Morrison (Jul 29 2024 at 11:16):

Usually we don't fix bump/v4.X.0 directly (beyond a best effort merge from master), just make the next PR coming from a bump/nightly-YYYY-MM-DD green.

github mathlib4 bot (Jul 29 2024 at 12:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 29 2024 at 12:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 29 2024 at 13:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 29 2024 at 13:57):

This was a big adaptation, with a lot of stuff upstreamed. (And a few = replaced by == in low level List theorems, causing some disruption here in Mathlib.) Hopefully it is about to come green.

github mathlib4 bot (Jul 29 2024 at 14:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 30 2024 at 03:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 30 2024 at 06:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 30 2024 at 07:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 30 2024 at 09:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Jul 30 2024 at 10:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 30 2024 at 12:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Ruben Van de Velde (Jul 30 2024 at 12:38):

Afk for 6 hours probably, if someone else wants to

github mathlib4 bot (Jul 30 2024 at 12:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 30 2024 at 12:49):

Ah, oops, when I merged lean-pr-testing-4817 I missed up the batteries SHA.

github mathlib4 bot (Jul 30 2024 at 13:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

Kim Morrison (Jul 30 2024 at 13:55):

just a shake.

github mathlib4 bot (Jul 30 2024 at 14:10):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Kim Morrison (Jul 31 2024 at 03:21):

Note to self (or anyone): when Mathlib breaks tonight, merge nightly-testing-pre-2024-07-31 into nightly-testing, and reset the Batteries dependency back to nightly-testing.

github mathlib4 bot (Jul 31 2024 at 04:40):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Ruben Van de Velde (Jul 31 2024 at 08:49):

r? #15340

github mathlib4 bot (Jul 31 2024 at 09:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 31 2024 at 10:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 31 2024 at 11:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Jul 31 2024 at 12:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

Ruben Van de Velde (Jul 31 2024 at 13:54):

Can I also get a quick review on #15299 and #15368?

github mathlib4 bot (Jul 31 2024 at 13:55):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded!

github mathlib4 bot (Aug 01 2024 at 06:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed.

github mathlib4 bot (Aug 01 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2df7d9446f22706562263d8b55076dc073e10d02).

github mathlib4 bot (Aug 01 2024 at 11:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

Johan Commelin (Aug 01 2024 at 12:25):

Looks like something went wrong with inserting the commit hash

Kim Morrison (Aug 01 2024 at 13:00):

Sigh.

github mathlib4 bot (Aug 01 2024 at 14:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0139a899fdb48caffb0277abf97006b8dace569e).

Ruben Van de Velde (Aug 01 2024 at 14:28):

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0139a899fdb48caffb0277abf97006b8dace569e).

Looks like mathlib built but some file in batteries that we don't use, didn't

github mathlib4 bot (Aug 01 2024 at 16:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a33cf03c4f57826d8dcb653483916aaeb0b55e65).

github mathlib4 bot (Aug 01 2024 at 19:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (852c1ad8be5a7ea86187ef929ae0b18feb9cf3eb).

github mathlib4 bot (Aug 01 2024 at 22:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (246247f72011e56c8d1740763f0b070b1471f067).

Kim Morrison (Aug 01 2024 at 23:53):

Ruben Van de Velde said:

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0139a899fdb48caffb0277abf97006b8dace569e).

Looks like mathlib built but some file in batteries that we don't use, didn't

Trivial fix, include became a keyword. Not sure why the bot didn't complain about Batteries failing, however...

github mathlib4 bot (Aug 02 2024 at 00:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (35ccd78e25895200656760dd478f0ad21c6f9046).

Kim Morrison (Aug 02 2024 at 00:00):

Transient network error, restarted.

github mathlib4 bot (Aug 02 2024 at 01:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (35ccd78e25895200656760dd478f0ad21c6f9046).

github mathlib4 bot (Aug 02 2024 at 09:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (01959f98a3774783925316cdfa88343f49515bae).

github mathlib4 bot (Aug 02 2024 at 10:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (01959f98a3774783925316cdfa88343f49515bae).

github mathlib4 bot (Aug 02 2024 at 10:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (743a5e8b688cdb0cae231901dc222e469268d5a8)

Ruben Van de Velde (Aug 02 2024 at 11:24):

What's the timeline for merging the 4.11 bump?

github mathlib4 bot (Aug 02 2024 at 16:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

Kim Morrison (Aug 02 2024 at 22:53):

Ruben Van de Velde said:

What's the timeline for merging the 4.11 bump?

I'd been hoping to cut v4.11.0-rc1 from nightly-2024-08-02, but we're still making some last minute decisions about other things to go in. I think it is very likely that I'll cut it from nightly-2024-08-04 when I'm back at work on Monday.

github mathlib4 bot (Aug 03 2024 at 01:06):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 03 2024 at 09:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (76800560a1efa8663ed89214fc1196c97b89ff89)

github mathlib4 bot (Aug 03 2024 at 10:43):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 04 2024 at 16:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1f03949ae423ae9fb010318e73f8969e44288c92).

github mathlib4 bot (Aug 05 2024 at 01:31):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 05 2024 at 01:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1f03949ae423ae9fb010318e73f8969e44288c92).

github mathlib4 bot (Aug 05 2024 at 08:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8c4038b2507733e36fe8af2a3a92e662efb9fc0f).

github mathlib4 bot (Aug 05 2024 at 10:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5025874dc5f9f8dd1598190e60ef20dda7b42566).

github mathlib4 bot (Aug 05 2024 at 13:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5ff8d6041626a80e1385e3c49856513e8709d0aa).

github mathlib4 bot (Aug 07 2024 at 01:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c2f3c7e48850127da856a7da0f433e51cbeaf9e7).

github mathlib4 bot (Aug 07 2024 at 03:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c7dfc55407acc6697e2f8d8ece42887d9634a000).

github mathlib4 bot (Aug 07 2024 at 06:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (53f5571e327fb37c1da77b0ddd80289f1bde8890).

github mathlib4 bot (Aug 07 2024 at 09:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a38c21c21b5a747fb2ae8b1ff6e8adba89cfd207).

github mathlib4 bot (Aug 07 2024 at 12:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aeb3c05894d02069f1bc626babe6249945362bcf).

github mathlib4 bot (Aug 07 2024 at 15:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f0edccd743c8550bc00a713769d249bf8ad0e0d5).

github mathlib4 bot (Aug 07 2024 at 19:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bdfc2b33b94a81651385eaa46c1e410ed9e2fb97).

github mathlib4 bot (Aug 07 2024 at 21:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e860e3b8a9fe291681487172a0cb1f99303e3c8d).

github mathlib4 bot (Aug 08 2024 at 03:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f786e149de0df265c1ffd26d3cc5dfb3767440e5).

github mathlib4 bot (Aug 08 2024 at 09:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15720c78a8142f7d35418f15b528bdb3f184989a).

github mathlib4 bot (Aug 08 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15720c78a8142f7d35418f15b528bdb3f184989a).

github mathlib4 bot (Aug 08 2024 at 11:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2edef7d509a7aeba89793a84905121a9f19171b6).

github mathlib4 bot (Aug 08 2024 at 11:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2edef7d509a7aeba89793a84905121a9f19171b6).

github mathlib4 bot (Aug 08 2024 at 12:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2edef7d509a7aeba89793a84905121a9f19171b6).

Kim Morrison (Aug 08 2024 at 12:22):

Hmm, I made a fair bit of progress (it involved updating all of batteries, quote4, aesop, and proofwidgets, phew!)

Kim Morrison (Aug 08 2024 at 12:23):

but there are still some mysterious errors here on nightly-testing, that will have to wait (for me, at least) until tomorrow.

github mathlib4 bot (Aug 08 2024 at 13:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2edef7d509a7aeba89793a84905121a9f19171b6).

github mathlib4 bot (Aug 08 2024 at 15:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a180e024b196dd867dd317c18b03cbc638d3d67e).

github mathlib4 bot (Aug 08 2024 at 18:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (71182adddbfdcb452d72959c4ddca10c54591de7).

github mathlib4 bot (Aug 08 2024 at 21:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (faf7c200e4b9b8220bec3e33b01f8494b7a7e1e5).

github mathlib4 bot (Aug 08 2024 at 23:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (faf7c200e4b9b8220bec3e33b01f8494b7a7e1e5).

github mathlib4 bot (Aug 09 2024 at 00:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (faf7c200e4b9b8220bec3e33b01f8494b7a7e1e5).

github mathlib4 bot (Aug 09 2024 at 01:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e8110d4997635efe76820a06ee6f009ada2ce683).

github mathlib4 bot (Aug 09 2024 at 03:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bc37ac3c35807d44e9caba747eeebb9171bbf802).

github mathlib4 bot (Aug 09 2024 at 04:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c37e54b849a33204619ff98c136c5a9fd0fe0cf2).

github mathlib4 bot (Aug 09 2024 at 04:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c37e54b849a33204619ff98c136c5a9fd0fe0cf2).

github mathlib4 bot (Aug 09 2024 at 07:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (01f726d5a3c5297f1bd3c4fc3b1219d96939d5d9)

github mathlib4 bot (Aug 09 2024 at 08:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a528f200ec83eae34a93fabb6270e0db1a8be8e4).

github mathlib4 bot (Aug 09 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a528f200ec83eae34a93fabb6270e0db1a8be8e4).

github mathlib4 bot (Aug 09 2024 at 11:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a528f200ec83eae34a93fabb6270e0db1a8be8e4).

github mathlib4 bot (Aug 09 2024 at 11:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a528f200ec83eae34a93fabb6270e0db1a8be8e4).

github mathlib4 bot (Aug 09 2024 at 12:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (74b685eb4a4f351a394e04504877bc7d133e8205).

github mathlib4 bot (Aug 09 2024 at 14:30):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (be8b9b9ab7bfa348400a35cdfabc27957f910d4e)

github mathlib4 bot (Aug 09 2024 at 16:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 10 2024 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a43394c090100a2ef35302ed549e9e60cac51516).

Kim Morrison (Aug 10 2024 at 10:34):

Oof, the new variable has arrived. :fingers_crossed: for merging lean-pr-testing-4814 into nightly-testing!

github mathlib4 bot (Aug 10 2024 at 13:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (be734717404579a0b842c06f1786335dc526b514)

github mathlib4 bot (Aug 10 2024 at 15:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 10 2024 at 21:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0077925cbead60622b55b430eb5109f7365954c8).

github mathlib4 bot (Aug 11 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (19796eea79b36c81ba5b1de34f5500e0348c84a2).

github mathlib4 bot (Aug 11 2024 at 03:55):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 11 2024 at 09:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7e5b9c79c533fd8202193a1b9207a3d2f87ff9cc)

github mathlib4 bot (Aug 11 2024 at 10:37):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 11 2024 at 13:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0b0394f530ed451a7431d78fcf3832effcf080e8).

github mathlib4 bot (Aug 11 2024 at 18:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c78e6881c0732682e4bd15eb06ba55a5e1d7e810).

github mathlib4 bot (Aug 11 2024 at 22:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1c0bc97cf3db27c7843717ddb46f908eb84d987f).

github mathlib4 bot (Aug 12 2024 at 01:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (055d766c68bd10e70d7adf8fe87f44add3d806fa).

github mathlib4 bot (Aug 12 2024 at 02:30):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 12 2024 at 03:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e5d297f01115fdd418d45ee9a0f4ea5df7639835).

github mathlib4 bot (Aug 12 2024 at 06:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c4b300a09c200cb3d5bfca7e032f9c8a1379d86).

github mathlib4 bot (Aug 12 2024 at 08:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c4b300a09c200cb3d5bfca7e032f9c8a1379d86).

github mathlib4 bot (Aug 12 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c4b300a09c200cb3d5bfca7e032f9c8a1379d86).

github mathlib4 bot (Aug 12 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (81b928ca2905b3abbed5ef4c41dd561ac6e98055).

github mathlib4 bot (Aug 12 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2215b9e43b7cd64e43162ea8125a7f88f93ab85a).

github mathlib4 bot (Aug 12 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3a48abadbb2bb75b975e8eb6e6d59dc4178abcd).

github mathlib4 bot (Aug 12 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (68d96e18b0bbca45b0f3bcfb4555f5766eff6a32).

github mathlib4 bot (Aug 13 2024 at 02:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dcf33608c8706b1ee9e8a4d1a7e3e066282a036b)

github mathlib4 bot (Aug 13 2024 at 07:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 13 2024 at 09:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7a9da2458527a3d008be0c061e897623fec034a5)

github mathlib4 bot (Aug 13 2024 at 10:38):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 13 2024 at 22:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d694ae6caaa2c0c7d98cd73a995c6a7d808c0c25).

github mathlib4 bot (Aug 14 2024 at 00:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15f92d5ddaf35f96f002e041f5cf7def7d2c5c1c).

github mathlib4 bot (Aug 14 2024 at 01:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15f92d5ddaf35f96f002e041f5cf7def7d2c5c1c).

github mathlib4 bot (Aug 14 2024 at 01:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15f92d5ddaf35f96f002e041f5cf7def7d2c5c1c).

github mathlib4 bot (Aug 14 2024 at 02:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15f92d5ddaf35f96f002e041f5cf7def7d2c5c1c).

github mathlib4 bot (Aug 14 2024 at 03:35):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 14 2024 at 08:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (077d38eee589991c0b64ca315d0166286ec428e2).

github mathlib4 bot (Aug 14 2024 at 09:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (077d38eee589991c0b64ca315d0166286ec428e2).

github mathlib4 bot (Aug 14 2024 at 12:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b74124c74c234d628473646ae4e5f851b4d64f16).

github mathlib4 bot (Aug 14 2024 at 15:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5e8e4a238e119f36df439c824802a60c6dd2bef9).

github mathlib4 bot (Aug 14 2024 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (508aeb0a850841872c7a54d33b2b629ed87542ac).

github mathlib4 bot (Aug 14 2024 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7a75f1dfdbf1e153e9f09695117f3d67fbac423d).

github mathlib4 bot (Aug 15 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0458ef860b78346c2bde5f2a56e45d35af21fda0).

github mathlib4 bot (Aug 15 2024 at 02:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (08ecf4c7e62daf335fa2f9e42d6ad90574211eb5).

github mathlib4 bot (Aug 15 2024 at 05:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (08ecf4c7e62daf335fa2f9e42d6ad90574211eb5).

github mathlib4 bot (Aug 15 2024 at 08:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b8ad879889282e043c011bdf4643eb4af5e3f99f)

github mathlib4 bot (Aug 15 2024 at 10:14):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 15 2024 at 17:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (28a935cb927c6f2c8a0e27d90ab79892fa042af5).

github mathlib4 bot (Aug 15 2024 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a2c3bef6080c5ed16bdf8daaf6e723e3da52834c).

github mathlib4 bot (Aug 15 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b73e0accb1f783c3f3347523a90b7eecba0b150f).

github mathlib4 bot (Aug 15 2024 at 23:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c98ad2f61380a2c6a894fd76473450c05147c7d4).

github mathlib4 bot (Aug 15 2024 at 23:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c98ad2f61380a2c6a894fd76473450c05147c7d4).

github mathlib4 bot (Aug 16 2024 at 00:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7a3e6979684c0f6f30bd9b8896b54e472cf153ae).

github mathlib4 bot (Aug 16 2024 at 01:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dc5804b64c1d397a30ef524d1a85a4557944f3fd).

github mathlib4 bot (Aug 16 2024 at 03:02):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (626dfe1a5ad9509244c7dbd82d36e803b8995f46)

github mathlib4 bot (Aug 16 2024 at 04:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (https://github.com/leanprover-community/mathlib4/commit/)

github mathlib4 bot (Aug 16 2024 at 08:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (07a0ae9126dff1d2838a59b03ac6763e22ed6cb4).

github mathlib4 bot (Aug 16 2024 at 09:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a6b7481a9abf30111d5efb2a336f2a1137857cc5).

github mathlib4 bot (Aug 16 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f66c0d7d3e938a825479b94afc611e50c92bfd49).

github mathlib4 bot (Aug 16 2024 at 14:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7e532b5232b22bddd9d2122a6f27862c1fb81046).

github mathlib4 bot (Aug 16 2024 at 15:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d03203d6da0a936fb8aabe8618f38a35d983b5d1).

github mathlib4 bot (Aug 16 2024 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (249c5361016c6265d2c82d9e24fa4702b713f11d).

github mathlib4 bot (Aug 16 2024 at 21:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (224578708b4f82f7a3cbdd4f506a7ff98a337364).

github mathlib4 bot (Aug 16 2024 at 22:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (537997c9ab39c53e49e52947399dbf0c9239d353).

Kim Morrison (Aug 16 2024 at 22:38):

Haha, thoroughly broken, induction' is now naming all the hypotheses in reverse order. Haven't work out what caused this yet, and off for orienteering :woman_running_facing_right: for the morning!

Ruben Van de Velde (Aug 16 2024 at 22:43):

Oh no

Kim Morrison (Aug 16 2024 at 22:43):

I had a quick look through the recent Lean 4 commits, and don't yet see anything that touched induction internals.

Ruben Van de Velde (Aug 16 2024 at 22:44):

Only about ~1600 uses of induction', we could replace them all overnight, right?

Kim Morrison (Aug 16 2024 at 22:44):

Haha no, something must have moved under induction''s feet, we'll find it. :-)

Kim Morrison (Aug 16 2024 at 22:50):

Oh, maybe it is a problem in batteries

Kim Morrison (Aug 16 2024 at 22:50):

Updating Mathlib master to Batteries main has the same symptoms.

Mario Carneiro (Aug 16 2024 at 22:51):

did I mess something up?

Mario Carneiro (Aug 16 2024 at 22:51):

I'm currently clearing the batteries queue, LMK if something needs my attention

Kim Morrison (Aug 16 2024 at 22:52):

Running lake update in Mathlib causes induction' to name hypotheses backwards.

Kim Morrison (Aug 16 2024 at 22:52):

About to run out the door for most of the day, not sure if I'll get further diagnosing than that.

Mario Carneiro (Aug 16 2024 at 22:52):

how could that be a batteries issue, it doesn't even have induction'

Kim Morrison (Aug 16 2024 at 22:53):

cases' too

Mario Carneiro (Aug 16 2024 at 22:53):

I'll look into it, enjoy your run

Ruben Van de Velde (Aug 16 2024 at 23:00):

Found it

Ruben Van de Velde (Aug 16 2024 at 23:01):

induction' uses splitAtD which reverses since https://github.com/leanprover-community/batteries/pull/919 by one @Kim Morrison

Mario Carneiro (Aug 16 2024 at 23:04):

pushed a fix

github mathlib4 bot (Aug 17 2024 at 01:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0dd5858ed899ab9af9621480ca63655b01548c29).

Kim Morrison (Aug 17 2024 at 02:15):

Oops. :-) Apparently I got splitAt right, but splitAtD wrong? Need some lemmas! :-)

Kim Morrison (Aug 17 2024 at 02:27):

Actually, why is the [] case there in splitAt.go? It makes the signature awkward by pulling in l. batteries#921

Kim Morrison (Aug 17 2024 at 02:33):

I added a theorem too, replacing a very messy proof down in Mathlib.

Mario Carneiro (Aug 17 2024 at 02:38):

that was there for a reason... it's so that it returns the input unchanged instead of rebuilding it

Kim Morrison (Aug 17 2024 at 02:39):

I don't understand: it was still running through all of l though, what would it save?

Mario Carneiro (Aug 17 2024 at 02:41):

it returns an object pointer-equal to the original

Kim Morrison (Aug 17 2024 at 02:41):

Hmm, okay. I can change it back, but have to be afk for a bit now.

Kim Morrison (Aug 17 2024 at 02:42):

It's a bit unusual to do this, e.g. we don't do it in take.

Kim Morrison (Aug 17 2024 at 02:42):

Was there a particular reason to do it here?

Mario Carneiro (Aug 17 2024 at 02:42):

batteries does it consistently

Kim Morrison (Aug 17 2024 at 02:44):

Hmm. I'd be interested to see other examples and/or evidence that it really helps. I'm open to the idea, but it does come at a slight cost on the verification side.

Mario Carneiro (Aug 17 2024 at 02:45):

obviously circa 6 months ago there is no way I'm making a PR to core to fix list methods to do this

Kim Morrison (Aug 17 2024 at 02:45):

(Sorry for moving precipitiously on that PR; I may not have a lot of time this weekend and wanted to try getting nightly-testing green again. I'll have time to come back to this later.)

Mario Carneiro (Aug 17 2024 at 02:45):

batteries doesn't optimize for ease of verification of internal invariants

Kim Morrison (Aug 17 2024 at 02:46):

I'd love to see a case study or benchmark demonstrating a gain; if it's really there I'm game to take advantage of it.

github mathlib4 bot (Aug 17 2024 at 02:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd0dba7f3a926163728a44e4a29507cf14474e3c).

github mathlib4 bot (Aug 17 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd0dba7f3a926163728a44e4a29507cf14474e3c).

github mathlib4 bot (Aug 17 2024 at 04:43):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ab5eb1f399ea2e8d4ea27c7bc61b27364217fbef)

github mathlib4 bot (Aug 17 2024 at 07:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3805ed6e8b8a81617ebfe7db6b0dbe9862075594).

github mathlib4 bot (Aug 17 2024 at 08:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3805ed6e8b8a81617ebfe7db6b0dbe9862075594).

github mathlib4 bot (Aug 17 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3805ed6e8b8a81617ebfe7db6b0dbe9862075594).

github mathlib4 bot (Aug 17 2024 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b2af0a88e4928979df8926e973e7175f7bcecc52).

github mathlib4 bot (Aug 17 2024 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aae0e915a7ea38179de2a1dfb4c1eeb830e1be4b).

github mathlib4 bot (Aug 17 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ee9adf282e4a53845c94b42073dd67b8d816dfa1).

github mathlib4 bot (Aug 17 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f94496f04c5cce69012ed0a9bcd62ae064576d74).

github mathlib4 bot (Aug 18 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (afd4d849e5cf6d8b456b03f7a8eba088b69be393).

github mathlib4 bot (Aug 18 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6ad8df9e3d0e236db6708d8819da132935f9b752).

github mathlib4 bot (Aug 18 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bbc4793a86a022d3c00f327b678e2725d95a21af).

github mathlib4 bot (Aug 19 2024 at 00:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5dccde47166d00d485a5d6ad8cc3cb4431edcb38).

github mathlib4 bot (Aug 19 2024 at 03:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (74ed7693458847faae657f3489f6d1d228607280).

github mathlib4 bot (Aug 19 2024 at 04:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (74ed7693458847faae657f3489f6d1d228607280).

github mathlib4 bot (Aug 19 2024 at 05:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e82727aab149b1515caa9c29547ebf629b9bb195)

github mathlib4 bot (Aug 19 2024 at 09:25):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3b7ff954eebc4f837bfd98fc2aba23a79ec7affb)

github mathlib4 bot (Aug 19 2024 at 21:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (be86c9939f1613ff2587566ab390f3d1610950c1).

Kim Morrison (Aug 20 2024 at 00:26):

Runner failed because it was out of space. I've restarted.

github mathlib4 bot (Aug 20 2024 at 00:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (35c50a55b4e1b6c43f1122d26a842a3003793797).

github mathlib4 bot (Aug 20 2024 at 01:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (35c50a55b4e1b6c43f1122d26a842a3003793797).

Kim Morrison (Aug 20 2024 at 01:24):

Woah, failed with:

System.ArgumentOutOfRangeException: Specified argument was out of the range of valid values. (Parameter ''using: node20' is not supported, use 'docker', 'node12' or 'node16' instead.') at GitHub.Runner.Worker.ActionManife

Not sure what that is about. I've restarted and am hoping it goes away?

Yakov Pechersky (Aug 20 2024 at 01:34):

https://github.com/actions/runner/issues/2619

Yakov Pechersky (Aug 20 2024 at 01:34):

Not sure which action procced the error

Kim Morrison (Aug 20 2024 at 01:35):

Wojciech was just rebooting the Hoskinson runners, it seems to have been a transient issue from that.

Yakov Pechersky (Aug 20 2024 at 01:36):

Possibly it was caught in an out of date GitHub runner state :)

github mathlib4 bot (Aug 20 2024 at 02:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3b7ff954eebc4f837bfd98fc2aba23a79ec7affb)

github mathlib4 bot (Aug 20 2024 at 03:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e0c470ac1765a2479763f07753cef18f685b7133).

github mathlib4 bot (Aug 20 2024 at 06:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2b86f5b2281ad282bd3ef8dc24ce1ba50d269c65).

github mathlib4 bot (Aug 20 2024 at 08:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2b86f5b2281ad282bd3ef8dc24ce1ba50d269c65).

github mathlib4 bot (Aug 20 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (63c2523fb9294684c4ed11bdbf24d200909a908b).

github mathlib4 bot (Aug 20 2024 at 11:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5f2879ac9e132974c6e229f6139d2d0ab2fdd4dd).

github mathlib4 bot (Aug 20 2024 at 12:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5f2879ac9e132974c6e229f6139d2d0ab2fdd4dd).

Kim Morrison (Aug 20 2024 at 12:32):

There's now a new mergeSort in Lean 4, which is unlike the Batteries (merge) + Mathlib (mergeSort) version is stable (i.e. doesn't reorder equivalent elements).

However it's not a drop-in replacement, because it uses a X -> X -> Bool sort order, rather than a DecidableRel. (And doesn't use the IsTrans / IsTotal / IsAntisymm classes.)

For now, I am just going to rename all the Mathlib declarations with a prime mergeSort', etc, and immediately stitch these back together again.

Johan Commelin (Aug 20 2024 at 12:35):

sorry for being dense, what do you mean with the stitching back together?

Kim Morrison (Aug 20 2024 at 12:35):

We should just be able to throw out Mathlib's List.mergeSort' and use List.mergeSort from Lean 4.

Kim Morrison (Aug 20 2024 at 12:36):

However because of the difference between X -> X -> Prop and X -> X -> Bool this isn't trivial.

Kim Morrison (Aug 20 2024 at 12:38):

I'm not entirely certain of the solution:

  1. Just jump through the hoops of using the Bool version during the limited use required in Mathlib.
  2. attribute [local instance] boolPredToPred might be helpful?
  3. Perhaps decide to upstream IsTrans / IsTotal / IsAntisymm, and use those in the Lean4 theorems about mergeSort?

Johan Commelin (Aug 20 2024 at 12:42):

Aha. I think I don't have an opinion on any of those.

github mathlib4 bot (Aug 20 2024 at 13:47):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7ae246da82c3e747578f861e28e0cafa801ef711)

Ruben Van de Velde (Aug 20 2024 at 16:21):

Where do we use mathlib mergesort?

github mathlib4 bot (Aug 20 2024 at 19:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7ae246da82c3e747578f861e28e0cafa801ef711)

Kim Morrison (Aug 21 2024 at 00:02):

Ruben Van de Velde said:

Where do we use mathlib mergesort?

The only places that broke were setting up sort on Multiset, which in turn is only really used for the Repr instance. I didn't look carefully beyond that.

github mathlib4 bot (Aug 21 2024 at 00:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eb4b9428cd30375c27d434763e6f9de49a1da22c).

Johan Commelin (Aug 21 2024 at 02:33):

Finset.sort maybe uses it?

Kim Morrison (Aug 21 2024 at 03:14):

We will need to merge lean-pr-testing-5103 into nightly-testing tonight.

github mathlib4 bot (Aug 21 2024 at 03:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dcea6223d996f15ef4bf33dd7c597125a500c972).

Kim Morrison (Aug 21 2024 at 04:35):

also lean-pr-testing-5104

github mathlib4 bot (Aug 21 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (40f53e8a4bc4df18869668009d2ccd2ac15f4593).

github mathlib4 bot (Aug 21 2024 at 07:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (40f53e8a4bc4df18869668009d2ccd2ac15f4593).

github mathlib4 bot (Aug 21 2024 at 08:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2db1a34225d4b394f5e8f6744b59d55fc0baeb18).

github mathlib4 bot (Aug 21 2024 at 10:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (22e3994a32b5b88e8d81124b3e4ee1accbd00bd6).

Kim Morrison (Aug 21 2024 at 10:59):

Merged changes for #5103 and #5104.

Kim Morrison (Aug 21 2024 at 11:00):

Tomorrow, then, we'll need to merge lean-pr-testing-5102 and lean-pr-testing-5106.

github mathlib4 bot (Aug 21 2024 at 12:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (2f0739b82177aca39b85f7a6a5dfec6bef27f90f)

github mathlib4 bot (Aug 21 2024 at 22:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fc10eda313842ba732a6783f2cc634e3e307183e).

github mathlib4 bot (Aug 22 2024 at 01:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (25040ca7ee3241a452efbd6b7ee2e64b56a85513).

github mathlib4 bot (Aug 22 2024 at 04:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (25040ca7ee3241a452efbd6b7ee2e64b56a85513).

github mathlib4 bot (Aug 22 2024 at 05:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (2f0739b82177aca39b85f7a6a5dfec6bef27f90f)

github mathlib4 bot (Aug 22 2024 at 09:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7ed205ef984ad7571fa0d6f21e444be1731d200b).

Kim Morrison (Aug 22 2024 at 09:30):

Hmm, ran into an issue, #5126.

Kevin Buzzard (Aug 22 2024 at 09:54):

lean#5126

github mathlib4 bot (Aug 22 2024 at 10:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (bc78dd4064260799592666fb0013b04d7a69f4c6)

github mathlib4 bot (Aug 23 2024 at 08:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cae1b27ace5330f372b57f1051e228fe9b264d57).

github mathlib4 bot (Aug 23 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cae1b27ace5330f372b57f1051e228fe9b264d57).

github mathlib4 bot (Aug 23 2024 at 11:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b44ac12891226d0505df9595922aee44c46ed53e).

github mathlib4 bot (Aug 23 2024 at 12:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b0278f55cafee986abe1882e4ad0ec346f0fd9f9).

github mathlib4 bot (Aug 23 2024 at 13:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (faaca26a2c8fedf29de68375b439071ed6034e73).

github mathlib4 bot (Aug 23 2024 at 15:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5a4b605e9b5b793a0ea1fa648acd5400d3c4bf95).

github mathlib4 bot (Aug 23 2024 at 19:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6e23e47597afc030e36c0e4fab9d1473a420eb62).

github mathlib4 bot (Aug 23 2024 at 21:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca6a6fdc075f392d6d38c787d5f02f1aa61acfbc).

github mathlib4 bot (Aug 24 2024 at 04:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca6a6fdc075f392d6d38c787d5f02f1aa61acfbc).

github mathlib4 bot (Aug 24 2024 at 05:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (2b617ccc55051120657715a15bc52a6def10b03c)

github mathlib4 bot (Aug 24 2024 at 08:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca6a6fdc075f392d6d38c787d5f02f1aa61acfbc).

github mathlib4 bot (Aug 24 2024 at 09:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca6a6fdc075f392d6d38c787d5f02f1aa61acfbc).

github mathlib4 bot (Aug 24 2024 at 12:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (cf3b406e1eb61883ac6c23c4cd309f305240007c)

Kim Morrison (Aug 25 2024 at 07:02):

Need to merge lean-pr-testing-5151 tonight.

github mathlib4 bot (Aug 25 2024 at 08:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bf2d126d0b5fd0ed489eb0d562781a2116e1e4c2).

github mathlib4 bot (Aug 25 2024 at 10:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (55eed64af62e8326dd5bdcabedf20ea2ec0a9f2a).

github mathlib4 bot (Aug 25 2024 at 11:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d0e15f37f36d63abacef01b9687a26d35ee5260a).

github mathlib4 bot (Aug 25 2024 at 12:35):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (74dc3f9df45b8768b3662c978c25cdf9de8f17b1)

Kim Morrison (Aug 26 2024 at 02:16):

We'll need lean-pr-testing-5160 tonight. Also 5163 and 5162.

github mathlib4 bot (Aug 26 2024 at 04:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (74dc3f9df45b8768b3662c978c25cdf9de8f17b1)

github mathlib4 bot (Aug 26 2024 at 08:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d011eb150be9174beb66ab43bae0ae39addb9bea).

github mathlib4 bot (Aug 26 2024 at 08:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ec00a8f1a1c8b2c2a8f71626847bf97b814eedf8).

github mathlib4 bot (Aug 26 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ec00a8f1a1c8b2c2a8f71626847bf97b814eedf8).

Kim Morrison (Aug 26 2024 at 09:45):

Forgot to push! :woman_facepalming:

github mathlib4 bot (Aug 26 2024 at 09:59):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5608be6564551cffcaf5048d7a3ff5330225e5b8)

github mathlib4 bot (Aug 26 2024 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b5f7e1c26c6cb2be97c2ad36bf7038c159e359b3).

Kim Morrison (Aug 26 2024 at 22:54):

Wow, everything is broken. (quote4, aesop, batteries, mathlib)

Kim Morrison (Aug 26 2024 at 22:57):

oh, just the lakefile is messed up

github mathlib4 bot (Aug 26 2024 at 23:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cbe86e0d47de1e6c520ba10227801ae6507b5806).

github mathlib4 bot (Aug 27 2024 at 02:45):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5608be6564551cffcaf5048d7a3ff5330225e5b8)

github mathlib4 bot (Aug 27 2024 at 08:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (99d679b4aee9537ea6e5faa22aa3896ce4c91444).

github mathlib4 bot (Aug 27 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ba7a809408aae010a202e38d72936f14d8f99417).

github mathlib4 bot (Aug 27 2024 at 10:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (45e815c5edc12baa16b76deaa2438068de46f60d).

Kim Morrison (Aug 27 2024 at 11:00):

Still many errors in basic files. We have to add reduceCtorEq to many simp only statements, but the errors currently on the branch are not that. I don't see immediately what has changed, and may not have a chance to look until tomorrow, so if anyone feels like investigating a mystery... !

github mathlib4 bot (Aug 27 2024 at 11:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (45e815c5edc12baa16b76deaa2438068de46f60d).

github mathlib4 bot (Aug 27 2024 at 12:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bf1047068974f5ebc957a30d55f6ff5d3989f0d3).

github mathlib4 bot (Aug 27 2024 at 15:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a0f40a65cbacf56cba6412055afb18dfafcfe313).

github mathlib4 bot (Aug 27 2024 at 17:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca2b360151bc0a386a9ab6926e137e131c8c0cfd).

github mathlib4 bot (Aug 27 2024 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cc33cb3e55f5d5fe9349a46e6a9aeed0a6d193cb).

github mathlib4 bot (Aug 27 2024 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0fb4c9738c70dd974f160816f130078e808fd14a).

github mathlib4 bot (Aug 28 2024 at 00:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0935a3efa9a095b3498db84676b7fee4eec1f858).

Kim Morrison (Aug 28 2024 at 01:45):

Some of the breakages will need to wait on lean#5187.

Kim Morrison (Aug 28 2024 at 01:46):

@María Inés de Frutos Fernández and @Filippo A. E. Nuccio, would one of you be able to look at Mathlib.RingTheory.Valuation.AlgebraInstances on branch#nightly-testing. It is thoroughly broken, and I'm failing to see why.

Kim Morrison (Aug 28 2024 at 01:47):

(And apologies for subscribing you to this very boring channel. Feel free to unsubscribe again. :-)

github mathlib4 bot (Aug 28 2024 at 03:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (28bae8a509df8153663da5729ec079240eb18ed2).

github mathlib4 bot (Aug 28 2024 at 04:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5e87714ac146cae34fb76ba713bf7e74b9f7c7a5).

github mathlib4 bot (Aug 28 2024 at 06:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e5cd4b4f321f6b9714857cc7c3ca9297ba23f409).

github mathlib4 bot (Aug 28 2024 at 08:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e5cd4b4f321f6b9714857cc7c3ca9297ba23f409).

Filippo A. E. Nuccio (Aug 28 2024 at 09:03):

@Kim Morrison I found the problem and the fix: some instances are not automatically found any more. How do you want me to proceed? By opening a PR against master which is not currently needed but will be later on; or to push the fix to nightly-testing or anything else?

Ruben Van de Velde (Aug 28 2024 at 09:14):

Start with pushing the fix to nightly-testing

Filippo A. E. Nuccio (Aug 28 2024 at 09:18):

Done!

Kim Morrison (Aug 28 2024 at 09:30):

Thanks @Filippo A. E. Nuccio, that's very helpful. If you want to backport the change to master that's helpful too, but not essential.

Kim Morrison (Aug 28 2024 at 09:30):

(The main difference is whether the change shows up in its own commit to master, or as part of a big batch of changes on bump day.)

Filippo A. E. Nuccio (Aug 28 2024 at 09:33):

... well, opening a PR would take me 30 secs, since it is just two added lines. I confess I don't understand the details of this, so I leave it to you to tell me what you prefer :smile:

Kim Morrison (Aug 28 2024 at 09:35):

It's fine as is, thanks.

github mathlib4 bot (Aug 28 2024 at 10:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d0a9ca947996b4445409cdc846769bff65aa2999).

github mathlib4 bot (Aug 28 2024 at 11:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (33d4a4af3e67a4561bbb0dacdc9800fc8785fa44).

Kim Morrison (Aug 28 2024 at 11:23):

Invisible changes to emojis ... :-)

github mathlib4 bot (Aug 28 2024 at 11:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8397433488042b9adf0d37952a2cef2d0abb8cfa)

github mathlib4 bot (Aug 28 2024 at 19:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (acef93c91bde53df0b4d3eb208ce82ecff2b80ac).

github mathlib4 bot (Aug 29 2024 at 01:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6eb5bd61a5fad977409660b35258bf8153ec6445).

github mathlib4 bot (Aug 29 2024 at 04:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (076f780c6129a3ea4940fab0596b3c64b89c062d).

github mathlib4 bot (Aug 29 2024 at 06:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8397433488042b9adf0d37952a2cef2d0abb8cfa)

github mathlib4 bot (Aug 29 2024 at 06:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f0887abf32a12f3566ef60f73ca3b43c984ed81a).

github mathlib4 bot (Aug 29 2024 at 08:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a93d39d22ddf49cd011ef65ff8ab33f19ab58163).

github mathlib4 bot (Aug 29 2024 at 08:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11329efdbefd74bc02b9cc7544b189953c6fd7cc).

github mathlib4 bot (Aug 29 2024 at 09:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11329efdbefd74bc02b9cc7544b189953c6fd7cc).

github mathlib4 bot (Aug 29 2024 at 10:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11329efdbefd74bc02b9cc7544b189953c6fd7cc).

github mathlib4 bot (Aug 29 2024 at 11:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11329efdbefd74bc02b9cc7544b189953c6fd7cc).

github mathlib4 bot (Aug 29 2024 at 13:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6da6b5512d764c784ffef6f19bf5c3dfcec6d3f9).

github mathlib4 bot (Aug 29 2024 at 16:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (015472f59577e14c0d4465ceb8d89795134a65af).

github mathlib4 bot (Aug 29 2024 at 18:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (92f9ab8bc286d0d035c63dd386f598693be4cabf).

github mathlib4 bot (Aug 29 2024 at 21:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0844193bcedb553ac72342e6ac8b6ae9a5287a14).

Kim Morrison (Aug 29 2024 at 23:55):

Somehow there is an import loop?

error: build cycle detected:
  +Mathlib.Init:olean
  +Mathlib.Tactic.Linter.Lint:deps
  +Mathlib.Tactic.Linter.Lint:leanArts
  +Mathlib.Tactic.Linter.Lint:olean
  +Mathlib.Init:deps
  +Mathlib.Init:leanArts
  +Mathlib.Data.Nat.Notation:deps
  +Mathlib.Data.Nat.Notation:leanArts
  +Mathlib.Data.Nat.Notation:olean
  +Mathlib.Tactic.Linter.TextBased:deps
  +Mathlib.Tactic.Linter.TextBased:leanArts
  +Mathlib.Tactic.Linter.TextBased:olean
  +mathliblint-style»:deps
  +mathliblint-style»:leanArts
  +mathliblint-style»:c
  +mathliblint-style»:c.o.export
  +mathliblint-style»:c.o
  +mathliblint-style»:o
  mathliblint-style»:leanExe
  +Mathlib.Init:olean

Kim Morrison (Aug 29 2024 at 23:57):

And lake build just hangs at ⣿ [?/?] Computing build jobs. @Mac Malone, you might want to look at the above commit and see if you can identify why it is hanging? Even in the presence of import loops I thought that shouldn't happen.

Kim Morrison (Aug 29 2024 at 23:59):

Removing Mathlib.Init from Mathlib.Tactic.Linter.Lint seems to have fixed it. I'm not going to investigate further.

github mathlib4 bot (Aug 30 2024 at 01:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ea3ee6af494fcc4cbaab83222535f3c51d5ed461).

github mathlib4 bot (Aug 30 2024 at 03:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5c9109f1e3374f00eafacd4affb2ecbed8a521c1).

github mathlib4 bot (Aug 30 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5c9109f1e3374f00eafacd4affb2ecbed8a521c1).

github mathlib4 bot (Aug 30 2024 at 06:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5c9109f1e3374f00eafacd4affb2ecbed8a521c1).

github mathlib4 bot (Aug 30 2024 at 07:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f49cbbb9d3fa2bd13ebdf748587f3105fb998c68).

github mathlib4 bot (Aug 30 2024 at 09:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f49cbbb9d3fa2bd13ebdf748587f3105fb998c68).

github mathlib4 bot (Aug 30 2024 at 13:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3fb4b747d628e29772c3366d3816949dc5a07e48).

github mathlib4 bot (Aug 30 2024 at 16:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d83c091e0583288ea944304c5ca03115c6d2e776).

github mathlib4 bot (Aug 30 2024 at 19:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (813f45d118afbabc6f56e156c0796d67785dec38).

github mathlib4 bot (Aug 30 2024 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (968aead20dc339a53759909215b9d082eec20d85).

github mathlib4 bot (Aug 31 2024 at 01:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (44e298ccfa9426aaa9c3ffc7e139ed833ed420ca).

github mathlib4 bot (Aug 31 2024 at 08:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3fbbef3432df1055bf2afdd8f04082ab3e680f45).

github mathlib4 bot (Aug 31 2024 at 09:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3fbbef3432df1055bf2afdd8f04082ab3e680f45).

github mathlib4 bot (Aug 31 2024 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9748aeb7ecb6c9ad971fc9864cb75fdecdf1a5e5).

github mathlib4 bot (Aug 31 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (816c3ce1e9303c9bf68bdc1901e1641b585b9601).

github mathlib4 bot (Aug 31 2024 at 18:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a2abea1e72e1c20ca68aace68bd8b4bca02f0281).

github mathlib4 bot (Aug 31 2024 at 21:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dae5d2d4be3fc19ef7a9c1a3b784fecf76b04589).

github mathlib4 bot (Sep 01 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1cc0616978727e4d3e48b2ccde54b3a5327243d1).

github mathlib4 bot (Sep 01 2024 at 03:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (63cced2a6b7c4ed2afb8e6cdf7443d6dbcc975e0).

github mathlib4 bot (Sep 01 2024 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fc860709ca856260a44258347ab1779a1c2476f9).

github mathlib4 bot (Sep 01 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (06d443eab23c40af08453ebbcf97bd546f793a46).

github mathlib4 bot (Sep 01 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bceec0497e2858063cfdc794f7a9c777d2cf0277).

Kim Morrison (Sep 01 2024 at 23:24):

Offline all weekend. :-) :humpback_whale: Breakage doesn't look bad, hopefully back shortly.

github mathlib4 bot (Sep 02 2024 at 00:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (780bdc8ce37b762b58b11e8cd50d6232b9ef7bab).

github mathlib4 bot (Sep 02 2024 at 02:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2e0035068318c6433bf22063e470d666837e5f55).

github mathlib4 bot (Sep 02 2024 at 03:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8edf04f0977c3183d3b633792e03fd570be1777f).

github mathlib4 bot (Sep 02 2024 at 06:03):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d2a59c1717b96952920b6d524e98452e6207e8e1)

github mathlib4 bot (Sep 02 2024 at 07:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f43d6924ffa649dee16e93e0b8b70715327252ba).

github mathlib4 bot (Sep 02 2024 at 08:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (00df099f8ed42c12b35cdedcfbf1fde6c7413662).

github mathlib4 bot (Sep 02 2024 at 08:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (00df099f8ed42c12b35cdedcfbf1fde6c7413662).

github mathlib4 bot (Sep 02 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (00df099f8ed42c12b35cdedcfbf1fde6c7413662).

Kim Morrison (Sep 02 2024 at 11:20):

Merging lean-pr-testing-5227. 3.5% instruction count improvement incoming!

github mathlib4 bot (Sep 02 2024 at 12:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c04874b19dcffe9a39644a00d8be23b104ab7976).

github mathlib4 bot (Sep 02 2024 at 12:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0194b29f8e8bda212a44bbd34bf8b8c37a88db25).

github mathlib4 bot (Sep 02 2024 at 16:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f8afc330d092ff1a5abdaa07104164e783cba124).

github mathlib4 bot (Sep 02 2024 at 19:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fad568051fdc3d3b669c7843278094d5e7126800).

github mathlib4 bot (Sep 02 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab33bb5c271a057417993d6c38c0339fcafa0f1c).

github mathlib4 bot (Sep 03 2024 at 00:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b21451955e08c69f627055e9f7fcb78105c7507b)

github mathlib4 bot (Sep 03 2024 at 01:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4bb220d475bdd8da3778c0f73d6f60449929a221).

github mathlib4 bot (Sep 03 2024 at 02:59):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b21451955e08c69f627055e9f7fcb78105c7507b)

github mathlib4 bot (Sep 03 2024 at 08:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b191738f9875e429b3680fecf251652a03f77cee).

github mathlib4 bot (Sep 03 2024 at 10:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ba7dc41500c8e6b10775da7e2c62f172776926c9).

github mathlib4 bot (Sep 03 2024 at 13:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3a97fe99a8c8180b83efac3be780aa9342a2529c).

github mathlib4 bot (Sep 03 2024 at 15:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b8e23f0e68aedd151d681df5c966f64b0516282b).

github mathlib4 bot (Sep 03 2024 at 18:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b804674c8f6d8a3611b64ab36e5636b20b877459).

github mathlib4 bot (Sep 03 2024 at 21:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (91d155587e2c92d55afb8565687863555bfc300c).

Kim Morrison (Sep 03 2024 at 23:55):

Just needed lean-pr-testing-5228 merged.

Kim Morrison (Sep 03 2024 at 23:55):

(I also reset nightly-testing to match master. The old history is still available on the nightly-testing-YYYY-MM-DD tags.)

github mathlib4 bot (Sep 04 2024 at 01:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e5003139f419c2f87f122db01fe513dc34b784d3)

Kim Morrison (Sep 04 2024 at 03:06):

Hmm, the reminder bot didn't fire.

Bryan Gin-ge Chen (Sep 04 2024 at 03:11):

This might be the failed run: https://github.com/leanprover-community/mathlib4/actions/runs/10693508556/job/29643765613

github mathlib4 bot (Sep 04 2024 at 04:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e5003139f419c2f87f122db01fe513dc34b784d3)

Kim Morrison (Sep 04 2024 at 05:23):

Ahha! bump/v4.13.0 doesn't exist yet.

Kim Morrison (Sep 04 2024 at 05:23):

I guess that is okay to expect a human to do.

github mathlib4 bot (Sep 04 2024 at 05:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e5003139f419c2f87f122db01fe513dc34b784d3)

Kim Morrison (Sep 04 2024 at 05:37):

Hmm, it seems that not only bump/v4.13.0 has to exist, it needs to be on a nightly toolchain, otherwise the reminder script breaks.

github mathlib4 bot (Sep 04 2024 at 07:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e5003139f419c2f87f122db01fe513dc34b784d3)

github mathlib4 bot (Sep 04 2024 at 08:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ee3c8402eccc71786028ca6017afbabc062c7e33).

github mathlib4 bot (Sep 04 2024 at 08:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ee3c8402eccc71786028ca6017afbabc062c7e33).

github mathlib4 bot (Sep 04 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8ffca2e3dc174e47e8c1485fdcfc0aefa60aac1d).

Kim Morrison (Sep 04 2024 at 09:44):

I messed up the implicitness of arguments to ite_eq_right_iff, but these will revert tomorrow.

github mathlib4 bot (Sep 04 2024 at 10:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca494e4ebf0a0fe88fece8992fce8a2f48595c41).

github mathlib4 bot (Sep 04 2024 at 11:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (836a022752c7e6b6e393471e806b7d6f3de0d583).

github mathlib4 bot (Sep 04 2024 at 13:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (df80b0dd2548c76fbdc3fe5d3a96873dfd46c0dc).

github mathlib4 bot (Sep 04 2024 at 15:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (df80b0dd2548c76fbdc3fe5d3a96873dfd46c0dc).

github mathlib4 bot (Sep 04 2024 at 22:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0cf4af7d5425a51328f68d50fa2a8a0eb3933044).

github mathlib4 bot (Sep 05 2024 at 01:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (77f1a316718621d501b76280518655ff338d46b1).

github mathlib4 bot (Sep 05 2024 at 03:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b5a83ea0c40bb96f710a523dbf14796352c8ce31)

github mathlib4 bot (Sep 05 2024 at 08:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d6ca7ae2c9d2c513b5bffdf8870661596a302b64).

github mathlib4 bot (Sep 05 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9f9fa6c201a1b4dae2124fc04e7dab05f26b0f27).

github mathlib4 bot (Sep 05 2024 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3e18f1777d9adc6889ce44a51a451bbd54e691aa).

github mathlib4 bot (Sep 05 2024 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0445181569cd643b35186a80605b2c36d4ad8368).

github mathlib4 bot (Sep 05 2024 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (19f71879399780e2a3d1fa707169593f9facac18).

github mathlib4 bot (Sep 05 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f1e24ddc39307f7b3c9d8717d5a61a46cd8a8dc2).

github mathlib4 bot (Sep 05 2024 at 23:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (23475ea6b9362d20e7574f6575faf3e01587f368).

github mathlib4 bot (Sep 05 2024 at 23:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (05afde3d650f212c4c310e5c8e1276e9d458a04b).

github mathlib4 bot (Sep 06 2024 at 01:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b67303d4adb07719517e69a05ae97614aa349879).

github mathlib4 bot (Sep 06 2024 at 02:54):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dfbd837a1da3cc0257ec101c10561cb85c0ca325)

github mathlib4 bot (Sep 06 2024 at 07:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd6c31182d6b88c28e04d9bee8df7e6a54e279e4).

github mathlib4 bot (Sep 06 2024 at 08:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dfbd837a1da3cc0257ec101c10561cb85c0ca325)

github mathlib4 bot (Sep 06 2024 at 08:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd6c31182d6b88c28e04d9bee8df7e6a54e279e4).

github mathlib4 bot (Sep 06 2024 at 09:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3733a7d6b281e3747174fd89a25399abb9d74db8).

github mathlib4 bot (Sep 06 2024 at 11:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd286d4a4ae0633563f7b7f8cab33c43289877d5).

github mathlib4 bot (Sep 06 2024 at 12:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (24fce2d2db1a7ed39c8c5bdaf300d2ddfc83313f).

github mathlib4 bot (Sep 06 2024 at 13:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (24fce2d2db1a7ed39c8c5bdaf300d2ddfc83313f).

github mathlib4 bot (Sep 06 2024 at 13:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (24fce2d2db1a7ed39c8c5bdaf300d2ddfc83313f).

github mathlib4 bot (Sep 06 2024 at 16:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca6172cd68f7d0ed10ebeafe185369830a80a0a1).

github mathlib4 bot (Sep 06 2024 at 19:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a4b56a06989de44e5758843c8ee1557c39e8d313).

github mathlib4 bot (Sep 06 2024 at 21:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b0bb2eabcd30264cc87468a8ba6d1b898871e251).

github mathlib4 bot (Sep 06 2024 at 23:10):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8e11f3bb7182ebae9b94343eae182c6866962dad)

github mathlib4 bot (Sep 07 2024 at 08:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f90f08370493c760090c45a91fe9736556504346).

github mathlib4 bot (Sep 07 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ce32dd9cb55e73ae0b8f4340e4c8e8cd0ddf91e7).

github mathlib4 bot (Sep 07 2024 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (19b4c40bc454221b94bcaeb093d849639273e6cc).

github mathlib4 bot (Sep 07 2024 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (697358aac3153b635c90289bf62c757d4a387f94).

github mathlib4 bot (Sep 07 2024 at 18:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2969d0119259fdf37a81cca002481be932cc8953).

github mathlib4 bot (Sep 08 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (75f3daf8cc2fb299b4d1e6f32624e975571df02f).

github mathlib4 bot (Sep 08 2024 at 06:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d17749b757dec0421fa431f4b718b2eb32f45a0b).

github mathlib4 bot (Sep 08 2024 at 08:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (12972e5e1c216e329d4b99737393123dd01e228e).

github mathlib4 bot (Sep 08 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b63d3d7badd8425f556e02856b0f437bf782a612).

github mathlib4 bot (Sep 08 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (48b2de3ddb0ecf2389c032717dd9053797be3ad2).

github mathlib4 bot (Sep 08 2024 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3fecb249afcf5ba40efe0a3f92f69e2460f142c7).

github mathlib4 bot (Sep 09 2024 at 00:10):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (45faa3eea1dbc6c8336f8a8d288b8871564d5da4)

github mathlib4 bot (Sep 09 2024 at 06:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f7f80c239977dd8a06d9158a95efd03767d6ed68).

github mathlib4 bot (Sep 09 2024 at 08:02):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (45faa3eea1dbc6c8336f8a8d288b8871564d5da4)

github mathlib4 bot (Sep 09 2024 at 09:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1a0ce78731ee2c96b9823665cbb2052d1be9e400)

Kim Morrison (Sep 09 2024 at 12:15):

We will need to merge lean-pr-testing-5287 tomorrow.

github mathlib4 bot (Sep 09 2024 at 12:31):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1a0ce78731ee2c96b9823665cbb2052d1be9e400)

Kim Morrison (Sep 10 2024 at 04:59):

Also lean-pr-testing-5285.

Kim Morrison (Sep 10 2024 at 05:09):

Also lean-pr-testing-5288

github mathlib4 bot (Sep 10 2024 at 07:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1a0ce78731ee2c96b9823665cbb2052d1be9e400)

github mathlib4 bot (Sep 10 2024 at 08:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ba034836fdc5fe55f9903781364a9a1a4cbb0f55).

Kim Morrison (Sep 10 2024 at 08:43):

Merged those three branches into both batteries and mathlib, lets see what happens!

Kim Morrison (Sep 10 2024 at 08:52):

A few more breakages from List API changes that I didn't test Mathlib on ahead of time, but looking good!

Kim Morrison (Sep 10 2024 at 10:18):

We will need to merge lean-pr-testing-5231 tomorrow (2024-09-11)

github mathlib4 bot (Sep 10 2024 at 10:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3bebc671e9c9c1b535ad7ce3a6f96a2263835424).

github mathlib4 bot (Sep 10 2024 at 13:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a24b5c58241139e2f8d1d41d0ca75c77f66c1c6c)

Kim Morrison (Sep 11 2024 at 04:54):

also lean-pr-testing-5300

Kim Morrison (Sep 11 2024 at 06:16):

possibly also 5301, not sure if it will be in by the cut-off

github mathlib4 bot (Sep 11 2024 at 07:38):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a24b5c58241139e2f8d1d41d0ca75c77f66c1c6c)

github mathlib4 bot (Sep 11 2024 at 08:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4b83244f3ea8cf1ebc70f68bc5b94691e826c827).

Kim Morrison (Sep 11 2024 at 08:34):

Oof, merging lean-pr-testing-5231 was painful, many spurious diffs apparently. We'll have to check the next adaptation PR carefully to see I didn't mess up.

Kim Morrison (Sep 11 2024 at 08:38):

Merged all adaptations for 5231, 5300, 5301 (and 5301 to batteries too). Off to CI.

github mathlib4 bot (Sep 11 2024 at 09:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4b83244f3ea8cf1ebc70f68bc5b94691e826c827).

Kim Morrison (Sep 11 2024 at 09:58):

Just a shake!

github mathlib4 bot (Sep 11 2024 at 10:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (53d5e938e36f196da71b8397bb5b8bb62e2a2bdd).

github mathlib4 bot (Sep 11 2024 at 12:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ef71a8c9cccfbcebe64cf2d67f38bf09a01033fa).

github mathlib4 bot (Sep 11 2024 at 16:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ef7e491abf105a095ad1ad854cafb009dca3396c).

github mathlib4 bot (Sep 11 2024 at 19:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d1657b5fa11d79e2b5ccc9019c3ec8826d40e8c5).

github mathlib4 bot (Sep 11 2024 at 22:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (216c754008de909a8ecc89695c745846c9b736a3).

github mathlib4 bot (Sep 12 2024 at 00:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9405e9af9c4db56c19da07c118e4153fee571727)

Kim Morrison (Sep 12 2024 at 01:29):

lean-pr-testing-5302 needs merging tonight

github mathlib4 bot (Sep 12 2024 at 04:37):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9405e9af9c4db56c19da07c118e4153fee571727)

github mathlib4 bot (Sep 12 2024 at 08:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (002afcff4587088469cc9adf06068c4bd6f3daeb).

github mathlib4 bot (Sep 12 2024 at 09:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c64747cadc453f342f9560370252fa54ebf2db5).

github mathlib4 bot (Sep 12 2024 at 10:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a70901769a5f32a3298bda9265cfaa4b9621a075).

github mathlib4 bot (Sep 12 2024 at 11:07):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c8f802fb69c54d2c197eb1c2a31409da21d98d57)

github mathlib4 bot (Sep 12 2024 at 13:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (776511a5ea0680f999a3792344763bf898fa2246).

github mathlib4 bot (Sep 13 2024 at 08:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3c78bbdb01c312bd5143e44a38e6cbc8deb4b90).

github mathlib4 bot (Sep 13 2024 at 10:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8cefabf7abc9875bcbe0656ebb4b83fa65a76a5c)

github mathlib4 bot (Sep 14 2024 at 08:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f19f21c054039f3bcf6e96fbbea4fb78937daeb4).

Kim Morrison (Sep 14 2024 at 08:56):

Merged lean-pr-testing-5329, back to CI.

github mathlib4 bot (Sep 14 2024 at 09:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9e2a933e5b9357cd2b4802f7b02bdea98f580c14).

github mathlib4 bot (Sep 14 2024 at 09:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4f3889a86ffac7efae3ba1b0024b34f7ac1a8bc1)

github mathlib4 bot (Sep 15 2024 at 09:09):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (fcf04cd57e0d8399ce3f21dae009d2ca2d3abd26)

Kim Morrison (Sep 16 2024 at 02:01):

We will need lean-pr-testing-5303 tonight.

Kim Morrison (Sep 16 2024 at 02:46):

Also lean-pr-testing-5351

Kim Morrison (Sep 16 2024 at 03:09):

Also lean-pr-testing-5331

Kim Morrison (Sep 16 2024 at 03:40):

Also lean-pr-testing-5294

Kim Morrison (Sep 16 2024 at 04:44):

Also lean-pr-testing-5354

github mathlib4 bot (Sep 16 2024 at 06:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (fcf04cd57e0d8399ce3f21dae009d2ca2d3abd26)

Kim Morrison (Sep 16 2024 at 07:38):

Also lean-pr-testing-5356 (I slightly delayed the nightly to squeeze this one in.)

github mathlib4 bot (Sep 16 2024 at 09:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cc2c5288193edfd09bc4bf4eb6e0b26459c8572e).

Kim Morrison (Sep 16 2024 at 09:17):

All merged.

github mathlib4 bot (Sep 16 2024 at 10:45):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e9842c947725cc37c92d023e414f946a318bfd86)

github mathlib4 bot (Sep 17 2024 at 03:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab21cb1b654a53e71fa3c950f9650c544bb582e6).

github mathlib4 bot (Sep 17 2024 at 08:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e4699dfe66fd5a01a8a0f85b8cde6c555f25c3a1).

github mathlib4 bot (Sep 17 2024 at 10:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b755dda4cc224e363581d92a4d0b470d28742d4c).

github mathlib4 bot (Sep 17 2024 at 13:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9a321de82209309619b2f76efee973b6ab5808b1).

github mathlib4 bot (Sep 17 2024 at 15:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9801c67765e45f8224d33f2d1863ab5ec08548b8).

github mathlib4 bot (Sep 17 2024 at 19:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a5f5e464b94b32dbc60917f5e49e58c4b0bce6e0).

github mathlib4 bot (Sep 17 2024 at 22:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3b220c587207ebfe48e7bcc3634b403756877e90).

github mathlib4 bot (Sep 18 2024 at 01:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e645d886ff9a51fe2ee08f962b5e51beaaba8119)

github mathlib4 bot (Sep 18 2024 at 09:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (58d12e884e3ad7168e1278fcde332ba843964afe)

Kim Morrison (Sep 18 2024 at 10:07):

We will need to merge lean-pr-testing-5380 and lean-pr-testing-5381 tomorrow.

github mathlib4 bot (Sep 18 2024 at 10:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (58d12e884e3ad7168e1278fcde332ba843964afe)

github mathlib4 bot (Sep 18 2024 at 15:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca613b5c52e6c064681fc5da427208e8fa9fbb52).

github mathlib4 bot (Sep 18 2024 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (51a9d75766204ed306daf9b12f34105a477e2a1b).

github mathlib4 bot (Sep 18 2024 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (38dfa07f6fae335a6df1eed502afb7783ced97dd).

github mathlib4 bot (Sep 19 2024 at 00:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6b33760c50695343a2a94aa9e67dd9b84aa71868).

github mathlib4 bot (Sep 19 2024 at 01:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6b33760c50695343a2a94aa9e67dd9b84aa71868).

github mathlib4 bot (Sep 19 2024 at 06:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f2c6dd5e664931cac7e67308425179ff12b9c568).

Kim Morrison (Sep 19 2024 at 08:25):

Kim Morrison said:

We will need to merge lean-pr-testing-5380 and lean-pr-testing-5381 tomorrow.

Done.

github mathlib4 bot (Sep 19 2024 at 09:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (74fc63fadb6c60c2d7bf1a74cf9db7a76666b3ad).

github mathlib4 bot (Sep 19 2024 at 10:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d31ca8563e6e8db1130c64236aaae695ae9282c1).

github mathlib4 bot (Sep 19 2024 at 10:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (094c514c02044ce08421952aef5a9fc1e8600f61).

github mathlib4 bot (Sep 19 2024 at 13:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0e7d55443d22f4e179f761356d0247fd2e122c00).

github mathlib4 bot (Sep 19 2024 at 15:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (02caa3e1a58598830039cdfc9f277714e1846dfc)

github mathlib4 bot (Sep 20 2024 at 08:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6dcd0d943385f315b956fc76968c842a3ad4072c).

github mathlib4 bot (Sep 20 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (33b95b3e8b1593c67e03565adbc04b323e2437a4).

Kim Morrison (Sep 20 2024 at 11:34):

merging lean-pr-testing-5376, wish me luck :-)

github mathlib4 bot (Sep 20 2024 at 12:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8975918ef97a48d09b1b8706a91bdfd0e1a3361e)

github mathlib4 bot (Sep 21 2024 at 09:21):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4cebeb5b6632e5e738dcecc6831c6ea4ec20e9ee)

Kim Morrison (Sep 23 2024 at 03:44):

We will need to merge lean-pr-testing-5405 tonight.

github mathlib4 bot (Sep 23 2024 at 03:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4cebeb5b6632e5e738dcecc6831c6ea4ec20e9ee)

github mathlib4 bot (Sep 23 2024 at 08:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6fd58d5c798b0c1754df37d5eb213c1ce5326b33).

github mathlib4 bot (Sep 23 2024 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b4dda71e1bd8297df387af10ff0ca7f0a5127385).

Joachim Breitner (Sep 23 2024 at 10:24):

Kim Morrison said:

We will need to merge lean-pr-testing-5405 tonight.

NB: this changes batteries only, not really mathlib.

github mathlib4 bot (Sep 23 2024 at 11:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (09c50fb84c0b5e89b270ff20af6ae7e4bd61511e).

github mathlib4 bot (Sep 23 2024 at 12:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b3bc833ae962ba9c7eafa4116e7dc8dfe967b0fe)

github mathlib4 bot (Sep 23 2024 at 13:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9a329fb9ed78734d85679055a2a748ea804ea403).

github mathlib4 bot (Sep 23 2024 at 16:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (305ddf1349def3aa813838a62f73592b81759784).

github mathlib4 bot (Sep 23 2024 at 17:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b978dc4ce9ac8b9d3b46b5fe1c22dc11a010dd8b).

github mathlib4 bot (Sep 23 2024 at 18:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8192b1aeed705058e2c7369599897104813e0ba0).

github mathlib4 bot (Sep 23 2024 at 22:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3b44012533a6ff066c683a2a4a4320b7997c27df).

github mathlib4 bot (Sep 24 2024 at 01:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd587965db77dd971e90f7d1861a2863b1b6c367).

github mathlib4 bot (Sep 24 2024 at 02:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b3bc833ae962ba9c7eafa4116e7dc8dfe967b0fe)

github mathlib4 bot (Sep 24 2024 at 08:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c15e46e9bd6a62f3d9187d1b433ceefd9bea4749).

github mathlib4 bot (Sep 24 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f9a6642793ae66d29f800b7d153fb2af807a18ad).

github mathlib4 bot (Sep 24 2024 at 13:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (08a9b5c185b952bb4a0c628361f4b2f8fe7eb623)

github mathlib4 bot (Sep 24 2024 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b479ce63ba159bc287f99242ed9fb313ea7668da).

github mathlib4 bot (Sep 24 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6d0638698bd9e481c26abc2827b7d7a53ebbc115).

github mathlib4 bot (Sep 24 2024 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9c5f43190beca396e21a967800dd977750acbb78).

github mathlib4 bot (Sep 25 2024 at 01:02):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (08a9b5c185b952bb4a0c628361f4b2f8fe7eb623)

Kim Morrison (Sep 25 2024 at 06:27):

@Johan Commelin, the bot did not generate a reminder today.

Johan Commelin (Sep 25 2024 at 06:29):

Oops, weird. I didn't touch that workflow at all. Will try to find time to investigate. But lots of teaching and meetings today.

Kim Morrison (Sep 25 2024 at 06:30):

Oh, false alarm, sorry, I am just confused.

Kim Morrison (Sep 25 2024 at 06:30):

We're not expecting one yet

github mathlib4 bot (Sep 25 2024 at 08:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f7eb186981d26df6a660ad65bc92771d8bcf146b).

github mathlib4 bot (Sep 25 2024 at 09:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7c93f8663cb1931f808aae5066e978e043557dbd).

Kim Morrison (Sep 25 2024 at 10:02):

We'll need to merge lean-pr-testing-5464 tomorrow.

github mathlib4 bot (Sep 25 2024 at 10:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4591e55bbcc5a0ff893487a5a8db65953909ea48).

github mathlib4 bot (Sep 25 2024 at 12:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f22e9cb44e572aa5c27f2b3e5136e365e36bf1c3)

github mathlib4 bot (Sep 25 2024 at 16:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a95aae112143332f4f21618ff217e17b50be5dc7).

github mathlib4 bot (Sep 25 2024 at 19:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5f551d9f89a062d62820d2b02d2f7782fc5dbf98).

github mathlib4 bot (Sep 25 2024 at 19:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15dec28087d004fe2b06c085b54c795c7c3b3c54).

github mathlib4 bot (Sep 25 2024 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (88787b217c3255058d0046f800a349f773ce27b2).

github mathlib4 bot (Sep 26 2024 at 01:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f22e9cb44e572aa5c27f2b3e5136e365e36bf1c3)

github mathlib4 bot (Sep 26 2024 at 08:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (78a0b2f466ea466316f4a918ecdc26aab4a38cd9).

github mathlib4 bot (Sep 26 2024 at 09:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (78a0b2f466ea466316f4a918ecdc26aab4a38cd9).

github mathlib4 bot (Sep 26 2024 at 10:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (78a0b2f466ea466316f4a918ecdc26aab4a38cd9).

github mathlib4 bot (Sep 26 2024 at 13:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a60d315e0ec15d6a373325b2e60e80b8638384dc).

github mathlib4 bot (Sep 26 2024 at 16:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d86f6e1c768d3f101574832ac726a4516fe7f4e9).

github mathlib4 bot (Sep 26 2024 at 19:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aaff5ad5b038e792f9225de7fe6a37c9689b6ec8).

github mathlib4 bot (Sep 26 2024 at 22:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aaff5ad5b038e792f9225de7fe6a37c9689b6ec8).

github mathlib4 bot (Sep 27 2024 at 00:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (20ec679d5169e14e3aea2592db220a2753f840d1).

github mathlib4 bot (Sep 27 2024 at 00:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (20ec679d5169e14e3aea2592db220a2753f840d1).

github mathlib4 bot (Sep 27 2024 at 04:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (28af5205699f7d1945d148ebb846cd60a08e74a6).

github mathlib4 bot (Sep 27 2024 at 06:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (28af5205699f7d1945d148ebb846cd60a08e74a6).

github mathlib4 bot (Sep 27 2024 at 06:33):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (0510a8eb7a3628edd2b79c33efa04c93f377281d)

github mathlib4 bot (Sep 27 2024 at 08:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a94fd6ee3ccf9fde6e47075859d8c1f682579fd3).

github mathlib4 bot (Sep 27 2024 at 09:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a94fd6ee3ccf9fde6e47075859d8c1f682579fd3).

github mathlib4 bot (Sep 27 2024 at 12:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a94fd6ee3ccf9fde6e47075859d8c1f682579fd3).

github mathlib4 bot (Sep 27 2024 at 12:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0f85ae293d320fb099968a022574b5a427ce253c).

github mathlib4 bot (Sep 27 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7abd698384e16028dce447cb84f5f342512deaec).

github mathlib4 bot (Sep 27 2024 at 18:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (418c53780957030e8fd99d2007872a87ad82d9e6).

github mathlib4 bot (Sep 27 2024 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7da2960d5ff6656028a8d2bece5370ad5859b270).

github mathlib4 bot (Sep 28 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2b108d1e9018455f2a4d06b17b06a0f689f42278).

github mathlib4 bot (Sep 28 2024 at 05:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c0c2c8fac501e8c0580177432e21fd461cb64580)

github mathlib4 bot (Sep 28 2024 at 18:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a087cde0a3dc36762e4954ff1b2763540431aa18).

github mathlib4 bot (Sep 28 2024 at 19:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a087cde0a3dc36762e4954ff1b2763540431aa18).

github mathlib4 bot (Sep 28 2024 at 21:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b9053eacfc271ea559687f4336b6f3f34d92ecc).

Kim Morrison (Sep 29 2024 at 00:03):

There are some failures now in AlgebraicGeometry, that I probably won't have time to look at until tomorrow. If any algebraic geoemeters who see this want to take a look, that would be great. :-)

Kim Morrison (Sep 29 2024 at 00:05):

Oh, actually they were easy.

Kim Morrison (Sep 29 2024 at 00:06):

Kyle's changes to how @ and named arguments interact.

Kim Morrison (Sep 29 2024 at 00:06):

lean4#5283

Kim Morrison (Sep 29 2024 at 00:08):

and just found Kyle's better adaptations on lean-pr-testing-5283. We really need to automate discovery / merging of these branches in nightly-testing..

Kyle Miller (Sep 29 2024 at 00:10):

Darn, I thought about mentioning the fixes in lean-pr-testing-5283, but I wasn't sure if that was just going to be noise

Kim Morrison (Sep 29 2024 at 00:10):

No, all good, it's a process problem we have here.

Kim Morrison (Sep 29 2024 at 00:11):

We either need a bot that, after the release of a new Lean nightly, either:

  1. posts here with a summary of all the relevant lean-pr-testing-NNNN branches that have changes on them
  2. actually merges them directly into nightly-testing

Kim Morrison (Sep 29 2024 at 00:12):

  1. feels somewhat scary, but would significantly reduce work/confusion on my part

Kim Morrison (Sep 29 2024 at 00:12):

hmm, lean-pr-testing-5283 didn't quite work, there is now a problem in Data/Nat/Defs involving a named argument

Kim Morrison (Sep 29 2024 at 00:12):

(on nightly-testing)

Kim Morrison (Sep 29 2024 at 00:12):

and I really should run now.

Kyle Miller (Sep 29 2024 at 00:13):

What's the current status of nightly-testing? Are they my adaptations?

Kyle Miller (Sep 29 2024 at 00:13):

I can take a look

Kim Morrison (Sep 29 2024 at 00:13):

Yes, I just merged lean-pr-testing-5283 into nightly-testing

github mathlib4 bot (Sep 29 2024 at 00:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2845f11d96267fc699a8c1024e3caf998d4b3fdc).

Kim Morrison (Sep 29 2024 at 00:13):

(I was about to say you won't have a cache, but ...)

Kyle Miller (Sep 29 2024 at 00:28):

Something went very wrong with the merge for lean4#5283 itself... I need to figure out where the changes actually went!

Kyle Miller (Sep 29 2024 at 00:37):

I see, I did a last-minute rebase on the wrong computer, using early version of the branch :man_facepalming:

github mathlib4 bot (Sep 29 2024 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (197417dc8fc00c22a2e575192767564190f1417e).

Kyle Miller (Sep 29 2024 at 00:51):

That's an embarrassing mistake. I now have lean4#5512 with the missing part of the PR, and I'll merge it after some testing. We'll need a new nightly before the 5283 fixes will work.

github mathlib4 bot (Sep 29 2024 at 03:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4cd4cfb8ebb1f63252cdeaf0f82009b4cf19ae06).

Kim Morrison (Sep 29 2024 at 03:41):

(As Kyle says above, we'll wait for the next nightly before fixing this.)

github mathlib4 bot (Sep 29 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c8df482f4de3224efdb7bb67160f0af3ef3bc065).

github mathlib4 bot (Sep 29 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9491960f1f448fa353e840f5b146feea22d5dbfd).

github mathlib4 bot (Sep 29 2024 at 09:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a6006d2f1d3d5ffc24da15256c54ff36b26d9f61).

github mathlib4 bot (Sep 29 2024 at 11:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a6006d2f1d3d5ffc24da15256c54ff36b26d9f61).

github mathlib4 bot (Sep 29 2024 at 12:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a6006d2f1d3d5ffc24da15256c54ff36b26d9f61).

Kim Morrison (Sep 29 2024 at 12:19):

We'll need to merge lean-pr-testing-5520 tomorrow.

github mathlib4 bot (Sep 29 2024 at 13:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (62eccbcb33b8a9fc8e7cc61cd546298b52f0c29b).

github mathlib4 bot (Sep 29 2024 at 16:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (54358ec938bcf95978586464cbd1010833f6970a).

github mathlib4 bot (Sep 29 2024 at 22:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (301f54abf16c4d7706fb65a94ece16e384d6622e).

github mathlib4 bot (Sep 30 2024 at 00:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (301f54abf16c4d7706fb65a94ece16e384d6622e).

github mathlib4 bot (Sep 30 2024 at 00:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4a9dd28c84b0d3bf0bc7b70e1767c367da41de99)

Kim Morrison (Sep 30 2024 at 03:41):

We'll need to merge lean-pr-testing-5526 here and at batteries tonight.

github mathlib4 bot (Sep 30 2024 at 04:47):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4a9dd28c84b0d3bf0bc7b70e1767c367da41de99)

github mathlib4 bot (Sep 30 2024 at 08:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eed3300c27c9f168d53e13bb198a92a147b671d0).

github mathlib4 bot (Sep 30 2024 at 10:37):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (0c3346c1787354ee3398f5cefa726ff51938f9b1)

github mathlib4 bot (Sep 30 2024 at 15:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2db234e2d5db1c1df0efbbaf581cc1c46194a12c).

github mathlib4 bot (Sep 30 2024 at 15:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cb03ac23046975efec06f8795593e438d39a373b).

github mathlib4 bot (Sep 30 2024 at 18:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (0c3346c1787354ee3398f5cefa726ff51938f9b1)

Johan Commelin (Oct 01 2024 at 03:58):

Huh? That's the exact same hash as 3 messages above it...

Kim Morrison (Oct 01 2024 at 05:38):

We'll need to merge lean-pr-testing-5529

github mathlib4 bot (Oct 01 2024 at 07:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0da2361bd278b7158de3a93c1e39b29b63aae58c).

github mathlib4 bot (Oct 01 2024 at 08:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (809c3fb3b5c8f5d7dace56e200b426187516535a).

github mathlib4 bot (Oct 01 2024 at 09:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (809c3fb3b5c8f5d7dace56e200b426187516535a).

github mathlib4 bot (Oct 01 2024 at 12:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2cb73c7a2936f65cffe50de51138795da5df8939).

Johan Commelin (Oct 01 2024 at 14:10):

#17329 makes these messages a bit more actionable

Johan Commelin (Oct 01 2024 at 14:57):

Branches that we should probably merge today:

lean-pr-testing-5486
lean-pr-testing-5529
lean-pr-testing-5530
lean-pr-testing-5546

github mathlib4 bot (Oct 01 2024 at 15:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f73be5b0ca97f80cde7c032e61b68b20a5835794).

Johan Commelin (Oct 01 2024 at 18:01):

Only the branch that Kim posted has an actual diff.

Johan Commelin (Oct 01 2024 at 18:06):

@Kim Morrison I merged that branch.

github mathlib4 bot (Oct 01 2024 at 18:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1fe4aec4735318982df91ad8ff0581406c6b625e).

github mathlib4 bot (Oct 01 2024 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1fe4aec4735318982df91ad8ff0581406c6b625e).

github mathlib4 bot (Oct 01 2024 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ebdf9cca3c351868ae7c2786096256474715e5e2).

github mathlib4 bot (Oct 02 2024 at 01:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ebabb3402ee09467a5836072a47b298486eacf4a).

github mathlib4 bot (Oct 02 2024 at 02:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ebabb3402ee09467a5836072a47b298486eacf4a).

Kim Morrison (Oct 02 2024 at 02:55):

transient

github mathlib4 bot (Oct 02 2024 at 04:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1235f45ece3c1f049543e58769e29b31340f7269).

Kim Morrison (Oct 02 2024 at 06:10):

Oh, I think we're not going to get further than that today because of the lake errors. Hopefully fixed in a few hours on the next nightly.

Kim Morrison (Oct 02 2024 at 06:10):

(Which, :fingers_crossed:, becomes v4.13.0-rc1!)

github mathlib4 bot (Oct 02 2024 at 07:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3fdb944d51949cc06cd938cdf78df3e87ef4c5c3).

github mathlib4 bot (Oct 02 2024 at 09:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7fc7838ae4893e5ae499695841fe5c57ee4c0a08).

Kim Morrison (Oct 02 2024 at 09:40):

Lots to do here, not sure if I'll get to it tonight.

Kim Morrison (Oct 02 2024 at 09:40):

Have to start in Batteries, some metaprogramming things were upstreamed.

Kim Morrison (Oct 02 2024 at 09:40):

and some HashSet stuff

github mathlib4 bot (Oct 02 2024 at 10:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b91c5b63fd9ad104b16ea34bd259162dd1850b9e).

Kim Morrison (Oct 02 2024 at 11:11):

Another problem with lake has come up, anyone touching nightly-testing will need to use lake --no-cache build.

github mathlib4 bot (Oct 02 2024 at 11:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c4b22ac853b671670de4eb12d2c36a3692d25673).

github mathlib4 bot (Oct 02 2024 at 13:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4236727d21dcfef1c709eb7801331d10755e06bc).

github mathlib4 bot (Oct 02 2024 at 16:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c472200bb60e0adf2bf0cea4b0d04985511b276d).

github mathlib4 bot (Oct 02 2024 at 19:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (551dfed37fb761cc7bc33eac160eae1771191226).

github mathlib4 bot (Oct 02 2024 at 22:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (20a854cda8bedffea00955e1b174ae4c7f72b269).

github mathlib4 bot (Oct 03 2024 at 02:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (655d653bfd6eb4968829ce8e2b5e4ed0419f6f05).

github mathlib4 bot (Oct 03 2024 at 07:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f84123514f85483265d95458b3203f81651de3f2).

Kim Morrison (Oct 03 2024 at 10:04):

nightly-2024-10-03 is out, and looking better locally.

Kim Morrison (Oct 03 2024 at 10:04):

Hopefully this will become v4.13.0-rc1 shortly after we get a tick here.

github mathlib4 bot (Oct 03 2024 at 11:03):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5da739c04be092369c9258dd09eb3c9d47841108)

github mathlib4 bot (Oct 03 2024 at 11:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (70102953aa125ae9abd08cd7d0ab8f4194055834).

github mathlib4 bot (Oct 03 2024 at 12:31):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5da739c04be092369c9258dd09eb3c9d47841108)

Johan Commelin (Oct 04 2024 at 07:17):

#17399 should hopefully automate determining which lean-pr-testing-NNNN branches need to be merged on a given day

github mathlib4 bot (Oct 07 2024 at 13:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (78b3a02235527543f0c61118f06b48d44fa96a32).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 07 2024 at 13:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (78b3a02235527543f0c61118f06b48d44fa96a32).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 07 2024 at 14:52):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3809315f2f79b1028a9a1e22c5f18be1f2da21bc)

Johan Commelin (Oct 07 2024 at 14:57):

Awesome!

Johan Commelin (Oct 07 2024 at 14:57):

It was bubbling to the top of my todo list to fix this.

Johan Commelin (Oct 07 2024 at 14:58):

@Joachim Breitner I guess that was you? Merci!

github mathlib4 bot (Oct 07 2024 at 16:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5017a681823e948dea4ad55740d86cc8754e4ea6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 07 2024 at 19:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3ce877a139a51fb84abba4cd2d86078d64e848f9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 07 2024 at 22:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a239b9573c31a8a440e726e42bdc39c956ef5e0e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2024 at 01:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dde8da66e3a5773f20dceaea8d37e91ffcb5183f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2024 at 03:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2e8a2b233a733bcfb8f95c9498a18d905e697558).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2024 at 06:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3693fb294c1201f0b69ba48e98d083d2bb3e630d).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Oct 08 2024 at 06:36):

I've merged lean-pr-testing-5560

Johan Commelin (Oct 08 2024 at 06:36):

Hopefully we'll have a green checkmark again today

Johan Commelin (Oct 08 2024 at 06:48):

I'm getting

warning: ././././Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean:608:44: `Isometry.uniformEmbedding` has been deprecated, use `Isometry.isUniformEmbedding` instead
warning: ././././Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean:629:52: `Isometry.uniformEmbedding` has been deprecated, use `Isometry.isUniformEmbedding` instead
warning: ././././Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean:653:63: `uniformEmbedding_subtype_val` has been deprecated, use `isUniformEmbedding_subtype_val` instead
warning: ././././Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean:659:4: `uniformEmbedding_subtype_val` has been deprecated, use `isUniformEmbedding_subtype_val` instead
warning: ././././Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean:678:4: `uniformEmbedding_subtype_val` has been deprecated, use `isUniformEmbedding_subtype_val` instead
warning: ././././Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean:684:4: `uniformEmbedding_subtype_val` has been deprecated, use `isUniformEmbedding_subtype_val` instead

which is fine, I can fix those. But I'm a bit surprised that they didn't go away after merging master.

github mathlib4 bot (Oct 08 2024 at 07:30):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3809315f2f79b1028a9a1e22c5f18be1f2da21bc)

Johan Commelin (Oct 08 2024 at 07:40):

:sweat_smile:

github mathlib4 bot (Oct 08 2024 at 09:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (bbd5da4d2d2b4e5950ad78a8ee60a6b477ccab6e)

github mathlib4 bot (Oct 08 2024 at 21:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0d4b02ed386a928bde1684cb15c64b7e2a1aa38d).
You can git fetch; git checkout nightly-testing and push a fix.

Damiano Testa (Oct 08 2024 at 21:47):

Sorry, I broke nightly-testing: I had pushed a fix that depends on lean4#5644, but it seems that the PR that makes my changes a fix is not implied by nightly-testing!

Damiano Testa (Oct 08 2024 at 21:47):

I don't really know what to do though...

github mathlib4 bot (Oct 08 2024 at 22:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (964c714dda9a83f8856e82be83ca185745bfc3a8).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 08 2024 at 22:29):

Damiano Testa said:

I don't really know what to do though...

We could wait for the next nightly :-)

github mathlib4 bot (Oct 09 2024 at 01:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fb07d0ded9b50108d6af885ddb66842e3396f1c2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 09 2024 at 04:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f4131e1aae877c36385bf386ad356471ddf6d6e0).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Oct 09 2024 at 04:50):

https://github.com/leanprover-community/mathlib4/actions/runs/11247758087/job/31271752035 shows that a bunch of tests are failing

Kyle Miller (Oct 09 2024 at 05:04):

I think we need the next nightly @Johan Commelin; nightly-testing is still on leanprover/lean4:nightly-2024-10-08.

Johan Commelin (Oct 09 2024 at 05:57):

Aah, I actually don't know what time of the day lean thinks is "night"  :rofl:

Damiano Testa (Oct 09 2024 at 06:03):

Btw, I think that the failing tests are due to the fact that I "adapted" the branch to the changes in #guard_msgs and I think that the should work using lean4#5644.

Kyle Miller (Oct 09 2024 at 06:04):

Judging by when https://github.com/leanprover-community/mathlib4/blob/nightly-testing/lean-toolchain was last updated, maybe it'll update again in about 2 hours 20 minutes

github mathlib4 bot (Oct 09 2024 at 07:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8e7a3003b71cbd354f44d2e204b36e937ba9eb39).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 09 2024 at 08:41):

The toolchain looks like it updated 18 minutes ago, so "Lean midnight" is 8:23AM UTC

github mathlib4 bot (Oct 09 2024 at 09:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (77a0e20869a4746d978f3b85ff8366d020728eef).
You can git fetch; git checkout nightly-testing and push a fix.

Damiano Testa (Oct 09 2024 at 09:29):

The failure is again "just" #guard_msgs, but at least the fixes that I introduced work! There are "new" failures.

github mathlib4 bot (Oct 09 2024 at 10:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e2b29fbc0b174dd424a34be581001dea179cd915).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Oct 09 2024 at 12:27):

@Kyle Miller @Damiano Testa Is this diff to be expected?

diff --git a/test/HashCommandLinter.lean b/test/HashCommandLinter.lean
index 7f77ef113f..073acaf21b 100644
--- a/test/HashCommandLinter.lean
+++ b/test/HashCommandLinter.lean
@@ -28,7 +28,8 @@ section ignored_commands
 #check 0

 /--
-info:
+warning: `#`-commands, such as '#eval', are not allowed in 'Mathlib'
+note: this linter can be disabled with `set_option linter.hashCommand false`
 -/
 #guard_msgs in
 -- emits an empty message -- the linter allows it
diff --git a/test/dfinsupp_notation.lean b/test/dfinsupp_notation.lean
index ed6511532b..e4988503d7 100644
--- a/test/dfinsupp_notation.lean
+++ b/test/dfinsupp_notation.lean
@@ -7,18 +7,12 @@ example : (fun₀ | 1 | 2 | 3 => 3 | 3 => 4 : Π₀ i, Fin (i + 10)) 1 = 3 := by
 example : (fun₀ | 1 | 2 | 3 => 3 | 3 => 4 : Π₀ i, Fin (i + 10)) 2 = 3 := by simp
 example : (fun₀ | 1 | 2 | 3 => 3 | 3 => 4 : Π₀ i, Fin (i + 10)) 3 = 4 := by simp

-/--
-info:
--/
 #guard_msgs in
 #eval show Lean.MetaM Unit from
   guard <|
     reprStr (fun₀ | 1 => 3 | 2 => 3 : Π₀ i, Fin (i + 10))
       = "fun₀ | 1 => 3 | 2 => 3"

-/--
-info:
--/
 #guard_msgs in
 #eval show Lean.MetaM Unit from
   guard <|
diff --git a/test/jacobiSym.lean b/test/jacobiSym.lean
index 916deb2aa2..0d010e4254 100644
--- a/test/jacobiSym.lean
+++ b/test/jacobiSym.lean
@@ -10,29 +10,29 @@ We test that `@[csimp]` replaces `jacobiSym` (i.e. `J(· | ·)`) and `legendreSy

 open scoped NumberTheorySymbols

-/-- info: -1 -/
+/-- info: Int.negSucc 0 -/
 #guard_msgs in
 #eval J(123 | 335)

-/-- info: -1 -/
+/-- info: Int.negSucc 0 -/
 #guard_msgs in
 #eval J(-2345 | 6789)

-/-- info: 1 -/
+/-- info: Int.ofNat 1 -/
 #guard_msgs in
 #eval J(-1 | 1655801)

-/-- info: -1 -/
+/-- info: Int.negSucc 0 -/
 #guard_msgs in
 #eval J(-102334155 | 165580141)

-/-- info: -1 -/
+/-- info: Int.negSucc 0 -/
 #guard_msgs in
 #eval J(58378362899022564339483801989973056405585914719065 |
   53974350278769849773003214636618718468638750007307)

 instance prime_1000003 : Fact (Nat.Prime 1000003) := ⟨by norm_num1⟩
-/-- info: -1 -/
+/-- info: Int.negSucc 0 -/
 #guard_msgs in
 #eval @legendreSym 1000003 prime_1000003 7

@@ -40,7 +40,7 @@ instance prime_1000003 : Fact (Nat.Prime 1000003) := ⟨by norm_num1⟩
 /--
 warning: declaration uses 'sorry'
 ---
-info: 1
+info: Int.ofNat 1
 -/
 #guard_msgs in
 #eval! @legendreSym (2 ^ 11213 - 1) sorry 7
diff --git a/test/success_if_fail_with_msg.lean b/test/success_if_fail_with_msg.lean
index 5f9f786e3e..1e190fde9d 100644
--- a/test/success_if_fail_with_msg.lean
+++ b/test/success_if_fail_with_msg.lean
@@ -54,8 +54,5 @@ def doesntFail : MetaM Unit := do
   try successIfFailWithMessage "I failed!" alwaysFails
   catch _ => throwError "I *really* failed."

-/--
-info:
--/
 #guard_msgs in
 #eval doesntFail

Johan Commelin (Oct 09 2024 at 12:27):

The

-/-- info: -1 -/
+/-- info: Int.negSucc 0 -/

looks suspicious to me.

Ruben Van de Velde (Oct 09 2024 at 12:28):

(deleted)

Johan Commelin (Oct 09 2024 at 12:29):

I pushed the diff above, but I'm happy to revert it later.

github mathlib4 bot (Oct 09 2024 at 12:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dacf74d6a54b0e776c97c90f3a1b9e8ef61f596e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 09 2024 at 13:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b43951ca72df001cffd7fbab1023a00282824ef).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Oct 09 2024 at 14:03):

So now a different set of tests is failing...

Kyle Miller (Oct 09 2024 at 14:07):

Johan Commelin said:

I pushed the diff above, but I'm happy to revert it later.

This seems to be that #eval is now using ToExpr instances, and there are some quirks that will need some attention.

We could set set_option eval.pp false for now in that file to go back to using Repr instances.

Kyle Miller (Oct 09 2024 at 14:09):

I can look at the failing DeriveFintype tests later, those are odd.

Johan Commelin (Oct 09 2024 at 14:10):

Merci!

Kyle Miller (Oct 09 2024 at 14:10):

But the rest of the failures look like they might be fixable with a set_option eval.pp false at the top

Johan Commelin (Oct 09 2024 at 14:15):

How do I run the tests locally? I can open a file, and that works. But I want to see the build output for all tests...

Johan Commelin (Oct 09 2024 at 14:15):

lake build test does something, but doesn't give warnings/errors.

Damiano Testa (Oct 09 2024 at 15:40):

I think that CI runs lake test.

github mathlib4 bot (Oct 09 2024 at 16:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7817d20eb8249e7a5acd2eef4e046b37407b7f2c).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 09 2024 at 17:52):

Tests might be fixed now

github mathlib4 bot (Oct 09 2024 at 18:04):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ccfb9511e1875f89123857f93865228ade8d0cef)

Johan Commelin (Oct 10 2024 at 01:12):

Awesome!

github mathlib4 bot (Oct 10 2024 at 01:50):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ccfb9511e1875f89123857f93865228ade8d0cef)

github mathlib4 bot (Oct 10 2024 at 08:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f7673a183937ba5589f2e3703634049778a222f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 10 2024 at 09:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (09585751583f599964186a8a58e01049d31867bd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 10 2024 at 12:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9d0db8d63b38ae04d5fcf91ce6f9e6da13d64402).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 10 2024 at 15:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f8265e0bc7f8d78fe5400a670368139e1aff0f2d).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 10 2024 at 16:18):

This error is waiting on #17567 to be merged

github mathlib4 bot (Oct 10 2024 at 19:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5c179825b962cca3ba1fae66444dea32a12de3f2)

github mathlib4 bot (Oct 11 2024 at 09:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7a7d5c09605f625446d7957ab54cbe9b486f0e34).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 11 2024 at 10:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e4fa33c4f2bc49e66f5d06e91e21fe2279ad7e14).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 11 2024 at 13:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9a934121c2756d98feab3cf79738ab3121d96deb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 11 2024 at 16:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (85cf1f190af7b00a5990fd5644f9a28c188eb4a6).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 11 2024 at 17:05):

#17655 will fix the failing tests

github mathlib4 bot (Oct 11 2024 at 19:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ae22b2a2e15bd80aa1472ec0cc5f25c043db4f5f).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 11 2024 at 22:20):

Ah, there are still a couple more structure ... :=s to address in tests. I can fix them tomorrow

github mathlib4 bot (Oct 11 2024 at 22:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9ba2d95ba478bcccea37c7f1f84932d364d9b314).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2024 at 03:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c35f067077ad7e27b7545e804de9ec7f477aa938).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2024 at 06:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (db094871afb9880e24c7558524a392fc998b96da).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2024 at 09:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0405d97af3ed0666079ab4ff41eab850d2867a17).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2024 at 10:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (90cf978d2237de99eb5a639301b5b0b3f913d744).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2024 at 13:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a02b71d090e5b5df65cda5ffbefb58b3ffb168b8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2024 at 16:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1fb2cbcfda77d978c076acdf586d370b83a7d4fb).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 12 2024 at 17:34):

#17688

github mathlib4 bot (Oct 12 2024 at 19:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1fb2cbcfda77d978c076acdf586d370b83a7d4fb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 13 2024 at 00:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e7062ed4631c76a999e1988a0d6a6b04a54684e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 13 2024 at 09:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e7062ed4631c76a999e1988a0d6a6b04a54684e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 13 2024 at 13:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (6125cddcb7541bb61d58f6f316cdd43b9c962e17)

github mathlib4 bot (Oct 14 2024 at 06:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5d2ccbb3e5b5df402d3b88f4c9aa0cd2ac986130).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 14 2024 at 08:07):

This should come good once #12540 lands in master.

github mathlib4 bot (Oct 14 2024 at 08:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7fe7e109014be7b69a513af14c44df3d3ab680c9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 14 2024 at 10:38):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (663637410a7edbee9fc0737ff0fdd01edd35a4b4)

github mathlib4 bot (Oct 15 2024 at 08:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d376bfc5782e90bafe2815b936ece41bf3b69f05).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (41475d2a4e4da9da4278bd2b328e51a8717cf53a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 15 2024 at 10:14):

We'll need to merge lean-pr-testing-5716 tomrrow

github mathlib4 bot (Oct 15 2024 at 10:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5f0628eab56cdcf7a33982a270433e0fc3a6e9a5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2024 at 11:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c9428b0dd6704e88e5703a7c1ab96dbcbac9ea41).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2024 at 13:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f87f0ec95cec45e45bdbeba6aa7f6c02a542f1cd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2024 at 16:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1b5eaee6c30b1cbe7669e1c4c125eb11d21ef5e8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2024 at 19:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (27ca8188dc20fb61ac2f2878268ce5748a324a6c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2024 at 22:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (af9a9c9ca2d15cc943a98510094e76a55cd8d988).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2024 at 23:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (244c025036bbbb74adc16d44932b3516c3aa9c93).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2024 at 00:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c63a0ac5dcbcea2165fdbbbe8be00cdf3b2a731c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2024 at 01:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (36bb3d003e48d0b7aef637b5e35e36f2389310e1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 16 2024 at 01:43):

Waiting on #17791 now

Kim Morrison (Oct 16 2024 at 01:45):

(which itself needs a shake)

github mathlib4 bot (Oct 16 2024 at 04:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ee226537119c803ac2a107a458a136994addf4d6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2024 at 04:38):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (264cb92bc96c0f0e1a92ea20524a1de270b3f008)

github mathlib4 bot (Oct 16 2024 at 08:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (765ccc9135f3ebeec047798d6c715dc3224c0c73).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2024 at 09:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b913345e5847bd22f23ab83b6256654095f161eb).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 16 2024 at 10:57):

We'll need to merge lean-pr-testing-5323 tomrrow

Kim Morrison (Oct 16 2024 at 11:13):

Hmm, right now on nightly-testing I get:

% lake build
 [?/?] Computing build jobs

hanging forever.

Kim Morrison (Oct 16 2024 at 11:13):

Can anymore else reproduce?

Kim Morrison (Oct 16 2024 at 11:13):

@Mac Malone, could you take a look at this?

Kim Morrison (Oct 16 2024 at 11:13):

(rm -rf .lake doesn't help)

Kim Morrison (Oct 16 2024 at 11:14):

I think this means I'm stuck on fixing nightly-testing.

Kim Morrison (Oct 16 2024 at 11:16):

CI appears to also be stuck at this point

Kim Morrison (Oct 16 2024 at 11:18):

Ah, it is a missing import. Still, lake shouldn't hang like that because of a missing import. @Mac Malone, 06dcc3e054eb5821fc61a639cf9a091e04bf716a is the commit where I fix the problem. Could you take a look?

Kim Morrison (Oct 16 2024 at 11:31):

We'll need to merge lean-pr-testing-5731 tomorrow into import-graph, aesop, batteries, and mathlib.

github mathlib4 bot (Oct 16 2024 at 12:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ebec1b61db40c3352391654316f3644e268fee46).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2024 at 13:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1aaa5b99d39e4bc03db73fd848a03062b974846f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2024 at 16:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8d6f380fde8631e39a62b5a009b2ffec2eb3c17f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2024 at 19:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ede775853cc9f271a9fcf1475dec887f82544e30).
You can git fetch; git checkout nightly-testing and push a fix.

Mac Malone (Oct 16 2024 at 20:52):

Kim Morrison said:

Ah, it is a missing import. Still, lake shouldn't hang like that because of a missing import. Mac Malone, 06dcc3e054eb5821fc61a639cf9a091e04bf716a is the commit where I fix the problem. Could you take a look?

Sadly, this hang on a missing import is a know issue that I have not yet been able to successfully debug. A significant problem is that it only seems to appear in Mathlib I cannot reproduce it in smaller examples. There should probably be an issue tracking this bug. Someone coming up with MWE would also be great! The good news is that my focus for the end of this month is addressing the Lake issue backlog, so this is something I could spend more time on debugging.

github mathlib4 bot (Oct 16 2024 at 21:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ede775853cc9f271a9fcf1475dec887f82544e30).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2024 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ede775853cc9f271a9fcf1475dec887f82544e30).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 16 2024 at 21:56):

@Mac Malone it seems we're stuck now on a different lake problem here. (Commit 3cf3909884d6457a49762a1d5bd514cfdebf9814 of nightly-testing for reproducibility.)

The current behaviour is:

% git checkout nightly-testing
% rm -rf .lake
% lake exe cache get
% lake build --no-build     ### Fails with exit code 3
% lake build                ### Doesn't appear to do anything
% lake build --no-build     ### Succeeds

I'm not sure why lake build --no-build is failing here, but it breaks the cache verification step in Mathlib CI.

Kim Morrison (Oct 16 2024 at 21:57):

(lake -v doesn't give any further information here)

Mac Malone (Oct 16 2024 at 22:05):

@Kim Morrison If I undestand correctly, the last successful nightly-testing was Oct 14. Thus, no Lake changes have been merged since then, right? If so, that should help me debug, as this is then likely a Lake bug to some unforseen configuration and not mrely due to a recent code change.

Kim Morrison (Oct 16 2024 at 22:06):

Yes, that's right.

Kim Morrison (Oct 16 2024 at 22:07):

There was some upstreaming of code from Batteries to Lean in the last nightly, and consequently files deleting in Batteries. We know that is relevant for the "getting stuck" bug, but may also be relevant here?

Kim Morrison (Oct 16 2024 at 22:11):

We will need to merge lean-pr-testing-5732 tonight.

Mac Malone (Oct 17 2024 at 00:13):

@Kim Morrison lake build --no-build --no-ache similarly fails, so it feels to me like something from the lake exe cache is inconsistent with Lake. I am currently debugging it.

Mac Malone (Oct 17 2024 at 00:16):

I looks like it may be rebuilding proofwidgets. Has proofwidgets had a new release?

Mac Malone (Oct 17 2024 at 00:29):

Yeah, on my machine, it builds ProofWidgets (and then the things depending on it). It seems lake exe cache is borked.

Mac Malone (Oct 17 2024 at 00:52):

ProofWidgets will need a new release eventually due to lean4#5641 (which changes its traces). While mathlib is not using ProofWidget's releases directly, the problem may be that one of its trace files has not been properly replaced the mathlib's cache/CI.

Sadly, I still do not know what in particular is tripping things up. Perhaps making a new release will be the easist fix?

github mathlib4 bot (Oct 17 2024 at 01:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (054aa6cbdca97165c441575e81897f4c1012b7c3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 17 2024 at 01:30):

Okay, new releases of ProofWidgets (v0.0.43 using v4.13.0-rc1, and v0.0.44-pre using leanprover/lean4:nightly-2024-10-16) coming up.

github mathlib4 bot (Oct 17 2024 at 02:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (054aa6cbdca97165c441575e81897f4c1012b7c3).
You can git fetch; git checkout nightly-testing and push a fix.

Mac Malone (Oct 17 2024 at 02:40):

Yay! It appears the bugs have been solved. (The new failure is just about unused imports.)

Kim Morrison (Oct 17 2024 at 03:26):

Thanks for your help diagnosing that one, @Mac Malone!

github mathlib4 bot (Oct 17 2024 at 03:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b33faadf563e7b3d6b9578d89a7f04292fc0f86d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 17 2024 at 03:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b33faadf563e7b3d6b9578d89a7f04292fc0f86d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 17 2024 at 04:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (08804ac5cc5dca54e6979de8388f59c937b60e8a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 17 2024 at 04:30):

We will (probably??) need to merge lean-pr-testing-5697 tonight.

github mathlib4 bot (Oct 17 2024 at 04:38):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e553fb0852ed7000d6b34eb25bb6d9a83ee069c4)

github mathlib4 bot (Oct 17 2024 at 08:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9caf52848a187af346984fdd790422b60183b41f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 17 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c1d3ebd51a1725828121397ad4a8f36aba2f3a07).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 17 2024 at 11:04):

Phew... we easily set a record of most lean-pr-testing-XXXX branches merged in a single nightly there.

Kim Morrison (Oct 17 2024 at 11:06):

Not quite done, however, something has broken in Mathlib.Order.KonigLemma, and I'm getting too sleepy to figure it out tonight.

A goal seems to have changed after just a have and a simp only, so I'm not quite sure what we've done to break it. Apologies ahead of time for which theorem statement I have presumably secretly changed under the hood!!

Kim Morrison (Oct 17 2024 at 11:06):

If anyone would like to take a look at that, much appreciated!

Kim Morrison (Oct 17 2024 at 11:17):

(Oh, perhaps I'll also ping @Peter Nelson as the original author of KonigLemma. Whatever the problem is here, it's certainly not your fault, just pinging in case you feel like doing some archaeology. The process here is to checkout nightly-testing, try to decipher what has gone wrong, and either fix it by pushing to the branch, or telling us we've done something stupid upstream.)

Anne Baanen (Oct 17 2024 at 11:21):

Looks like the issue was that Sigma.forall wasn't being applied to αs := (i : ℕ) × α i. So I added αs to the simp only calls and then they worked again.

Kim Morrison (Oct 17 2024 at 11:22):

That's ... weird, though?

Kim Morrison (Oct 17 2024 at 11:23):

oh

Kim Morrison (Oct 17 2024 at 11:25):

lean#5686

Kim Morrison (Oct 17 2024 at 11:25):

(and indeed, I forgot to merge lean-pr-testing-5686, which included the same fix!)

Kim Morrison (Oct 17 2024 at 11:25):

Thanks all.

Kim Morrison (Oct 17 2024 at 11:25):

Looking forward to Johan's automation which will prevent me forgetting about adaptation branches!

Johan Commelin (Oct 17 2024 at 11:26):

ci(.github/workflows): add discover-lean-pr-testing.yml #17399

waiting for review

github mathlib4 bot (Oct 17 2024 at 11:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d51a8c9ac5f7970ce1d50207a52ff800aa95d956).
You can git fetch; git checkout nightly-testing and push a fix.

Anne Baanen (Oct 17 2024 at 12:07):

Just a shake error, let me fix it...

github mathlib4 bot (Oct 17 2024 at 13:25):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (71802680628fbeb426c7a0c17107eeb67ac18fe0)

github mathlib4 bot (Oct 18 2024 at 04:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fb09b71265c60a58ebf2c1d4fd6b9477d4506d14).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2024 at 06:04):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (71802680628fbeb426c7a0c17107eeb67ac18fe0)

github mathlib4 bot (Oct 18 2024 at 07:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (319d7a37f0e813c9603b8df05901330e49aaf0eb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2024 at 08:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (71802680628fbeb426c7a0c17107eeb67ac18fe0)

github mathlib4 bot (Oct 18 2024 at 08:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b16c5d7fb54a2f624ce50e9b4f9de1e2a26b963).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2024 at 10:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd77f31972aa69d64ea2889b8d154417042e4aba).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2024 at 10:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (23752ee05683cc476abb6f9eb98b63c0eb5d3da1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2024 at 10:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (23752ee05683cc476abb6f9eb98b63c0eb5d3da1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 18 2024 at 10:52):

@Mac Malone, the exit code 3 problem has returned. :-(

Kim Morrison (Oct 18 2024 at 10:52):

I can't make a new release of ProofWidgets for every nightly toolchain. :-(

github mathlib4 bot (Oct 18 2024 at 13:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6c837c78f211be4560cf2b63adb5347e9854b808).
You can git fetch; git checkout nightly-testing and push a fix.

Mac Malone (Oct 18 2024 at 15:38):

Kim Morrison said:

I can't make a new release of ProofWidgets for every nightly toolchain. :-(

That's weird. You shouldn't need to. The Reservoir cache is the only thing I know of which uses the toolchain in its trace, but ProofWidgets doesn't use it (as it uses GitHub releases).

github mathlib4 bot (Oct 18 2024 at 16:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (94bb3a8e89c75b20472ec5a37df0f225cb08e003).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2024 at 19:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (df601e35b5257a5c391ee5ca5648201c4f46cc78).
You can git fetch; git checkout nightly-testing and push a fix.

Mac Malone (Oct 18 2024 at 19:13):

Kim Morrison said:

Mac Malone, the exit code 3 problem has returned. :-(

Which run produced this failure? I could not find that error in any of the recent links in this thread.

github mathlib4 bot (Oct 18 2024 at 22:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (de5d061f84a1fdff844f983aea367c3bdbf676b8).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 18 2024 at 22:27):

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (23752ee05683cc476abb6f9eb98b63c0eb5d3da1).
You can git fetch; git checkout nightly-testing and push a fix.

@Mac Malone, this is the one that failed with exit code 3. Indeed it has gone away again. However it does lot look it is a persistent intermittent problem at this point.

Mac Malone (Oct 18 2024 at 22:33):

@Kim Morrison Well that's even weirder. Nondeterministic trace mimsatches would be quite suprising. Maybe it is some form of network error? It might be worth appned --no-cache to lake build --no-build in that step just to ensure that is never causing the porblem.

github mathlib4 bot (Oct 19 2024 at 01:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6e38c6649191d8bf77deb739de42ae8df4581c0d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2024 at 03:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bd5ba6b8fd201d0165ca6068e0a9437a56c4b58f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2024 at 07:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (74600feef71163f17723cd491710cbe1cec142d7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2024 at 07:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (90c6be64b3540bf42afd057554434af4597f1367).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2024 at 07:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (90c6be64b3540bf42afd057554434af4597f1367).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2024 at 08:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (418a5eb7aec3fb639097cb13f74fc031ac4057f2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2024 at 09:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (66f63643834286e06540e60e459b22c7bbd25475).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (66f63643834286e06540e60e459b22c7bbd25475).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 19 2024 at 11:11):

There are some dubious fixes I just pushed on nightly-testing for lean#5650, in commit c2067f2d8656c8fa417133d981b027b99f47a227.

It's weekend here and I don't have time to think about it beyond getting it compiling right now, but we should revisit this, and see if we can make the API better.

github mathlib4 bot (Oct 19 2024 at 11:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (66f63643834286e06540e60e459b22c7bbd25475).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Oct 19 2024 at 12:17):

Kim Morrison said:

There are some dubious fixes I just pushed on nightly-testing for lean#5650, in commit c2067f2d8656c8fa417133d981b027b99f47a227.

It's weekend here and I don't have time to think about it beyond getting it compiling right now, but we should revisit this, and see if we can make the API better.

Oh my bad, I didn't see the Mathlib errors

github mathlib4 bot (Oct 19 2024 at 12:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (407a4459e2005e212bb230d2746afe980eba7003)

github mathlib4 bot (Oct 20 2024 at 22:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (69bbcb4a9d48465ffcabd3ef9581cc9064df7e06).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 20 2024 at 23:50):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (407a4459e2005e212bb230d2746afe980eba7003)

github mathlib4 bot (Oct 21 2024 at 06:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c8f7de855ad546b004a0ec1172f9c294105be0a4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 21 2024 at 07:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a60b09cd54613409d215c944aebb2cf75991287c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 21 2024 at 08:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (407a4459e2005e212bb230d2746afe980eba7003)

github mathlib4 bot (Oct 21 2024 at 10:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ff1b88672d4e66db5195c5c57684e4081fab209f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 21 2024 at 10:12):

Merging lean-pr-testing-5749 into Batteries, ProofWidgets, Mathlib

Kim Morrison (Oct 21 2024 at 10:22):

@Mac Malone, I just tagged v0.0.44-pre3 on ProofWidgets, than updated Mathlib's nightly-testing to use it.

This then results in:

% lake build
 [91/5264] Ran proofwidgets:extraDep
warning: building from source; failed to fetch GitHub release (run with '-v' for details)

which will result in CI failing for being noisy. How do we make this not happen? :-(

Kim Morrison (Oct 21 2024 at 10:22):

I'm presuming this is some reservoir thing, where it needs to catch up with the tagged release somehow?

github mathlib4 bot (Oct 21 2024 at 10:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1df44a89ac2cd5c83c4b6ea19b2aa5ed3f99c479).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 21 2024 at 10:27):

Oh, my mistake, the CI failed for the tag, it really was building from source. Sorry for the noise.

github mathlib4 bot (Oct 21 2024 at 11:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d43bc00b660d5456721455c8f4e4d1d2244f555b).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 21 2024 at 11:45):

import-graph needed a fix too

github mathlib4 bot (Oct 21 2024 at 12:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d43bc00b660d5456721455c8f4e4d1d2244f555b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 21 2024 at 12:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (26dafbb134ad1635c84c2c81363140e1ba78005e)

github mathlib4 bot (Oct 21 2024 at 13:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d43bc00b660d5456721455c8f4e4d1d2244f555b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 21 2024 at 13:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (26dafbb134ad1635c84c2c81363140e1ba78005e)

github mathlib4 bot (Oct 21 2024 at 19:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3f00b0c794c8e9d0f75cef11354d6efa9a8ceea).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 21 2024 at 21:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3f00b0c794c8e9d0f75cef11354d6efa9a8ceea).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 21 2024 at 22:20):

@Andrew Yang, any chance you could look at this failure in Morphisms/Constructors.lean on the branch nightly-testing?

Kim Morrison (Oct 21 2024 at 22:20):

It's from a PR of yours that landed a few hours ago.

Kim Morrison (Oct 21 2024 at 22:21):

It's fine to just push directly to nightly-testing.

Andrew Yang (Oct 21 2024 at 23:11):

Fixed.
Are syntaxes like this not supported anymore?

example {A B : Prop} (h : A  B) (a : A) : B := by
  refine by simpa using h ?_
  exact a

github mathlib4 bot (Oct 21 2024 at 23:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (26dafbb134ad1635c84c2c81363140e1ba78005e)

Johan Commelin (Oct 22 2024 at 03:56):

I would hope they still are...?

Markus Himmel (Oct 22 2024 at 05:41):

This looks like unintended breakage after lean#5648, which is supported by the fact that nightly-2024-10-09 is the first nightly where this doesn't work anymore. cc @Kyle Miller

github mathlib4 bot (Oct 22 2024 at 07:07):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (26dafbb134ad1635c84c2c81363140e1ba78005e)

github mathlib4 bot (Oct 22 2024 at 08:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (07013722cda97276225650bec2a9635f95807ed6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 22 2024 at 10:14):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5d9876da9e139761f55a9d3bba56cbd11fe5ecf4)

Kyle Miller (Oct 22 2024 at 15:27):

@Andrew Yang That's never supposed to have been supported — it was a bug that the ?_ could escape from its enclosing by.

That said, I think it's a good idea having a refine version of simpa. Maybe simp_refine h ?_ would be good syntax?

github mathlib4 bot (Oct 22 2024 at 16:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5d9876da9e139761f55a9d3bba56cbd11fe5ecf4)

github mathlib4 bot (Oct 23 2024 at 09:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3ed0adc8f4c5f3c0b1cdd195e1c16c0e6fae8e8c)

github mathlib4 bot (Oct 24 2024 at 08:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (893b3a846645d48ac45143ec02149cc551acd99d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 24 2024 at 09:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (893b3a846645d48ac45143ec02149cc551acd99d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 24 2024 at 10:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3307c67acbea9ff66f3a40e0c876b4af694000ab)

github mathlib4 bot (Oct 24 2024 at 14:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f72cbf5998335b7b2863a003a2ce58c11e982418).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 24 2024 at 19:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8fd75accaff95050c8b594847f537bdde54a54ef).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 24 2024 at 22:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0b6c6c4d8f70155aae4dc62d24758734babe479a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 24 2024 at 22:40):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3307c67acbea9ff66f3a40e0c876b4af694000ab)

Kim Morrison (Oct 24 2024 at 23:09):

I also merged lean-pr-testing-5788 in, which had some non-breaking cleanup from lean#5788

github mathlib4 bot (Oct 24 2024 at 23:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9dda7f5db42f6c0e303ca618e1b21995ac435f2f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 25 2024 at 00:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3307c67acbea9ff66f3a40e0c876b4af694000ab)

github mathlib4 bot (Oct 25 2024 at 09:11):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5b391bd6a2dafc56a16caeef82eb19c1c1518104)

Kyle Miller (Oct 25 2024 at 19:48):

(deleted, followed up on my note)

github mathlib4 bot (Oct 25 2024 at 22:02):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5b391bd6a2dafc56a16caeef82eb19c1c1518104)

github mathlib4 bot (Oct 26 2024 at 09:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e91cdbcf5a387801a6225b41b0056c63206a9f7f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 26 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e91cdbcf5a387801a6225b41b0056c63206a9f7f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 26 2024 at 12:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd050c2d54938c9a9b5b827fee930496295b1b0d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 26 2024 at 16:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bf23ca5445dd7509615c489b06dbfc93546c1276).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 26 2024 at 18:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (991921d3bd6203a88526aed794553b0ba2350735).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 26 2024 at 21:26):

https://github.com/leanprover/lean4-cli/pull/19 will fix this failure

github mathlib4 bot (Oct 27 2024 at 01:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (824887828166406874a8ef38feefc05597c91a80).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2024 at 03:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e0bd65eedfa4ffe9616fd33085402c213c4cb01f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2024 at 09:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f4ae1ea6c6f6511fec1a5d5f35a433ca2c977592).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2024 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (89bb4c76891eeef01b806d7dcfe3f19346ec3c0d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2024 at 13:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1a0cb23be5d4c6eae78ac6ac9ae8f365b1b1b2d6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2024 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6264905204f3ed595bc99032ec15af1910a0eddd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2024 at 19:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f0c67a9c1b8352739a65e8438f218cb11278ab12).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2024 at 22:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (380f469e41f87c305b0706bc38dc1b785603e481).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2024 at 23:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (be300cdc068254562106cb8ab789da120de5acf2)

Kyle Miller (Oct 28 2024 at 01:25):

I just put lean4#5853 on the merge queue. This breaks mathlib, but the only thing that should need doing is to bump aesop, which has already been fixed.

github mathlib4 bot (Oct 28 2024 at 01:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (be300cdc068254562106cb8ab789da120de5acf2)

github mathlib4 bot (Oct 28 2024 at 08:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9fc60c1ad982f142d6d0671bef8f4cda3b1590cd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 28 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (38a786e886cee8d56c2bdf03fa56b925828fa7b7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 28 2024 at 10:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f381acde43bf099c306f588941df4014ea3ecfcf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 28 2024 at 11:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (347ad1b741a37bbe745a46cd0d0ff06aa4f80965)

github mathlib4 bot (Oct 28 2024 at 13:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (73c9a6385f7abed888796762e8d6cc0877e6a267).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 28 2024 at 15:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (afa7411cbae5122045f191b6e2b9d7f7e799fce5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 28 2024 at 18:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4e5fa6379d912f52eb8a4bacac4dd9eb0c75fca3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 28 2024 at 21:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1d847d8cc0ca7c2e574a4a4ac22ba1b8607aea94).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Oct 28 2024 at 22:01):

This last failure is puzzling. It's a simp [forall_swap] that's started to reach max recursion steps (commit with fix: https://github.com/leanprover-community/mathlib4/commit/08c4816adebb4419e3e5f51aa27fe90d55f8afe7)

I'm not sure why it would suddenly start to fail. There don't seem to be any Lean changes that would have triggered it...

github mathlib4 bot (Oct 28 2024 at 22:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1d847d8cc0ca7c2e574a4a4ac22ba1b8607aea94).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 00:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ef637a3d76ee66c95ffd58ad10a8231e91744115).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 04:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3e82c092e760d870aa677ac508c210e28b715fa9).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Oct 29 2024 at 04:22):

Kyle Miller said:

This last failure is puzzling. It's a simp [forall_swap] that's started to reach max recursion steps (commit with fix: https://github.com/leanprover-community/mathlib4/commit/08c4816adebb4419e3e5f51aa27fe90d55f8afe7)

I'm not sure why it would suddenly start to fail. There don't seem to be any Lean changes that would have triggered it...

I worked around it on #18333 by changing to simp; tauto

github mathlib4 bot (Oct 29 2024 at 06:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5a7979109839909b50de2d135fb1f39c3dacebf5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 08:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fe4820c926372190e01f6404c555c1ad2f0cf7e0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 09:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d27f22898a74975360dd1387155c6031b501a90b).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 29 2024 at 10:17):

Merged lean-pr-testing-5719

github mathlib4 bot (Oct 29 2024 at 10:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6c2c697b464663f1ed09ade11e0204970ddd95aa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 13:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dfbe436509d43c243ecce8dac9782f7f5632c239).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 16:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f4f0b47a2f859d27e965c812344deb1435fe8d48).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 19:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5724fc0c3e05bb9d503aea86f8513a3696e595f3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c8dae00520db0c6b41b68a7a26af9527e8db4f6c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 22:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d77087c5820546f8f47eaffe2c13f16df19dd47d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2024 at 23:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c96009ebab6853de093abfa12ccae9601bfc6ec8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2024 at 00:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4478d113e456c870c14d99246808b74783756287)

github mathlib4 bot (Oct 30 2024 at 09:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (153aff575c32e0e84efb0b470bdf6cec96a6c29e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2024 at 10:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (250bf30b823d812379be4b3b5fe134edbc6ea8cc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2024 at 10:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (250bf30b823d812379be4b3b5fe134edbc6ea8cc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2024 at 11:05):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (19a2e289f248500411b87004e36f407e44c4c010)

github mathlib4 bot (Oct 31 2024 at 04:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2bf9cc643615d0e50a7db023ec645a0340f2e4dc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 31 2024 at 04:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (19a2e289f248500411b87004e36f407e44c4c010)

github mathlib4 bot (Oct 31 2024 at 08:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (348232e527e0363cd27a7a49302dad2de3817be6).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 31 2024 at 08:32):

Merged Kyle's lean-pr-testing-5883 here and at Batteries

github mathlib4 bot (Oct 31 2024 at 09:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (0af7fdf367d4a47093030a029e183fc2530cede4)

github mathlib4 bot (Nov 01 2024 at 08:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (318cb7184d6e13f32a69869057dab5bcfe652f0d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 01 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (50373971524c5c08b75a06665756d44fd30ac05a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 01 2024 at 09:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (50373971524c5c08b75a06665756d44fd30ac05a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 01 2024 at 09:52):

Merging Kyle's lean-pr-testing-5898 into batteries/aesop/mathlib's nightly-testing branches.

github mathlib4 bot (Nov 01 2024 at 09:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (50373971524c5c08b75a06665756d44fd30ac05a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 01 2024 at 09:59):

Oof, now plausible needs updating for nightlies. :-)

Kim Morrison (Nov 01 2024 at 10:01):

Hopefully all good now, local build is past all the dependencies / meta code.

github mathlib4 bot (Nov 01 2024 at 11:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c68aa1080b4c5bc32adfb1fe9cb3f161cf5b13d8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 01 2024 at 13:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (743d65a7ce14876af9021b7af600a1946a6b431d).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Nov 01 2024 at 15:54):

It seems to be just that there was a lingering Slimcheck file (deleted it)

Kyle Miller (Nov 01 2024 at 15:57):

It seems like the file came back from the dead because List.modifyNth became List.modify (commit), and it wanted to be around to see that happen.

github mathlib4 bot (Nov 01 2024 at 16:09):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (55da1f83fea32853a6da79f84316361e646fc365)

github mathlib4 bot (Nov 02 2024 at 09:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (df174a8a32fb9b7661ec4faa48a6a6a6bb4cf0d5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2024 at 10:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (21d62a67f9e364212415055c3138bf879c771b20).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2024 at 13:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c46b5e46c884d1448ba12aa9bdc04f71cc295cbc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2024 at 15:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c07a25e93dddd2ad980b28ea52881242dccbf90).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2024 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2fc69c7f2cf8a673b129d21c537c69c4d48cb774).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2024 at 19:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ef5ff126f83dceb492b40f3b30c19cc071eac163)

github mathlib4 bot (Nov 03 2024 at 09:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (022e83a3574b2369be549178ef7a785b7c716f51)

github mathlib4 bot (Nov 03 2024 at 15:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3a51a909fe294510e91d071384eeef5e7344bef9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 03 2024 at 19:06):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (022e83a3574b2369be549178ef7a785b7c716f51)

github mathlib4 bot (Nov 04 2024 at 04:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fef6aa3e68311f7ddb82e3db00441493b0e6f39a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2024 at 07:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a7fc949f1b05c2a01e01c027fd9f480496a1253e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2024 at 08:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cff2508ca636dcec162d11f5c0394f1705753a38).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 04 2024 at 09:16):

(I also made a new branch for nightly-testing here and at Batteries. The histories are still preserved via the nightly-testing-YYYY-MM-DD tags.)

github mathlib4 bot (Nov 04 2024 at 09:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6e98b4c07c04bcff5170ffd7adef179d951dbb0b).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Nov 04 2024 at 09:34):

@Kim Morrison Sorry, what do you mean by that exactly? You created a new bump/v15 branch? Or you deleted and recreated nightly-testing? Or did a hard reset to branch it off master again?

github mathlib4 bot (Nov 04 2024 at 10:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15f99d44becdf94acbc9f295f44b8f267b508a2c).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 04 2024 at 10:26):

I deleted and recreated nightly-testing.

github mathlib4 bot (Nov 04 2024 at 10:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15f99d44becdf94acbc9f295f44b8f267b508a2c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2024 at 11:21):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b28f0d7f7e9cc3949a9a3556a6b36513f37f690d)

github mathlib4 bot (Nov 04 2024 at 13:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0317a26931dd41612066dc1c8c91a8273673e2f4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2024 at 16:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ddff18e6d123171cc1d13d35fc0f2a062ebdcd48).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2024 at 19:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2f5cf5f572ab008ffe1ffad76ede50ef47df4df5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2024 at 22:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b28f0d7f7e9cc3949a9a3556a6b36513f37f690d)

Kim Morrison (Nov 05 2024 at 00:14):

We need to merge lean-pr-testing-5684 tonight.

github mathlib4 bot (Nov 05 2024 at 01:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8bad983b8e4adf7e111ef16e32e757bb95ef63e3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 05 2024 at 01:36):

Fixed by #18638, which I've pre-emptively merged into nightly-testing.

github mathlib4 bot (Nov 05 2024 at 01:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b28f0d7f7e9cc3949a9a3556a6b36513f37f690d)

github mathlib4 bot (Nov 07 2024 at 13:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (84343c902b917981ea5c2146ce0074c09c338984).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 07 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d08f234e81a8adb77a5df040dda32092d8964715).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 07 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c5adc80d438877328f3307b59a66357d9b1f95b3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 07 2024 at 21:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (66e27ecedabdda28d551ab10b40fbbdaedcba63a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 07 2024 at 22:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (97f7ee9b324296da144822b21fb35c2fce16bbbc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 08 2024 at 01:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9df8b6aac62ef81b72e7ff026ffb3dd7ea81371d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 08 2024 at 06:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9df8b6aac62ef81b72e7ff026ffb3dd7ea81371d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 08 2024 at 06:40):

@Mac Malone, again we have lake build --no-build failing with exit code 3. This has persisted across several commits to nightly-testing. Could you please take a look?

Damiano Testa (Nov 08 2024 at 07:21):

Yesterday I had a PR which restored the CI step that would skip looking for all the cache if the cache for Mathlib.Init was not available. Should this step be reverted again?

Damiano Testa (Nov 08 2024 at 07:22):

#18715 is the merged PR.

github mathlib4 bot (Nov 08 2024 at 08:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (48b340091dc38c6be2696ba59b63bc4f1cd86d24).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 08 2024 at 09:29):

As far as I understand, this problem is orthogonal to the fast-failing cache check.

Damiano Testa (Nov 08 2024 at 10:28):

Ok, good to know. I simply flagged it, since the restored CI step uses --no-build.

github mathlib4 bot (Nov 08 2024 at 12:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (682fb6e943f5985f9e7b3fc6681c3706fba888d8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 08 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (31c320e6adec695a8c070a78bb956e0fc5401431).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 08 2024 at 19:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd877e3244c9fc6f620484aa36b581ac20811878).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 08 2024 at 22:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (efb737da256e54a73006dbac848020821143eff8).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 08 2024 at 22:30):

Damiano Testa said:

Ok, good to know. I simply flagged it, since the restored CI step uses --no-build.

Oh, I see, then I'm wrong, and the restored CI step is revealing the bug in Lake.

Damiano Testa (Nov 08 2024 at 22:43):

Ok, sorry for re-introducing the issue. It is a little puzzling (to me) that this is affecting nightly-testing, but no one reported problems on mathlib.

github mathlib4 bot (Nov 09 2024 at 00:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (efb737da256e54a73006dbac848020821143eff8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 09 2024 at 09:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (905613ccc46988d1431e544d83158227cb015790).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 09 2024 at 13:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5476cef777111bb7a13cd11b7ba78b24fdb2d04f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 09 2024 at 13:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5476cef777111bb7a13cd11b7ba78b24fdb2d04f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 09 2024 at 15:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (42ff2ccb6d99b39a65e43b8da21a60f8e7d3f9ca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 09 2024 at 18:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7fc8954db7c3e9619b2055e97afeda277df11e5a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 09 2024 at 21:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (62a2cc31bac6416736c17a57383a622c208f21cb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 10 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (16c9d8c2fba7254dbeb6e41eeb0554c23e5776ec).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 10 2024 at 08:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1964227ee4bc4a748a0fd3b7538fb3624bd53cdf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 10 2024 at 10:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b696b3524d2dde1068fa8192e92f25c990e9eb15).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 10 2024 at 13:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dcd0c54029474826f732df2e67dad6f62d036801).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 10 2024 at 15:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b17bf258da6542cd3a553ea33c03db938506ae92).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 10 2024 at 22:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (984b731629ca16feec9631b2fe29c3f8119d2545).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 10 2024 at 22:56):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (db9c4895583aedbcffefebb9a1396e49dd353076)

github mathlib4 bot (Nov 11 2024 at 01:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9e22d44c80076d35898385cbd9b7603b9ad578b1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2024 at 04:19):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (db9c4895583aedbcffefebb9a1396e49dd353076)

github mathlib4 bot (Nov 11 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8fa662232f9bac9afad1064b6807f885ecb42a6b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2024 at 08:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5c97de1d46f7ea0dcaabd3689510f84926715b67).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2024 at 09:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (46252974983857475e0005be6539778f72aa506a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2024 at 10:43):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3894c72cbd6f4baba45c79678e75503123a51756)

github mathlib4 bot (Nov 11 2024 at 11:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ba0f793af59c9d09b2590bb84bed18e0c953598d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7f8c9accc0593e2d7adfe688ba65214abd9f44b4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2024 at 15:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b0171e1b8e46b017a2622acbb69a741228c5a9f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2024 at 18:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (25a6e587b921c3b70390d43d3e304d0a9e44e480).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2024 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (33a52a30ef58e82cba9f316ddad5fc903c45b30d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 00:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (69fd87072626b8778f5553717c4f0f9646ce9664).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 03:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3894c72cbd6f4baba45c79678e75503123a51756)

github mathlib4 bot (Nov 12 2024 at 08:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6e5c57744c0c760f11f5a74683da6c6ff1e73816).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (62c60f4c54985095037900d549069c5afa055b9f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 09:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (62c60f4c54985095037900d549069c5afa055b9f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 09:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (62c60f4c54985095037900d549069c5afa055b9f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 12 2024 at 10:00):

Merged lean-pr-testing-5988 here and on Aesop's nightly-testing.

Kim Morrison (Nov 12 2024 at 10:09):

Merged lean-pr-testing-5920

github mathlib4 bot (Nov 12 2024 at 10:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (92699559c4c13dd39c2fa73633c20bf5da322a19).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 13:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (601e532385c74a1527c61fce3042634418c09171).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 16:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b00c9dba4d70ab0ba583936391d41c5d5df86681).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 18:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15ae5b0cba066b5763f837b84afa57cce9a600c7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 20:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (66f0c7ed474d768e06dd41e9c30783069aefb1ef).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 12 2024 at 21:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (6c3ffb61f93289ca8959e436efe546e7d3465f78)

github mathlib4 bot (Nov 13 2024 at 01:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aafab103590f19e7d5dc03f376a4622a8c5249e7).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 13 2024 at 03:14):

We'll need to merge lean-pr-testing-6054 at Batteries, Aesop, and Mathlib tonight.

github mathlib4 bot (Nov 13 2024 at 03:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aafab103590f19e7d5dc03f376a4622a8c5249e7).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 13 2024 at 05:20):

We're waiting on me getting #18947 in.

github mathlib4 bot (Nov 13 2024 at 07:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ce14f6c28d27d389898dc60307f76ca511001b31).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 08:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5b7d4f674417bd4f778070920a6e206c08142eab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0a4bd52842b793900a2d13769c73f41c9cd6ed79).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 10:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c2ac85e66c4afd79b177c6e4dd6c4a801a97c435).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 11:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a98955eeb755f7c066f31e9e4d896b90c4d83b31).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 13 2024 at 11:11):

Separately from the linter problems we're having at the moment, nightly-testing is failing in Mathlib/AlgebraicGeometry/Spec.lean.

If either @Andrew Yang or @Jujian Zhang (recently touching the relevant declaration! :-) might have a chance to take a look that would be much appreciated.

Andrew Yang (Nov 13 2024 at 11:53):

I'm not sure what's the best way to solve the missing IsLocalHom instance. Can @Jiang Jiedong please take a look? Thanks!

Kim Morrison (Nov 13 2024 at 11:57):

Oh -- this is probably fallout from Kyle's bug fix PR. I didn't merge all of his changes yet.

Kim Morrison (Nov 13 2024 at 11:58):

Not at a computer, but maybe trying to merge in lean-pr-testing-6204??

Kim Morrison (Nov 13 2024 at 12:00):

Sorry, 6024.

Jiang Jiedong (Nov 13 2024 at 12:20):

I fixed the error by filling an underline with explicit argument. Shall I commit directly to this branch?

Jiang Jiedong (Nov 13 2024 at 12:32):

I have just pushed my fixing commit

github mathlib4 bot (Nov 13 2024 at 12:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3597f15bb5cd3e841064f98286c5549b22818a99).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 13:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1cf210c363adf58a21a13e28695c1c3989ff1869).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 16:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b99f4d538e246c7205bcb081030d98eaa81ab47).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 19:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (798302c55eff0d7f2543f7540e8cdb205efbc48c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 20:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b9e10907eb01edd5d7c088a0e7aa9164f28e0dae).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2024 at 22:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (00a090b2e31c5b97ac9b6aa8b49d6e6319b74c6b).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 13 2024 at 22:51):

Just getting back to this now. The simpNF linter is thoroughly broken, and reports Left-hand side does not simplify, when using the simp lemma on itself. on essentially everything.

Kim Morrison (Nov 13 2024 at 22:56):

This is not unexpected: we just changed the interface for calling into the simplifier from meta code. Presumably I've made a mistake in adapting to this interface change.

Kim Morrison (Nov 13 2024 at 22:56):

But so far I am not seeing it. :-(

Kim Morrison (Nov 14 2024 at 00:13):

Should come good shortly.

github mathlib4 bot (Nov 14 2024 at 01:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (749157dda17c2c89da84d1dec01607893379fb73).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 14 2024 at 01:29):

Sigh, these appear to be genuine linter failures.

Kim Morrison (Nov 14 2024 at 01:39):

Nope, more mistakes in me updating tactics.

github mathlib4 bot (Nov 14 2024 at 02:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (bae40f51101fe0dbebff6d6a5f56532ca845f1f4)

github mathlib4 bot (Nov 14 2024 at 04:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4ac7881bba2522f56411a175689efe7039731fb9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2024 at 05:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (bae40f51101fe0dbebff6d6a5f56532ca845f1f4)

github mathlib4 bot (Nov 14 2024 at 07:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a5a981b8ba66b70614f0e096595389e7a46d17c5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2024 at 08:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (334be41cd6a4737ac24813c926c6f61fcedd1998).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 14 2024 at 08:32):

The recently added file Mathlib/FieldTheory/Relrank.lean (mathlib4#14987) almost goes over the synthInstance.maxHeartbeats limit on master, and goes over on nightly-testing. I've had to add five copies of

set_option synthInstance.maxHeartbeats 400000 in

in this file on nightly-testing.

Kim Morrison (Nov 14 2024 at 08:34):

Just pinging @Jz Pan, @Andrew Yang, @Johan Commelin, who authored/reviewed the PR in case any are available to take a look at this and see if anything can be done.

github mathlib4 bot (Nov 14 2024 at 08:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (334be41cd6a4737ac24813c926c6f61fcedd1998).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 14 2024 at 08:53):

Just a heads up @Mac Malone that nightly-testing at b0a9ae37ac9cfaf7f106c8c88253e09beab56c34 gets stuck at

% lake build
 [?/?] Computing build jobs

As usual, this is probably because I've deleted a file in Batteries; although this time Mathlib itself doesn't import the deleted file. I'll go look through the intermediate repos to see if they use it.

Kim Morrison (Nov 14 2024 at 08:57):

Indeed, import-graph used the deleted file. Once I remove those imports from import-graph, and run lake update importGraph in Mathlib, the build starts properly.

Kim Morrison (Nov 14 2024 at 08:57):

So perhaps this is a clue about reproducing the problem -- we need a chain of three projects?

github mathlib4 bot (Nov 14 2024 at 09:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (334be41cd6a4737ac24813c926c6f61fcedd1998).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2024 at 09:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e3d7d7f053ea862ffb7d1613eff6de0f2e3e8e14).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 14 2024 at 09:24):

Some more fallout from lean#6024

github mathlib4 bot (Nov 14 2024 at 10:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4bd54c44efaeb057176edd9431ce5c38ab0f41db).
You can git fetch; git checkout nightly-testing and push a fix.

Jannis Limperg (Nov 14 2024 at 10:25):

Kim Morrison said:

This is not unexpected: we just changed the interface for calling into the simplifier from meta code. Presumably I've made a mistake in adapting to this interface change.

Could you point me to this change? Might be relevant for Aesop as well.

Kim Morrison (Nov 14 2024 at 10:26):

@Jannis Limperg, the aesop changes are on https://github.com/leanprover-community/aesop/commit/1aab79ccb4119e27c123d8e237af34097d865187

Kim Morrison (Nov 14 2024 at 10:26):

(this is already present in Aesop's nightly-testing branch)

Kim Morrison (Nov 14 2024 at 10:26):

lean#6054

Jannis Limperg (Nov 14 2024 at 10:28):

Ah great, thanks!

Kim Morrison (Nov 14 2024 at 10:33):

(Haven't run lake test on Aesop's nightly-testing branch recently; that might not hurt! :-)

github mathlib4 bot (Nov 14 2024 at 10:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4bd54c44efaeb057176edd9431ce5c38ab0f41db).
You can git fetch; git checkout nightly-testing and push a fix.

Jannis Limperg (Nov 14 2024 at 12:02):

Kim Morrison said:

(Haven't run lake test on Aesop's nightly-testing branch recently; that might not hurt! :-)

You're braver than I, but lake test succeeds on nightly-testing. :tada:

github mathlib4 bot (Nov 14 2024 at 13:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fd92bc36215a9632f15c6482fb0132d24e6c49ab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2024 at 16:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (95ee83bc7ead3af5cf774c227781aa79c01d9b02).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2024 at 19:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2ee23a34530f8024d3c41b837aca27f979aa129e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2024 at 21:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (daed990be85bb8fa9ad519b2c3249146f6ca11b7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2024 at 23:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5d03a2cd14f5dbfd233359a68d31fd12ad9a535e)

github mathlib4 bot (Nov 15 2024 at 08:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3805203e1e80948a62f00d3c3923bd8b31f16533).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 15 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15661bfd114cd662e6db347d7869fe509a5f5333).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 15 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (089baee31dfe119a919641184bea4b0d0401c30b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 15 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f9aff52fa3e370883f017c09cfc12be23edae5c5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 15 2024 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4887c6cd78f40a84bf1f1597c9fe79028968efdc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 15 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (290eb3b99a6390afda429a510a0dd7ae2b52b65e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 16 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (22b5743395628f2dc74e4acdbbe3856b03053722).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 16 2024 at 03:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (46215793fb6b682b6eeae1960e3266f0aadd5794).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 16 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bc7827342b0d7a3025f4a34100174550c59c4ca1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 16 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6270f3467257beb5cf5118e21a98a0734356657e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 16 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7b8edbb98887af54a4cb8e8f76fa279960233c22).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 16 2024 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2aeb15532ae2dcb0c4119ce6e5e5825811af14f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fe4de19cc7609bc70565b7a712202dc78ee54336).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 03:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e3327a6356ba7550fa37b50f16e934a4d59dc6af).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 07:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e3327a6356ba7550fa37b50f16e934a4d59dc6af).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 09:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (59e75948eb18b0946b93c99d666844ca885675c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 09:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (59e75948eb18b0946b93c99d666844ca885675c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 09:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (59e75948eb18b0946b93c99d666844ca885675c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 09:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (59e75948eb18b0946b93c99d666844ca885675c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 11:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (59e75948eb18b0946b93c99d666844ca885675c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 11:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (89e8f886145b9fbd4543ff7b8e1f0cf39a4e009c)

github mathlib4 bot (Nov 17 2024 at 19:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (08ac4589995d198221a35f21c83467aba483fb3a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (38affacc35abeefc7fd0c782d547d6b745281ad7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 23:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (38affacc35abeefc7fd0c782d547d6b745281ad7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2024 at 23:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (89e8f886145b9fbd4543ff7b8e1f0cf39a4e009c)

github mathlib4 bot (Nov 18 2024 at 06:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d2568da6e252a1bb378b585d39dcf12dd814f946).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2024 at 08:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6d297a4172e6c37d3bf82e68924c45d72621ac5d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2024 at 09:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6d297a4172e6c37d3bf82e68924c45d72621ac5d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2024 at 10:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (66df24a8e2b60b44dbe1def58ad03a083b80e865).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2024 at 13:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c6450e45a0b2b45662a8289c3d0fbf09883939f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2024 at 16:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b04165d049454c0676bf3fa5e3633555af887f6e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2024 at 19:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2ff73d5985b6084b9a7b3f402b90de35951c3e1c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2024 at 22:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (654802e5ec7c62e0cf1f45dfbdaa746af1b81967).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2024 at 22:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (436211744e3cfc6ceefe33edf3f22adf4fce6aff).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 19 2024 at 01:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (812897a4585e90015527a14b09bd40d68c996be7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 19 2024 at 01:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (971d01d592ff5787e284ab48d59340f1715ad2d6)

github mathlib4 bot (Nov 19 2024 at 01:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (812897a4585e90015527a14b09bd40d68c996be7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 19 2024 at 02:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (971d01d592ff5787e284ab48d59340f1715ad2d6)

github mathlib4 bot (Nov 19 2024 at 09:21):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (60a189e5bc5c59e67faa3f3445229e76298ce4dc)

github mathlib4 bot (Nov 19 2024 at 22:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (29f545b8110e796db8de688fa9e3950ce95cf678).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 19 2024 at 22:53):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (60a189e5bc5c59e67faa3f3445229e76298ce4dc)

Kim Morrison (Nov 20 2024 at 10:42):

I was about to say "wow, a day without breakages", except that it is the nightly itself that broke. :-)

github mathlib4 bot (Nov 20 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cd4d2185e67b7387e303150dab86521007c56fb6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2024 at 13:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cd4d2185e67b7387e303150dab86521007c56fb6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2024 at 13:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cd4d2185e67b7387e303150dab86521007c56fb6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (92f63d5c1988987aa375830b9b41cbfd269c3625).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8e0d70c35dcdbe42cd6fa06c579a118735380526).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (961ee9dbff2b14a178fa757f097b5bb27c274e99).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 20 2024 at 22:02):

I think #19204 still didn't run today, @Johan Commelin, could you check the error log?

github mathlib4 bot (Nov 20 2024 at 22:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (33e7503de887ec81d3b24de62cfce9440ffa55a8)

github mathlib4 bot (Nov 21 2024 at 01:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (50c8065ea373f936358889d6eae523a8fde8ae34).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Nov 21 2024 at 04:15):

@Kim Morrison I configured the workflow to only run when lean-toolchain changes. And the last time that happened, we still had the old workflow file.

Johan Commelin (Nov 21 2024 at 04:16):

But it's good that I realize this now. Because it means we shouldn't just use the latest two nightly tags.

Johan Commelin (Nov 21 2024 at 04:47):

@Kim Morrison #19316 should improve two things:

  • actually determine the two nightlies that were used on nightly-testing before and after bumping
  • actually fetch all the history between those two

Kim Morrison (Nov 21 2024 at 04:55):

actionlint points out a syntactical problem, otherwise :peace_sign:

github mathlib4 bot (Nov 21 2024 at 07:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab49b8360a2fb3a08e63cf0c0bc344d4827eeb53).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 21 2024 at 08:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab49b8360a2fb3a08e63cf0c0bc344d4827eeb53).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 21 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1e5f38b9c9889a1375c1007ac707aa325c895a18).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 21 2024 at 11:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8ce05c99ea86bd5531e5a84a45f04cefa20df502)

Johan Commelin (Nov 22 2024 at 05:11):

@Kim Morrison Guess what... passing around multiline strings vs $GITHUB_OUTPUT needs a different strategy: #19355

Johan Commelin (Nov 22 2024 at 05:11):

I really hope people 10 years from now will look back in horror upon our "how to write and test CI workflow" workflows.

Johan Commelin (Nov 22 2024 at 05:12):

Because if they don't, it means that our current workflows will have become normal

Kim Morrison (Nov 22 2024 at 06:01):

It will all be written in Lean, and verified (via AI, silently unless something is wrong) against a formal model of the CI environment. Right???

github mathlib4 bot (Nov 22 2024 at 06:33):

We will need to merge the following branches into nightly-testing:

origin/lean-pr-testing-6128

Johan Commelin (Nov 22 2024 at 06:33):

Does that look mildly correct?

Kim Morrison (Nov 22 2024 at 06:34):

Let me go check. :-)

Johan Commelin (Nov 22 2024 at 06:34):

Most importantly: I'm about to leave my computer, and this action now runs on every push to nightly-testing. If that becomes annoying, please partially revert #19355, so that it only runs when lean-toolchain changes.

Johan Commelin (Nov 22 2024 at 06:34):

Also, I guess we should linkify the output.

Johan Commelin (Nov 22 2024 at 06:35):

But now I need to run

Kim Morrison (Nov 22 2024 at 06:35):

No, I think it is wrong, and we merged that one already yesterday.

Kim Morrison (Nov 22 2024 at 06:35):

But what's an off by one error. :-)

Johan Commelin (Nov 22 2024 at 06:36):

https://github.com/leanprover-community/mathlib4/actions/runs/11967694089/job/33365313381#step:5:35 also shows that we should expect more than 1 PR to be posted

Johan Commelin (Nov 22 2024 at 06:37):

Ghaaarhg, anyway, this was progress

Johan Commelin (Nov 22 2024 at 06:37):

Now I'm really gone for real until +3hrs

github mathlib4 bot (Nov 22 2024 at 06:56):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8ce05c99ea86bd5531e5a84a45f04cefa20df502)

github mathlib4 bot (Nov 22 2024 at 08:34):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 22 2024 at 08:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2bb0410843932d03ff2c12cd9bf2e996f514a36b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 22 2024 at 09:34):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

Damiano Testa (Nov 22 2024 at 09:48):

Would it be better to print the branches on separate lines? Maybe even printing lines of the form

git merge origin/adomani/bench_update
git merge origin/ci-update-checkout
git merge origin/eric-wieser/fix-update_dependencies-errors
...

github mathlib4 bot (Nov 22 2024 at 09:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8e3e89e9b3c5b0a719dea497f46946c860381031).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 22 2024 at 12:10):

In fact, the correct branch to be merging right now is lean-pr-testing-6139. :-)

github mathlib4 bot (Nov 22 2024 at 12:13):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 22 2024 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0c44f3226511eec8ec0fbef477cc35921fe0fa2d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 22 2024 at 12:44):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 22 2024 at 13:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0c44f3226511eec8ec0fbef477cc35921fe0fa2d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 22 2024 at 15:35):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 22 2024 at 16:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (be959a9ade921f874584eb5761e7c4f6c82f6651).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 22 2024 at 18:37):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 22 2024 at 19:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3d401e0bb3b0295605d8083d5683efd6dbbea2eb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 22 2024 at 21:33):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 22 2024 at 21:39):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 22 2024 at 22:10):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (714674cc3646c9d15485e7cf26fb8c1b22655a64)

github mathlib4 bot (Nov 23 2024 at 00:47):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 01:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (714674cc3646c9d15485e7cf26fb8c1b22655a64)

github mathlib4 bot (Nov 23 2024 at 02:31):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 02:42):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (714674cc3646c9d15485e7cf26fb8c1b22655a64)

Johan Commelin (Nov 23 2024 at 04:30):

#19392 does better tracing and better output formatting of the list of PRs.
I hope the better tracing will allow me to understand why we are matching branch names that do not even contain digits.

github mathlib4 bot (Nov 23 2024 at 06:37):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6139 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 07:18):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (714674cc3646c9d15485e7cf26fb8c1b22655a64)

github mathlib4 bot (Nov 23 2024 at 08:36):

We will need to merge the following branches into nightly-testing:

origin/adomani/bench_update origin/ci-update-checkout origin/eric-wieser/fix-update_dependencies-errors origin/lean-pr-testing-6125 origin/mrb/updates origin/tfae-block-syntax-update origin/update-PrincipalIdealDomain-docs origin/update-dependencies-2024-06-26-03-06 origin/update-dependencies-2024-06-26-04-06 origin/update-dependencies-bot-use-only origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 09:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ba61bf3e0b903f7186a3861a6cf1d704a1bed7c0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 23 2024 at 09:33):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-PrincipalIdealDomain-docs\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 09:45):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-PrincipalIdealDomain-docs\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 10:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d1d52a625399fe9f91ef60a29818f4005053e70c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 23 2024 at 11:31):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-PrincipalIdealDomain-docs\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-dependencies-bot-use-only\n- origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 11:42):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d1f4f68c3cd7162e8b86e5ae3a27eb0250fb8095)

Johan Commelin (Nov 23 2024 at 12:27):

Aahrg, why is escaping so hard.

Ruben Van de Velde (Nov 23 2024 at 12:35):

Because you're writing shell code :)

Johan Commelin (Nov 23 2024 at 12:38):

#19405 filters out stage0 updates from the lean4 commit log, since those are not made by PRs.

github mathlib4 bot (Nov 23 2024 at 12:44):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-PrincipalIdealDomain-docs\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-dependencies-bot-use-only\n- origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 13:16):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d1f4f68c3cd7162e8b86e5ae3a27eb0250fb8095)

github mathlib4 bot (Nov 23 2024 at 15:33):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-dependencies-bot-use-only\n- origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 16:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d1f4f68c3cd7162e8b86e5ae3a27eb0250fb8095)

github mathlib4 bot (Nov 23 2024 at 18:36):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-dependencies-bot-use-only\n- origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 18:53):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d1f4f68c3cd7162e8b86e5ae3a27eb0250fb8095)

github mathlib4 bot (Nov 23 2024 at 21:33):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-dependencies-bot-use-only\n- origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 21:49):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d1f4f68c3cd7162e8b86e5ae3a27eb0250fb8095)

github mathlib4 bot (Nov 23 2024 at 22:43):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-dependencies-bot-use-only\n- origin/update-import-script

github mathlib4 bot (Nov 23 2024 at 22:54):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d1f4f68c3cd7162e8b86e5ae3a27eb0250fb8095)

github mathlib4 bot (Nov 24 2024 at 00:48):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-dependencies-bot-use-only\n- origin/update-import-script\n- origin/update_deprecations

github mathlib4 bot (Nov 24 2024 at 01:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d1f4f68c3cd7162e8b86e5ae3a27eb0250fb8095)

github mathlib4 bot (Nov 24 2024 at 09:34):

We will need to merge the following branches into nightly-testing:

\n- origin/adomani/bench_update\n- origin/ci-update-checkout\n- origin/eric-wieser/fix-update_dependencies-errors\n- origin/lean-pr-testing-6125\n- origin/mrb/updates\n- origin/tfae-block-syntax-update\n- origin/update-dependencies-2024-06-26-03-06\n- origin/update-dependencies-2024-06-26-04-06\n- origin/update-dependencies-bot-use-only\n- origin/update-import-script\n- origin/update_deprecations

github mathlib4 bot (Nov 24 2024 at 10:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (db0487a4dbe7caa9f45514455f4edddbc56d0505)

github mathlib4 bot (Nov 25 2024 at 08:38):

We will need to merge the following branches into nightly-testing:

  • origin/lean-pr-testing-6194

Kim Morrison (Nov 25 2024 at 08:39):

The formatting is correct!

github mathlib4 bot (Nov 25 2024 at 08:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a41d8f43ee87309b9bb3c4f23c473a5fcbc2e922).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 25 2024 at 08:40):

and lean#6194 was merged today, and lean-pr-testing-6194 has adaptations on it. Looks great!

Johan Commelin (Nov 25 2024 at 08:43):

@Kim Morrison Shall I switch back to running the workflow only when lean-toolchain is touched?
Because atm it runs on every push to nightly-testing.

github mathlib4 bot (Nov 25 2024 at 08:43):

We will need to merge the following branches into nightly-testing:

  • origin/lean-pr-testing-6194

Kim Morrison (Nov 25 2024 at 08:43):

Yes please. :-)

Kim Morrison (Nov 25 2024 at 08:44):

I've now merged lean-pr-testing-6194 into both batteries and mathlib's nightly-testing.

Kim Morrison (Nov 25 2024 at 08:45):

There are still errors, because I merged lean#6195 without fixing Mathlib. (i.e. the bot is correctly not mentioning that!)

github mathlib4 bot (Nov 25 2024 at 08:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a41d8f43ee87309b9bb3c4f23c473a5fcbc2e922).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Nov 25 2024 at 08:47):

@Kim Morrison @Damiano Testa voila: #19450

github mathlib4 bot (Nov 25 2024 at 08:47):

We will need to merge the following branches into nightly-testing:

  • origin/lean-pr-testing-6194

Johan Commelin (Nov 25 2024 at 08:49):

I'm really happy that the formatting was fixed here. Kudos to @Damiano Testa !

Damiano Testa (Nov 25 2024 at 08:49):

I don't know why formatting is so hard: it feels like there would be nothing special to it, and yet...

github mathlib4 bot (Nov 25 2024 at 08:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a41d8f43ee87309b9bb3c4f23c473a5fcbc2e922).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5fde9dcf705fe1d732a15da3dda14a624a95237f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 11:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b96544419e0739c6aefecfc4ee368400a77266ce).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 13:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7f28d7f73f74b31f72449bb9eb240db3ca68fe38).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 16:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (04cd3d0afc11a0bcb07934a8e2f12a72793b2f28).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 18:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3646342693db92ccb97e120635ea7d068d60e738).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (69eeb7456e3ae4dbacb7ea34191d938acb9275e7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 22:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6e1b417164a9b2dba4c7f38925e8b4ba4c22e7f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 23:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6e1b417164a9b2dba4c7f38925e8b4ba4c22e7f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2024 at 23:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6e1b417164a9b2dba4c7f38925e8b4ba4c22e7f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 26 2024 at 00:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dbb613fb80683eeae413deddb3ad5189b7c3ba81)

github mathlib4 bot (Nov 26 2024 at 06:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b58a55482b9cbe092750d326c261e04667ef0c04).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 26 2024 at 08:37):

We will need to merge the following branches into nightly-testing:

  • origin/lean-pr-testing-6189

github mathlib4 bot (Nov 26 2024 at 09:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a2a544ab0cc7d3e1d2a07cda2e9dedef8dbe0749).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 26 2024 at 10:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (83238e24b9113e84b6e4a66801a7dc8c4e9c8320).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 26 2024 at 10:15):

Just merged lean-pr-testing-6189, per instructions.

Kim Morrison (Nov 26 2024 at 10:17):

I guess we need a script to assist merging these branches. I think the steps are:

  1. git fetch
  2. git merge origin/lean-pr-testing-NNNN
  3. Resolve conflicts in lean-toolchain, lakefile.lean, and lake-manifest.json in favour of current version.
  4. Replace all strings lean-pr-testing-NNNN in lakefile.lean with nightly-testing.
  5. Run lake update
  6. If there are no further conflicts, git commit -am "merge lean-pr-testing-NNNN" and exit code 0.
  7. Otherwise show the output of git status and exit code 1.

Does that sound right?

Kim Morrison (Nov 26 2024 at 10:18):

Also -- it would be great if the script that posts these messages could linkify them a bit. Both a link to the original Lean PR (for context) and a link to the diff in the branch would be very helpful.

github mathlib4 bot (Nov 26 2024 at 11:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a10eba97bbf9fccde39aaa51c640a0716513b627)

github mathlib4 bot (Nov 26 2024 at 13:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5ad34c033417c6e6efd3fcd9062fa1764d240209).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 26 2024 at 15:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e6b14d47d78f3846fbf3c5d50bb1eccd71abc6e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 26 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (19094c4d59858e7ff3ef353faebf2e5bd009dacb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 26 2024 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b25c29685772c4e73f377e6746ed44c2d3d29907).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 26 2024 at 22:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (21af8545cb9daf04f22cddc30a99fd7dbbf3543b).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 27 2024 at 00:16):

@Heather Macbeth, just a heads up that I just increased 1100 to 1200 on nightly-testing in:

/- When `linear_combination` is used to prove inequalities, its speed is very sensitive to how much
typeclass inference is demanded by the lemmas it orchestrates.  This example took 2146 heartbeats
(and 73 ms on a good laptop) on an implementation with "minimal" typeclasses everywhere, e.g. lots of
`CovariantClass`/`ContravariantClass`, and takes 206 heartbeats (10 ms on a good laptop) on the
implementation at the time of joining Mathlib (November 2024). -/
set_option maxHeartbeats 1200 in
example {a b : } (h : a < b) : 0 < b - a := by
  linear_combination (norm := skip) h
  exact test_sorry

Kim Morrison (Nov 27 2024 at 00:16):

Do you want to investigate? :-)

github mathlib4 bot (Nov 27 2024 at 00:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a10eba97bbf9fccde39aaa51c640a0716513b627)

Heather Macbeth (Nov 27 2024 at 01:33):

@Kim Morrison That test has been pretty weird -- as you can see the actual heartbeat count was 206 heartbeats, but it wouldn't pass CI without upping the limit to 1000 heartbeats (and apparently subsequently to 1200). If you have the branch checked out, could you run count_heartbeats to see whether the actual heartbeat count has increased?

github mathlib4 bot (Nov 27 2024 at 03:53):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a10eba97bbf9fccde39aaa51c640a0716513b627)

github mathlib4 bot (Nov 27 2024 at 08:36):

We will need to merge the following branches into nightly-testing:

  • origin/lean-pr-testing-6112
  • origin/lean-pr-testing-6200
  • origin/lean-pr-testing-6220

github mathlib4 bot (Nov 27 2024 at 08:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8a7a0b7d493c44f352e65718307fce1c052d20e2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 27 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7e86316a6a2b02c4957950b7ee550b17506485f5).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Nov 27 2024 at 10:08):

I'm working on a script as outlined by Kim Morrison

Johan Commelin (Nov 27 2024 at 10:08):

Will test it on the PRs above.

Kim Morrison (Nov 27 2024 at 10:21):

One subtlety here is that often we need to merge some subset of these on batteries as well...

Johan Commelin (Nov 27 2024 at 10:23):

  • 6200 merged with script

Johan Commelin (Nov 27 2024 at 10:23):

  • 6220 merged with script

Johan Commelin (Nov 27 2024 at 10:23):

6112 has nontrivial conflicts.

Kim Morrison (Nov 27 2024 at 10:23):

That actually sounds right!

Kim Morrison (Nov 27 2024 at 10:24):

I did some preliminary work on lean#6112, but then ended up doing most of it via a PR to master, so I'm not surprised there are conflicts.

Johan Commelin (Nov 27 2024 at 10:25):

#19531 for the script

Johan Commelin (Nov 27 2024 at 10:25):

I'll now work on linkifying the report

github mathlib4 bot (Nov 27 2024 at 10:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3942daa810bd06acd4daefa3fc3771378c5b2acb).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Nov 27 2024 at 10:35):

#19532 should hopefully create a linkified report.

Kim Morrison (Nov 27 2024 at 11:05):

I manually merged lean-pr-testing-6112

github mathlib4 bot (Nov 27 2024 at 11:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (01b31e1d1d58001128368257a32bd3337a5b576e).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 27 2024 at 21:13):

Kim Morrison said:

Just a heads up Mac Malone that nightly-testing at b0a9ae37ac9cfaf7f106c8c88253e09beab56c34 gets stuck at

% lake build
 [?/?] Computing build jobs

As usual, this is probably because I've deleted a file in Batteries; although this time Mathlib itself doesn't import the deleted file. I'll go look through the intermediate repos to see if they use it.

This is happening again. I've filed an issue at lean#6240.

Kim Morrison (Nov 27 2024 at 21:14):

This time at 3ad5449927085b63f4304a13d534105004783bdd.

Kim Morrison (Nov 27 2024 at 21:18):

I can't find any recently deleted files in Batteries via git log --diff-filter=D --summary | grep delete.

Kim Morrison (Nov 27 2024 at 21:19):

Ah, the Batteries dependency on the Mathlib nightly-testing branch was accidentally set to lean-pr-testing-6112. Correcting this means lake no longer hangs. Still, it shouldn't hang. :-)

github mathlib4 bot (Nov 27 2024 at 22:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (53a5bce08b5099841ffdd06a32c37340fcd2e47a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 27 2024 at 23:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (53a5bce08b5099841ffdd06a32c37340fcd2e47a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 28 2024 at 01:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (606995ead3bc421c5ebd78e4112a588f188fada3)

github mathlib4 bot (Nov 28 2024 at 09:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8d6349409589ff07b4d82f5b59384ba4cf177092).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 28 2024 at 10:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8d6349409589ff07b4d82f5b59384ba4cf177092).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 28 2024 at 11:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1ef016d640f5e5ff5f6b566e8f886073db310e80)

Ruben Van de Velde (Nov 28 2024 at 13:19):

Heather Macbeth said:

Kim Morrison That test has been pretty weird -- as you can see the actual heartbeat count was 206 heartbeats, but it wouldn't pass CI without upping the limit to 1000 heartbeats (and apparently subsequently to 1200). If you have the branch checked out, could you run count_heartbeats to see whether the actual heartbeat count has increased?

Same in #19342; count_heartbeats says 215 but needs 1200

github mathlib4 bot (Nov 28 2024 at 16:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1ef016d640f5e5ff5f6b566e8f886073db310e80)

github mathlib4 bot (Nov 28 2024 at 19:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a315e3e56aeeb979335b4f3507ad1e8db2f60edf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 28 2024 at 21:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (698148763dd29cf98dd2c56b8a44ac8e825461ae).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 28 2024 at 23:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (698148763dd29cf98dd2c56b8a44ac8e825461ae).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 29 2024 at 00:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1ef016d640f5e5ff5f6b566e8f886073db310e80)

github mathlib4 bot (Nov 29 2024 at 07:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab780650a6c8db2942d137b91ede7c94c47a4950).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 29 2024 at 10:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8f06fcac7450cf3e5fc78bcbcb53acfd74121828).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 29 2024 at 11:07):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1ef016d640f5e5ff5f6b566e8f886073db310e80)

github mathlib4 bot (Nov 29 2024 at 16:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cf80f345a26ac93fc5f71ff245ae7089fcc97adc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 29 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cf80f345a26ac93fc5f71ff245ae7089fcc97adc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 29 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f9e900aae7c006d8e9a0f23f222ceb91e522f942).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2024 at 00:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (21608d1f823014e49969e44316d30c5ea6de2335).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 30 2024 at 02:29):

Oof, thoroughly broken in ways. :-)

Kim Morrison (Nov 30 2024 at 02:30):

I think there are lean-pr-testing-6205 and/or lean-pr-testing-6190 branches, but for Batteries, not Mathlib.

github mathlib4 bot (Nov 30 2024 at 03:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eb9d9b39a42ac6b69b6f2c56de429cb31ac80e69).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2024 at 03:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eb9d9b39a42ac6b69b6f2c56de429cb31ac80e69).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2024 at 04:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eb9d9b39a42ac6b69b6f2c56de429cb31ac80e69).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2024 at 04:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eb9d9b39a42ac6b69b6f2c56de429cb31ac80e69).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2024 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c73ab4cda826a2c4a78a21bf064c41c4f74b91fb).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 30 2024 at 09:45):

Almost there.

github mathlib4 bot (Nov 30 2024 at 10:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1d86c526627b20fe1a580aae4341ff166747b8ea)

github mathlib4 bot (Nov 30 2024 at 11:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ba7312b5aafeb13465bb9283536208f2158e6150).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2024 at 13:29):

We will need to merge the following branches into nightly-testing:

Kim Morrison (Nov 30 2024 at 13:40):

Nice! False alarm on to-additive-4595, I guess.

github mathlib4 bot (Nov 30 2024 at 14:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ba7312b5aafeb13465bb9283536208f2158e6150).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2024 at 18:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (883af569cadb60cf1e7b203baa14dc4a5c964622).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2024 at 21:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4fafb9f5b76af48f96d2366beee76af2113161f7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 01 2024 at 01:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (222e64d6bc042156d6e39860ad9f0c79552de8e0)

github mathlib4 bot (Dec 01 2024 at 08:46):

We will need to merge the following branches into nightly-testing:

github mathlib4 bot (Dec 01 2024 at 08:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b8b8a288609c214ad2aac7d3837bedce7e2b4875).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 01 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b8b8a288609c214ad2aac7d3837bedce7e2b4875).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 01 2024 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a3fcd535e9295e67a5a9d10eef9ed013a5d90f12).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 01 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (65cc54340c823eff8861b7d448c2755bbc87bae8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 01 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2aefce62d6d933585e9c688b080ebeadc5c8e7ee).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 01 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6926cee95dfac950113a35dda8c99defd6fb5442).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 01 2024 at 23:52):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5f67609288d56f40ab174ea90db3dda888223a81)

github mathlib4 bot (Dec 02 2024 at 09:10):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (15569f37660f60880bab6ff414dba791ae78fbb4)

github mathlib4 bot (Dec 03 2024 at 08:41):

We will need to merge the following branches into nightly-testing:

github mathlib4 bot (Dec 03 2024 at 08:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5358a537cab9e63ab57d9ec41b64e112e275315d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 03 2024 at 08:59):

Ah... I restarted the nightly-testing branch, but this was a terrible idea, because now it shows diffs against all the old lean-pr-testing-NNNN branches.

Kim Morrison (Dec 03 2024 at 08:59):

In particular, I doubt there are actually changes in any of the three above.

github mathlib4 bot (Dec 03 2024 at 10:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1443a7f471cfdde855509db68de15981c2d73096).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 03 2024 at 11:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1ec33a404152f54bbabe1162c3dfa356a6f8b0ab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 03 2024 at 11:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ba241aff369d124b50f9fefc5ba46ddf3b02c437)

Kim Morrison (Dec 03 2024 at 11:53):

But no automatic reminder to create an adaptation PR, because I'd forgotten to create bump/v4.16.0.

Kim Morrison (Dec 03 2024 at 11:54):

Just did that.

github mathlib4 bot (Dec 03 2024 at 12:07):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ba241aff369d124b50f9fefc5ba46ddf3b02c437)

github mathlib4 bot (Dec 03 2024 at 13:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1ec33a404152f54bbabe1162c3dfa356a6f8b0ab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 03 2024 at 15:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a8931809d8cef5ce0c893acc2f907ecef61e8ac8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 03 2024 at 18:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (14e2a6b76e28622f84380169ed4f37b13d596a1c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 03 2024 at 21:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (da9df8db61024281c6beb7853df1ccec445ba61b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 03 2024 at 22:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (da9df8db61024281c6beb7853df1ccec445ba61b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 04 2024 at 00:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ba241aff369d124b50f9fefc5ba46ddf3b02c437)

github mathlib4 bot (Dec 04 2024 at 08:37):

We will need to merge the following branches into nightly-testing:

github mathlib4 bot (Dec 04 2024 at 09:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ea515836ea82a84277b33b28c840a24da4318c4f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 04 2024 at 09:42):

github mathlib4 bot said:

We will need to merge the following branches into nightly-testing:

Okay, I've repaired the nightly-testing branch. All these diffs now become trivial, so hopefully these false positive reports will go away.

Kim Morrison (Dec 04 2024 at 09:44):

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ea515836ea82a84277b33b28c840a24da4318c4f).
You can git fetch; git checkout nightly-testing and push a fix.

Hmm, can't reproduce locally, let's see if it repeats.

github mathlib4 bot (Dec 04 2024 at 10:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (da0cfc4d741436ce977bb835884026094ff2a16f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 04 2024 at 11:26):

Both the haveLetLinter and the hashCommandLinter now fail after https://github.com/leanprover/lean4/pull/6299, unless we set_option Elab.async false.

Kim Morrison (Dec 04 2024 at 11:26):

For now I've just set Elab.async false in the two test files, but obviously this is not a solution.

Kim Morrison (Dec 04 2024 at 11:26):

@Damiano Testa, I know you're very busy right now, but just pinging you for sometime later. :-)

Kim Morrison (Dec 04 2024 at 11:27):

@Sebastian Ullrich, in case you already understand what is going on and can suggest a quick fix!

Sebastian Ullrich (Dec 04 2024 at 12:06):

Thanks, that should definitely be on my side. I'll take look.

Sebastian Ullrich (Dec 04 2024 at 13:01):

lean#6299 actually simply uncovered an issue that already existed outside of #guard_msgs. @Damiano Testa This part of the linter now breaks:

However, in order to avoid local clutter, when warningAsError is false, the linter
logs a warning only for the #-commands that do not already emit a message.

The problem is that linters do not have access to the prior message log anymore. I don't think I understand the quote: what # commands don't emit a message, what are we linting against here?

Sebastian Ullrich (Dec 04 2024 at 13:02):

Similarly for the haveLetLinter, why does it care about "noisy" declarations?

Ruben Van de Velde (Dec 04 2024 at 13:12):

I don't have the context here, but I think there's two relevant rules for mathlib:

  • We don't want to have code on master that triggers warnings
  • We don't want to have code on master that triggers output (e.g. #check or #synth)

I don't know how these linters are related to that

Damiano Testa (Dec 04 2024 at 13:22):

Here is some more context: I think that #guard true is a "silent" #-command and the linter should flag it.

Damiano Testa (Dec 04 2024 at 13:22):

However, if a command already emits a warning, it is not going to make it past CI anyway, so the linter is just noise.

Damiano Testa (Dec 04 2024 at 13:23):

This is why the linter only makes noisy the hash-commands that would not themselves already trigger a CI error.

Sebastian Ullrich (Dec 04 2024 at 13:23):

But a #check 0 is not linted?

Damiano Testa (Dec 04 2024 at 13:24):

Correct: #check 0 would fail the noisy check on CI.

Sebastian Ullrich (Dec 04 2024 at 13:24):

Okay, it is not about warnings specifically

Damiano Testa (Dec 04 2024 at 13:24):

No, it is about any output at all.

Damiano Testa (Dec 04 2024 at 13:26):

Basically, the linter only tries to say something when it does not detect some noise already.

Sebastian Ullrich (Dec 04 2024 at 13:26):

Well. I suppose I can extend the MessageLog structure to cover these use cases. We should carry the reported messages around instead of a mere hadErrors flag.

github mathlib4 bot (Dec 04 2024 at 13:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a38db992d088e602ba99cdf94f77435bf23e9b8e).
You can git fetch; git checkout nightly-testing and push a fix.

Damiano Testa (Dec 04 2024 at 13:32):

That would work, but if it is a maintenance burden, maybe there are different approaches for the linter.

Sebastian Ullrich (Dec 04 2024 at 13:33):

It is a neutral change in the code but might save us from other trouble as well, who knows

Damiano Testa (Dec 04 2024 at 13:33):

On the other hand, having access to the messages themselves, would allow (other) linters to react to those.

Damiano Testa (Dec 04 2024 at 13:35):

I have experimented a bit with linters to find "unused" code, such as unnecessary set_options or nolints and I think that for some of these (not developed) linters, the message log could be useful.

Sebastian Ullrich (Dec 04 2024 at 15:12):

lean#6307 introduces MessageLog.reportedPlusUnreported that should be usable to fix both linters

Sebastian Ullrich (Dec 04 2024 at 15:14):

What is the correct way to test that given that nightly-with-mathlib does not contain lean#6299 yet?

Johan Commelin (Dec 04 2024 at 15:16):

Does lean#6307 build on top of lean#6299? I guess then we should use the lean-pr-testing-6307 branch

Sebastian Ullrich (Dec 04 2024 at 15:18):

I assumed that branch wouldn't be created if my lean4 branch is not based on nightly-with-mathlib

Johan Commelin (Dec 04 2024 at 15:19):

Hmmm, I think that's right.

Sebastian Ullrich (Dec 04 2024 at 15:20):

Might be easier to merge 6307 and then fix on nightly-testing, I don't foresee any need for further revisions

Johan Commelin (Dec 04 2024 at 15:20):

Ok, alternative would be to rebase on nightly-with-mathlib

Sebastian Ullrich (Dec 04 2024 at 15:20):

Wait, then we'd have to wait for the next nightly

Sebastian Ullrich (Dec 04 2024 at 15:36):

Johan Commelin said:

Ok, alternative would be to rebase on nightly-with-mathlib

A bit annoying since I have to include the right commits in the rebase but I've done so now

github mathlib4 bot (Dec 04 2024 at 16:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a38db992d088e602ba99cdf94f77435bf23e9b8e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 04 2024 at 18:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0e2973b0fb7d17e76965ed500540c189787b571c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 04 2024 at 22:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9bec372f2c4bd188669f930fa1b74bd13a52131b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 04 2024 at 23:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4745c02319412eeffd9dedd0284b48f8e30eeee1)

Kim Morrison (Dec 05 2024 at 00:32):

@Johan Commelin, we're no longer getting "bump branch reminders". Last time, the problem as that bump/v4.15.0 didn't exist. But this month I've remembered, and bump/v4.16.0 is there.

github mathlib4 bot (Dec 05 2024 at 00:57):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4745c02319412eeffd9dedd0284b48f8e30eeee1)

Johan Commelin (Dec 05 2024 at 05:51):

In this part of the workflow:

    - name: Fetch lean-toolchain from latest bump branch
      id: bump_version
      uses: actions/github-script@v7
      with:
        script: |
          const response = await github.rest.repos.getContent({
            owner: context.repo.owner,
            repo: context.repo.repo,
            path: 'lean-toolchain',
            ref: ${{ steps.latest_bump_branch.outputs.result }}
          });
          const content = Buffer.from(response.data.content, 'base64').toString();
          const version = content.match(/leanprover\/lean4:nightly-(\d{4}-\d{2}-\d{2})/)[1];
          return version;

we are getting errors: https://github.com/leanprover-community/mathlib4/actions/runs/12173176628/job/33953099942#step:12:27

     github-token: ***
    debug: false
    user-agent: actions/github-script
    result-encoding: json
    retries: 0
    retry-exempt-status-codes: 400,401,403,404,422
  env:
    NIGHTLY: 2024-12-04
    SHA: 4745c02319412eeffd9dedd0284b48f8e30eeee1
TypeError: Cannot read properties of null (reading '1')
    at eval (eval at callAsyncFunction (/home/runner/work/_actions/actions/github-script/v7/dist/index.js:35424:16), <anonymous>:10:79)
    at process.processTicksAndRejections (node:internal/process/task_queues:95:5)
    at async main (/home/runner/work/_actions/actions/github-script/v7/dist/index.js:35522:20)

Bryan Gin-ge Chen (Dec 05 2024 at 05:53):

The error is saying that
content.match(/leanprover\/lean4:nightly-(\d{4}-\d{2}-\d{2})/) is returning no matches.

Johan Commelin (Dec 05 2024 at 05:58):

git checkout bump/v4.16.0; cat lean-toolchain
Switched to branch 'bump/v4.16.0'
Your branch is up to date with 'origin/bump/v4.16.0'.
leanprover/lean4:v4.15.0-rc1

Johan Commelin (Dec 05 2024 at 05:58):

Makes sense...

Johan Commelin (Dec 05 2024 at 05:59):

It is the start of the month, so lean-toolchain is on an rc, instead of a nightly.

Johan Commelin (Dec 05 2024 at 06:01):

Need to have breakfast now. But if we bump the toolchain to a nightly, it should start working again.

Johan Commelin (Dec 05 2024 at 06:01):

And I can try to make the script robust against this scenario.

github mathlib4 bot (Dec 05 2024 at 07:11):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4745c02319412eeffd9dedd0284b48f8e30eeee1)

github mathlib4 bot (Dec 05 2024 at 08:37):

We will need to merge the following branches into nightly-testing:

github mathlib4 bot (Dec 05 2024 at 08:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (06422de9546612e92bafe15d4aa557b4b6a220d1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 05 2024 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (39eac4b7b275d558516e3b2c182a003b01698e02).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 05 2024 at 10:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (498c8c34f7c7a2a41dd1ef4cc8295103caa07ca5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 05 2024 at 12:16):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b01be4bda23a785e988643a07f24c7e478b23c83)

Johan Commelin (Dec 05 2024 at 16:41):

github mathlib4 bot said:

We will need to merge the following branches into nightly-testing:

Did you intend to have the nightly-testing branch of mathlib depend on the lean-pr-testing-6315 branch of batteries?

github mathlib4 bot (Dec 05 2024 at 17:25):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b01be4bda23a785e988643a07f24c7e478b23c83)

Kim Morrison (Dec 05 2024 at 22:47):

No, that was a mistake, which presumably would have been avoided if I'd used your new script. :-)

github mathlib4 bot (Dec 06 2024 at 00:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b01be4bda23a785e988643a07f24c7e478b23c83)

github mathlib4 bot (Dec 06 2024 at 09:25):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c6f4e015f5c536740ae52ea5926112e95d330f5a)

github mathlib4 bot (Dec 07 2024 at 08:18):

We will need to merge the following branches into nightly-testing:

github mathlib4 bot (Dec 07 2024 at 08:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (653f17d0c439d2d9d55797995521660adc6df994).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 07 2024 at 10:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (37305b9e5eff20c7b426a9905ccd04b387203bf1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 07 2024 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (21d992dd68e83a90bc1b22b677f90246efaf214a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 07 2024 at 16:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a988e8b369e20ae90b4998923e4efcd732a1da62).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 08 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9a3b5ca02eeb6b8821b1adeed6d540da55cbf469).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 08 2024 at 03:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (19b191ae82eabc6ade3c07cc325998bd8bee478a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 08 2024 at 08:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (31530f31d529f37cde81d086fe10b68e9eb1ee2f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 08 2024 at 10:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (31530f31d529f37cde81d086fe10b68e9eb1ee2f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 08 2024 at 15:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (294458c5add8df2c106f392d97e53aec900e95f5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 08 2024 at 18:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (65c00859d05eb8ff717bb0f06ff355609be271b2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 08 2024 at 22:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (20b2fd4c7be9ad9e2acf3c4347aa02aac4209a68)

github mathlib4 bot (Dec 09 2024 at 09:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d9df436d7f9d6e2eb0aad05d429d2fc53d4e301d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 09 2024 at 10:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ded531d92e509cb63d09ed490f49dbe45dde217e)

github mathlib4 bot (Dec 10 2024 at 08:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5d2254fa2ab034e34b4ae1363d48ea7acf430a6b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 10 2024 at 09:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5d2254fa2ab034e34b4ae1363d48ea7acf430a6b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 10 2024 at 10:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5d2254fa2ab034e34b4ae1363d48ea7acf430a6b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 10 2024 at 11:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f0f251d299ff907bada73f4dbfba2dfd0d619b69)

github mathlib4 bot (Dec 10 2024 at 13:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bfdd6039bf11a194e78a351b27e21774684a016e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 10 2024 at 16:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (14375b940a8d2372f6eff562acf72b9a75393810).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 10 2024 at 19:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (16956ef06e49e3e4f34d7be6d97f170580b42a79).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 10 2024 at 23:10):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f0f251d299ff907bada73f4dbfba2dfd0d619b69)

github mathlib4 bot (Dec 11 2024 at 08:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5f72b2e28cefb818887e4a7b7de72b6062fa1fc1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 11 2024 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d840f50ab07fb0170966e100a11aef6123eaf306).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 11 2024 at 10:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d1a65ef8cb89d1abb40397f03aa58f55f7438556)

github mathlib4 bot (Dec 12 2024 at 08:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (67e672d5aba8e1e7cd4528bcc344c1af623ef4dd).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 12 2024 at 08:52):

Required a minor fix for lean#5757.

github mathlib4 bot (Dec 12 2024 at 10:19):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d337aa990393a12a169ce0198e119251442d574e)

github mathlib4 bot (Dec 13 2024 at 08:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (383b0748ba499f742d97bf6ff772502b1e458986).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2024 at 09:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e42ca30b426589436293e6f614df7349f9c3b043).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2f5c9675058cba44a8773c8e559b7d126b107570).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2024 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (98dbd12b96d0c47ff7292af3340fabc0d27dd125).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2024 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b0a22ed4c5641d49feb0bd02f469d2f0e0cc5daf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2024 at 22:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (24a956e927a627c16a104adc19ceca8b33569ea7)

github mathlib4 bot (Dec 14 2024 at 08:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0662d0b6717c1777680219f9308baa68dd10abd8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2024 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0662d0b6717c1777680219f9308baa68dd10abd8).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 14 2024 at 11:09):

Should be working now. Just a few final adaptations for lean#6123.

github mathlib4 bot (Dec 14 2024 at 11:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d19d8405b0688fc5ac60e53056a822f6e53a34ec).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2024 at 12:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b09464fc7b0ff4bcfd4de7ff54289799009b5913).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2024 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (79d29f84f37ec475db18dc902ccfdffab51ff0c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2024 at 18:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1ed7634f46ba697f891ebfb3577230329d4b7196).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2024 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (37a149f02b44682bb186c430d0a896dce3c1f17f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 15 2024 at 00:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a395cd00a4fbe946ca76ff1fd1d1c78129a135ff).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 15 2024 at 04:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (af60d5dfe21be6d33cc1592aec1b4a598efdd023).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 15 2024 at 05:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (af60d5dfe21be6d33cc1592aec1b4a598efdd023).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 15 2024 at 07:18):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ddcb85bddebd7fa5b7316dab25b7eae6e0ff1fbb)

github mathlib4 bot (Dec 15 2024 at 10:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (13dbab738d85e172eaed1ba05012dd6b48c72039)

github mathlib4 bot (Dec 16 2024 at 08:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3f813de52d8cffaa73e27edd62364eec90eac633).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 16 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ed2f6ae5860b941bc054f11d5e402a480667d9e0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 16 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (95e4d18407c257812c48cf37309b701918c5bf1d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 16 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2927e227ec9454096c0507b4ac8386b3f4f09e5e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 16 2024 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0f3e538b0b562f4ecf8baeebd1337c4c1ed138e7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2024 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (458cc7d8784d3b2c54e3e142ae76e5aca576bc94).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2024 at 03:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b18fc8a82981a8fbf1c48387e28cd63422e3fccb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2024 at 08:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b18fc8a82981a8fbf1c48387e28cd63422e3fccb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2024 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b18fc8a82981a8fbf1c48387e28cd63422e3fccb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2024 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d5bed454ee2c347b2d60a12fc609ed827c070617).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bb0575e329e059f7ec31c43337a2094282f6be3c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2024 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9890d5ff187e6a1625705cce1f16623a755a22db).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9282f9eb8423e3ef68a61e0a13d1129179d11821).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (495ec69bfbbe8fe20099db76e889e39b676ba43f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2024 at 03:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d8e48a35237bfc90f26ca475fc198fe520a2e8e2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2024 at 08:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2144977fb121989a45d3f6e4d74fd8ab2350db3e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2144977fb121989a45d3f6e4d74fd8ab2350db3e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2024 at 12:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b7666b8884e893f12010025b159a44acf6c293ab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cbe8d43a7e6c614db88fc2ad8f0520e50c1d3dae).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2024 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b0466d1f33bcd06da8603dfe618c721422b37ac6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (933ad5493803f4c495f252678466ede6e1e2ee79).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 19 2024 at 08:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (933ad5493803f4c495f252678466ede6e1e2ee79).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 19 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (054d75b44095e8390c2afd9744e30c3b2b6cbd42).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 19 2024 at 10:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dac878dc2fde17aa9d7678bab2aed47c227a9063).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 19 2024 at 10:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dac878dc2fde17aa9d7678bab2aed47c227a9063).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 19 2024 at 10:39):

@Mac Malone, despite releasing v0.0.49-pre1 of ProofWidgets, with your changes from https://github.com/leanprover-community/ProofWidgets4/pull/95, Mathlib CI on nightly-testing is failing with

 [427/5760] Building proofwidgets/widgetJsAll
trace: ././.lake/packages/proofwidgets/widget> npm clean-install
trace: stderr:
could not execute external process 'npm'
error: external command 'npm' exited with code 255
Some required builds logged failures:
- proofwidgets/widgetJsAll
error: build failed

Kim Morrison (Dec 19 2024 at 10:39):

(And this reproduces locally after I uninstall npm.)

Kim Morrison (Dec 19 2024 at 10:39):

If this something you'll be able to take a look at?

github mathlib4 bot (Dec 19 2024 at 12:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (32ba402fc2048299c9c0e153b72b4d4ea8aade19).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 19 2024 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7669cc54f7c5c7f632570bfc610874709fa9306d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 19 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (49ac6bf04dc187ffc0a056421c603fcefce6991a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 19 2024 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c9f97ab5091a2a3ac9eaba5745ee293ddfee8dde).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c91dd0e151d3f0b6755d35119cd7943a516addb8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 03:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0065e8d93b880f81391d0c21f3aa49a06f80ef87).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 06:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (af8d133b3172e865899d7c37a7df09c805f22130).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1f3a116fa040a90a1f9bfbd675a968ab171ee2f8).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 20 2024 at 10:59):

Local build is looking promising!

github mathlib4 bot (Dec 20 2024 at 11:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (78a1c375495f3164e10f544789cab6ca76fecb40).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 11:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5465191d90fbd463c69cf994a2648cb87be33b63).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 11:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5465191d90fbd463c69cf994a2648cb87be33b63).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 12:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5ba57828ba4b35ddea3f87fd09ce5a87ddef7142).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 15:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (81263905255dea7b1663a7749af7ee277c01f681).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (74c027f022e7dfcab00f7104dfcd29b2070d38f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2024 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (75faccb7c68b07af22d7a2bd5f44a3d6ce7d3d49).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 21 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5ba284dd1c79017ec5bfc667d7f193c73de3e595).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 21 2024 at 03:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (839e3f6ba9240d043d4ef510140f10d00cad36f5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 21 2024 at 04:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (839e3f6ba9240d043d4ef510140f10d00cad36f5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 21 2024 at 04:56):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8a4877456aa721f76724451be03284db54851891)

github mathlib4 bot (Dec 21 2024 at 08:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1c080cc45939aaef448022267a6965a19e53c7bf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 21 2024 at 09:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1468375308d1c9fb517d8a69cbac94218df8e723).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 21 2024 at 10:10):

Per discussions in the maintainer channel, I've commented out the entirety of Mathlib/Computability/TMToPartrec.lean and Mathlib/SetTheory/Ordinal/Notation.lean (these are both leaf files in Mathlib) on the nightly-testing branch for now.

@Mario Carneiro has offered to take a look at these and do the repair, thank you. (If this won't be possible before January 4, please let me know so we can make plans for what to do at the release of v4.15.0-rc1.)

Mario Carneiro (Dec 21 2024 at 10:11):

yep, should happen today or tomorrow

Mario Carneiro (Dec 21 2024 at 10:40):

@Kim Morrison I'm looking at the fallout and I don't really understand the new behavior of simp here.

def foo : Nat  Nat
  | 0 => 0
  | n+1 => n

example (n) : foo n = foo 0 := by
  rw [foo]
  -- ⊢ foo n = 0

example (n) : foo n = foo 0 := by
  simp only [foo]
-- ⊢ (match n with
--   | 0 => 0
--   | n.succ => n) =
--   0

Previously, definitions like foo would only be unfolded when applied to one of the match patterns, as in the rw version. But now simp only [foo] is unfolding all occurrences, which is taking us back to the situation where we had to create definitional lemmas and mark them @[simp]...

github mathlib4 bot (Dec 21 2024 at 10:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8df8f11ba8d462d3de44e7b2ee0b9ae1b3cefe61).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 21 2024 at 10:58):

I think this is by design, but I am double checking. Not sure if I'll have a response for you though before I go offline until the 3rd...

Mario Carneiro (Dec 21 2024 at 10:59):

looking back at things like List.map, I see that we still aren't marking the definition as @[simp], so maybe I hallucinated that we ever fixed this issue

Mario Carneiro (Dec 21 2024 at 11:01):

but for giant functions like this it's really painful to have to restate all the definitional lemmas manually, and especially since lean generates the lemmas itself I don't see any argument for this being a good design

Mario Carneiro (Dec 21 2024 at 11:02):

(not to say that the specific change in this PR wasn't a good idea for other reasons - it may simply be exposing this latent issue and/or making it obvious in more places)

github mathlib4 bot (Dec 21 2024 at 11:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8df8f11ba8d462d3de44e7b2ee0b9ae1b3cefe61).
You can git fetch; git checkout nightly-testing and push a fix.

Mario Carneiro (Dec 21 2024 at 11:11):

Oh, this also seems a bit bad: a definition by recursion on PosNum fails to reduce when applied to 1, because there are a handful of functions before it reduces to PosNum.one. I'm not really sure what the best solution here is

Mario Carneiro (Dec 21 2024 at 11:12):

How does this work for 1 : Nat? Or is lean just cheating here

Mario Carneiro (Dec 21 2024 at 11:26):

the issue in Ordinal/Notation.lean seems to be similar, 0 : ONote is not simplifying when used as an argument to a recursive function

Mario Carneiro (Dec 21 2024 at 11:33):

I had to mark

@[simp] theorem repr_one : repr 1 = (1 : ) := repr_ofNat 1

as simp but it's the n=1 case of a more general theorem about ofNat and I can't find a way to mark it such that simp will use it

Mario Carneiro (Dec 21 2024 at 11:42):

this is pretty bad... all functions are not working on 0, but it's the simp normal form

Mario Carneiro (Dec 21 2024 at 11:42):

I think I might have to just make the simp normal form be ONote.zero

github mathlib4 bot (Dec 21 2024 at 11:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8df8f11ba8d462d3de44e7b2ee0b9ae1b3cefe61).
You can git fetch; git checkout nightly-testing and push a fix.

Mario Carneiro (Dec 21 2024 at 12:09):

@Kim Morrison I've pushed fixes to lean-pr-testing-6397 branch. I will leave it to you to git revert the commenting PR and rebase this fix instead

github mathlib4 bot (Dec 21 2024 at 13:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (21a4ad338cabc3b995580c306dab8cc148159e09).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 21 2024 at 14:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (62fd5798b4a61e5cbeee6e32562dcb4cbd66e0b1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 21 2024 at 16:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (31ee34b844cdabf8b0d9a7adc42396b9974c8631).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 21 2024 at 19:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (765f372d01b18e5917ad3fa42cdd8f9d07d757ae).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 21 2024 at 20:31):

Mario Carneiro said:

Kim Morrison I've pushed fixes to lean-pr-testing-6397 branch. I will leave it to you to git revert the commenting PR and rebase this fix instead

Thank you! I've reverted and merged.

Kim Morrison (Dec 21 2024 at 20:34):

Mario Carneiro said:

Kim Morrison I'm looking at the fallout and I don't really understand the new behavior of simp here.

def foo : Nat  Nat
  | 0 => 0
  | n+1 => n

example (n) : foo n = foo 0 := by
  rw [foo]
  -- ⊢ foo n = 0

example (n) : foo n = foo 0 := by
  simp only [foo]
-- ⊢ (match n with
--   | 0 => 0
--   | n.succ => n) =
--   0

Previously, definitions like foo would only be unfolded when applied to one of the match patterns, as in the rw version. But now simp only [foo] is unfolding all occurrences, which is taking us back to the situation where we had to create definitional lemmas and mark them @[simp]...

This behaviour wasn't changed by lean#6397. We're planning further changes in this direction, however.

github mathlib4 bot (Dec 21 2024 at 20:45):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b774a65bf5d20fd92d63eb98d03be2b29dfd9f27)

github mathlib4 bot (Dec 22 2024 at 09:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (63618639886f3bea1260812a0e5b81aebdc8cc60)

github mathlib4 bot (Dec 23 2024 at 09:11):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ed546d89ba3b9fa2c93b3501b9f6aac3593c930d)

github mathlib4 bot (Dec 23 2024 at 13:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (df6f676c7ca09a603a90260ca0e8ada34c3bf155).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 23 2024 at 15:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cd2213b6efc7c0ce581044c1e187be9a5cb6caac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 23 2024 at 18:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7d83d27ad7bfeb08a2d858ef8028e9f9d12f77db).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 23 2024 at 20:06):

Just a heads up that I will not be touching nightly-testing until the 3rd. If anyone would like to fix it that would be amazing. :-)

github mathlib4 bot (Dec 24 2024 at 01:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0c3ebf2713efb1dd3d29fcdd5d3eabb1cd048b64).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 24 2024 at 03:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2f55464865131df719850a6eace00516f9f9a201).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 24 2024 at 06:04):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ed546d89ba3b9fa2c93b3501b9f6aac3593c930d)

github mathlib4 bot (Dec 24 2024 at 09:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9a6b101b298066238b15e3fbd66618c2088cc693)

github mathlib4 bot (Dec 25 2024 at 09:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8157db740f7cbf298fb4839f6b1b81b03f76d44e)

github mathlib4 bot (Dec 26 2024 at 09:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d97af69f33c3a73efddc6db118bf4ffdb0ff78cd)

github mathlib4 bot (Dec 27 2024 at 09:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9cbdb8573d4029e6ae53898ae6002b9f9b95328c)

github mathlib4 bot (Dec 27 2024 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1b71c694536f17c6bf6936100339f1cdad203588).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 03:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (054515ea2a5d7f68512934b27548725e733e8cbe).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 06:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e8a30842b99b9828a09461fffeaa56cd74287dac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 08:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e8a30842b99b9828a09461fffeaa56cd74287dac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 09:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e8a30842b99b9828a09461fffeaa56cd74287dac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 12:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (161c83c3e874142a5a1658146ac3d26e43a91dc6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 13:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (161c83c3e874142a5a1658146ac3d26e43a91dc6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 13:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (161c83c3e874142a5a1658146ac3d26e43a91dc6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 16:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0c419e32e8cc2b54b3ac18eafa3595cd17659e1e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 28 2024 at 16:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (84397c9ac1acff58fe69934a8d8ee44e2b9d85a0)

github mathlib4 bot (Dec 29 2024 at 01:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1a402974fd696ae8df2990028b9fac0752700d79).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 29 2024 at 06:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e423a1f0105a779265101af2bd177f5d8065c594).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 29 2024 at 09:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e423a1f0105a779265101af2bd177f5d8065c594).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 29 2024 at 10:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0da6485fb4629890947f49ed3ee5e3d5269ff32c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 29 2024 at 13:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (68fbd252aa5d0168c5f582c0f66b3005dba683e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 29 2024 at 14:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (007c83315419f9d66e0056ac22cd99fabbad8069)

github mathlib4 bot (Dec 30 2024 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b4e6697e701bb49bcf49c504b8335747f55171c8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 30 2024 at 01:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (007c83315419f9d66e0056ac22cd99fabbad8069)

github mathlib4 bot (Dec 30 2024 at 09:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (310c1aa3b3b315662b745a38d252e8668dbc15d5)

Johan Commelin (Dec 30 2024 at 15:31):

@Ruben Van de Velde Thanks so much for fixing these failures :tada: :octopus:

github mathlib4 bot (Dec 30 2024 at 15:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (310c1aa3b3b315662b745a38d252e8668dbc15d5)

github mathlib4 bot (Dec 31 2024 at 09:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c3cb62f4b4768c69484af8be1988e1d8ae00c3ce)

github mathlib4 bot (Jan 01 2025 at 08:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7178aee7a431bb7527da15c3507836d8dfefcda4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 01 2025 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7178aee7a431bb7527da15c3507836d8dfefcda4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 01 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bd681bc33a22201938feb3796dfad236496726dd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 01 2025 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9419c034110d02f83c8cf286f877c624e492e16f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 01 2025 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (504007f6f772de93ea967b17320baeac5a21cb55).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 01 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c781ca864408200f5f68bff153a83bd95b3775da).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 02 2025 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ec10d9ba44225d66e790787d0f5b19a14830337e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 02 2025 at 03:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5e5c6da9e047d879ce36de0761405785f64f61fb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 02 2025 at 08:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5e5c6da9e047d879ce36de0761405785f64f61fb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 02 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e814fc9cda4aed84c5302727cb7d2d0dd45c647e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 02 2025 at 11:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (38800e147b0bd6d9173e862c744609a4d8c18d1d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 02 2025 at 12:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d458ec9af73e637e20410d0496462c2426f887c3).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Jan 02 2025 at 12:20):

@Eric Wieser The problems have to do with RefinedDiscrTree. Could you please take a look?

Johan Commelin (Jan 02 2025 at 12:21):

Merging master doesn't fix the issues.

Johan Commelin (Jan 02 2025 at 12:21):

In particular, there seem to be two different RefinedDiscrTree types now. Is that right?

github mathlib4 bot (Jan 02 2025 at 12:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (041d59b4c1ad8df53c9ea0224b076f0f3c60ddc4).
You can git fetch; git checkout nightly-testing and push a fix.

Eric Wieser (Jan 02 2025 at 12:38):

No, there's still only one, but there was an intermediate commit where the filename and namespace didn't match

Eric Wieser (Jan 02 2025 at 12:40):

It looks like something has been merged badly into nightly-testing

Eric Wieser (Jan 02 2025 at 12:42):

Yeah, https://github.com/leanprover-community/mathlib4/blob/nightly-testing/Mathlib/Lean/Meta/RefinedDiscrTree.lean had its content moved to four new files, but somehow nightly-testing has the content both in the new files and in the original

Eric Wieser (Jan 02 2025 at 12:45):

The https://github.com/leanprover-community/mathlib4/commit/247f3aa825982e579b94881f13ac428472b6f85a merge commit is bad

Johan Commelin (Jan 02 2025 at 12:51):

Aha, how should it be fixed?

github mathlib4 bot (Jan 02 2025 at 12:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (041d59b4c1ad8df53c9ea0224b076f0f3c60ddc4).
You can git fetch; git checkout nightly-testing and push a fix.

Eric Wieser (Jan 02 2025 at 13:15):

Johan Commelin said:

Aha, how should it be fixed?

Paste the file at master on top of whatever nightly testing has, maybe?

Eric Wieser (Jan 02 2025 at 13:16):

I think it's better to make the adaptations over again from scratch than lose changes from master

Johan Commelin (Jan 02 2025 at 14:20):

Did that. Let's see if it worked.

github mathlib4 bot (Jan 02 2025 at 14:50):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c7c1e06e17bc790c799baec988d32a7abaa51875)

github mathlib4 bot (Jan 03 2025 at 09:25):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (15d915fa08f4c49f024aa59d1954fde50cca38c1)

github mathlib4 bot (Jan 04 2025 at 08:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a97b21ff86ea58a827f0d95be7ff3d799647b417).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 04 2025 at 09:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a97b21ff86ea58a827f0d95be7ff3d799647b417).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 04 2025 at 12:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c8e9d14233399d0c195b8dfd478fd96d4364fb10).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 04 2025 at 15:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6d2cbb58e68c7424d746005d5bbf75a31cb14cb6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 04 2025 at 18:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0061a577b405448e5bd709c059c2ac246fc0b1d3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 04 2025 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b43248be90578db4b4158698029b1200ab4df641).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 05 2025 at 00:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1e25efce54c09ee2321f801cb4b51126869ae8c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 05 2025 at 01:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (33876800b00716486c19466df8efee1440a3e777)

github mathlib4 bot (Jan 05 2025 at 09:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (bc1d910c4bf47623e9e4038ec005877c38183305)

github mathlib4 bot (Jan 06 2025 at 08:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9afdff78cbdf653902190167fd1429e4adc4ac89).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 06 2025 at 10:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (00495cea91b1d8614e4957572cb32d1679b4296f)

github mathlib4 bot (Jan 07 2025 at 09:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9f2fa6ce057e6b196523b83134f1db0b2adafada)

github mathlib4 bot (Jan 08 2025 at 10:21):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a5e74b31f33ac8d48faaad46d8b6da297aa46fcb)

github mathlib4 bot (Jan 09 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f227e4af164386c81166cdc4e8e263323b586a36).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 09 2025 at 10:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4755cdd41545a5cbb88c3a0c3092554467cd9886).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 09 2025 at 13:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab7742ecee7a124d8eb89d28cbd570252ff517b5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 09 2025 at 14:19):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1e7d93f1607609b889e37abf9cf87f9290b83b7c)

github mathlib4 bot (Jan 10 2025 at 01:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0a078d0b0c7fdf68a3e718818265e90116a05612).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jan 10 2025 at 01:25):

This is waiting on the update to import-graph needed after batteries#1091.

Kim Morrison (Jan 10 2025 at 01:26):

Ah, which is all ready to go at https://github.com/leanprover-community/import-graph/pull/49. I'll merge.

Kim Morrison (Jan 10 2025 at 01:28):

Merged, and bumped deps on nightly-testing, should come good now.

github mathlib4 bot (Jan 10 2025 at 01:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0a078d0b0c7fdf68a3e718818265e90116a05612).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 10 2025 at 02:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1e7d93f1607609b889e37abf9cf87f9290b83b7c)

github mathlib4 bot (Jan 10 2025 at 08:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (973fc78afb24119af738f370764bf7820a4e86a8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 10 2025 at 09:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (973fc78afb24119af738f370764bf7820a4e86a8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 10 2025 at 11:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (2a00a07c117d5c40c4bc779c66091fd8fc653155)

github mathlib4 bot (Jan 11 2025 at 04:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e0a7afcfbf892b9c888ae3c680036a140eee6479).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 11 2025 at 05:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (2a00a07c117d5c40c4bc779c66091fd8fc653155)

github mathlib4 bot (Jan 14 2025 at 06:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c083085d05d098ff6bae992740c6d7eadf1c4cf1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jan 14 2025 at 06:53):

We've been having trouble releasing nightlies due to a Windows linker issue. My understanding is that this will be fixed once lean#6622 is merged, but until then Mathlib's nightly-testing will remain broken.

github mathlib4 bot (Jan 14 2025 at 10:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a7b5e89018c3880ed1610530327aeb1ff9ac7b2c).
You can git fetch; git checkout nightly-testing and push a fix.

Henrik Böving (Jan 14 2025 at 10:14):

That's an actual failure now :tada:

github mathlib4 bot (Jan 14 2025 at 11:14):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ba207fbdbaa72544b58589ea3ae95a8ca6e5d595)

github mathlib4 bot (Jan 15 2025 at 08:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dc5b3f0c90e6e91580442a3ec4df5cf3ee638eb0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 15 2025 at 10:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d2f7b08b793953e9ce82db4d52979668fe94d71b).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jan 15 2025 at 10:17):

Hmm, that's a bit scary: part way through the build Lean just starts failing with incompatible header on every file.

lake exe cache build && lake build seems to be working locally, however.

 [4911/5895] Built Mathlib.Probability.ProbabilityMassFunction.Monad
 [4912/5895] Built Mathlib.RingTheory.Polynomial.SeparableDegree
 [4913/5895] Built Mathlib.LinearAlgebra.Eigenspace.Zero
 [4914/5895] Built Mathlib.RingTheory.AdjoinRoot
 [4915/5895] Building Mathlib.Analysis.NormedSpace.Multilinear.Curry
trace: .> LEAN_PATH=././.lake/packages/Cli/.lake/build/lib:././.lake/packages/batteries/.lake/build/lib:././.lake/packages/Qq/.lake/build/lib:././.lake/packages/aesop/.lake/build/lib:././.lake/packages/proofwidgets/.lake/build/lib:././.lake/packages/importGraph/.lake/build/lib:././.lake/packages/LeanSearchClient/.lake/build/lib:././.lake/packages/plausible/.lake/build/lib:././.lake/build/lib LD_LIBRARY_PATH= /home/lean/.elan/toolchains/leanprover--lean4---nightly-2025-01-15/bin/lean -Dpp.unicode.fun=true -DautoImplicit=false -Dweak.linter.docPrime=false -Dweak.linter.hashCommand=true -Dweak.linter.oldObtain=true -Dweak.linter.refine=true -Dweak.linter.style.cdot=true -Dweak.linter.style.dollarSyntax=true -Dweak.linter.style.header=true -Dweak.linter.style.lambdaSyntax=true -Dweak.linter.style.longLine=true -Dweak.linter.style.longFile=1500 -Dweak.linter.style.missingEnd=true -Dweak.linter.style.multiGoal=true -Dweak.linter.style.setOption=true ././././Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean -R ./././. -o ././.lake/build/lib/Mathlib/Analysis/NormedSpace/Multilinear/Curry.olean -i ././.lake/build/lib/Mathlib/Analysis/NormedSpace/Multilinear/Curry.ilean -c ././.lake/build/ir/Mathlib/Analysis/NormedSpace/Multilinear/Curry.c --json
error: ././././Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean:6:0: failed to read file '././.lake/packages/batteries/.lake/build/lib/Batteries/Data/NameSet.olean', incompatible header
error: Lean exited with code 1
 [4916/5895] Building Mathlib.RingTheory.DedekindDomain.Basic
trace: .> LEAN_PATH=././.lake/packages/Cli/.lake/build/lib:././.lake/packages/batteries/.lake/build/lib:././.lake/packages/Qq/.lake/build/lib:././.lake/packages/aesop/.lake/build/lib:././.lake/packages/proofwidgets/.lake/build/lib:././.lake/packages/importGraph/.lake/build/lib:././.lake/packages/LeanSearchClient/.lake/build/lib:././.lake/packages/plausible/.lake/build/lib:././.lake/build/lib LD_LIBRARY_PATH= /home/lean/.elan/toolchains/leanprover--lean4---nightly-2025-01-15/bin/lean -Dpp.unicode.fun=true -DautoImplicit=false -Dweak.linter.docPrime=false -Dweak.linter.hashCommand=true -Dweak.linter.oldObtain=true -Dweak.linter.refine=true -Dweak.linter.style.cdot=true -Dweak.linter.style.dollarSyntax=true -Dweak.linter.style.header=true -Dweak.linter.style.lambdaSyntax=true -Dweak.linter.style.longLine=true -Dweak.linter.style.longFile=1500 -Dweak.linter.style.missingEnd=true -Dweak.linter.style.multiGoal=true -Dweak.linter.style.setOption=true ././././Mathlib/RingTheory/DedekindDomain/Basic.lean -R ./././. -o ././.lake/build/lib/Mathlib/RingTheory/DedekindDomain/Basic.olean -i ././.lake/build/lib/Mathlib/RingTheory/DedekindDomain/Basic.ilean -c ././.lake/build/ir/Mathlib/RingTheory/DedekindDomain/Basic.c --json
error: ././././Mathlib/RingTheory/DedekindDomain/Basic.lean:6:0: failed to read file '././.lake/packages/batteries/.lake/build/lib/Batteries/Data/NameSet.olean', incompatible header
error: Lean exited with code 1

github mathlib4 bot (Jan 15 2025 at 10:43):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (db3b11e6f0e79ec5e416d03fd29c873739e748dc)

Ruben Van de Velde (Jan 15 2025 at 12:53):

Random bitflip in that one olean?

github mathlib4 bot (Jan 15 2025 at 16:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (db3b11e6f0e79ec5e416d03fd29c873739e748dc)

github mathlib4 bot (Jan 16 2025 at 08:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0ec82d5aaaa6562ad1758c7b6569bce8a7f5cf8b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 16 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0ec82d5aaaa6562ad1758c7b6569bce8a7f5cf8b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 16 2025 at 12:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (71e670b6034537743f154aacb706a8d568216c54).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 16 2025 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (94099b4e3e03fbb365bb797d566a2168442c7a34).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 16 2025 at 18:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0d3784625d21570a7f5e475ae27e34177107f6c3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 16 2025 at 22:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b57abe19e88c3b836e84c3b6d5690065376f7f3b)

github mathlib4 bot (Jan 16 2025 at 23:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e6c7f46380cd18cb17d8759249c26429e6893b09).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 17 2025 at 01:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e6c7f46380cd18cb17d8759249c26429e6893b09).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 17 2025 at 01:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b57abe19e88c3b836e84c3b6d5690065376f7f3b)

github mathlib4 bot (Jan 17 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (66e14198c9acbb7f21fd32c34d0bba8c2ff3c7b6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 17 2025 at 10:35):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f059ccdd26b54901d17ae8cc90c0ee58b88bedb0)

github mathlib4 bot (Jan 18 2025 at 10:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7de4ea33f32d8a5fe224e82e755a342fde3a0fa4)

github mathlib4 bot (Jan 19 2025 at 10:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a58a89a28f740bc7878e82806f3ddf2f67bfd65a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jan 19 2025 at 10:50):

Fixed.

Kim Morrison (Jan 19 2025 at 10:51):

Curiously, it was the #count_heartbeats test file, complaining that simple things like example (a : Nat) : a = a := rfl now take 8 heartbeats rather than 7.

Kim Morrison (Jan 19 2025 at 10:51):

It's only one heartbeat, but maybe it is a sign of something nasty?

Kim Morrison (Jan 19 2025 at 10:52):

I guess @Sebastian Ullrich landed some pretty fundamental changes today, so we shouldn't be too surprised.

github mathlib4 bot (Jan 19 2025 at 11:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5b336e4a3fbd4642747e804d86e4d31ba469119b)

github mathlib4 bot (Jan 20 2025 at 09:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0f52dbc81e1f931efb1b41f8ced91dae40d1d4f4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 20 2025 at 10:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c4510a08da413b6c60c3eb8d5304aa45426b3b64).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 20 2025 at 11:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e43c7732f3e074817dad5659dbc751a3a3bc9b1c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 20 2025 at 13:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6313738aeb18ad4aadb1d0c890a4baae06fd8180).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jan 20 2025 at 13:23):

Needs an update to ProofWidgets too..

github mathlib4 bot (Jan 20 2025 at 14:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a17fe140cca9b29dfa7ec9727deabd7bc114ba63)

github mathlib4 bot (Jan 21 2025 at 09:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1264ce95ed09c73b4aadc6ec45fc7db15897e79d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 21 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1264ce95ed09c73b4aadc6ec45fc7db15897e79d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 21 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1264ce95ed09c73b4aadc6ec45fc7db15897e79d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 21 2025 at 11:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1264ce95ed09c73b4aadc6ec45fc7db15897e79d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 21 2025 at 11:49):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dcf59332226749edf58a2cf191d2672c0083fa48)

github mathlib4 bot (Jan 22 2025 at 09:33):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9bfb7cd4e59c6c6d16d745f27e2370d1d8a4d638)

github mathlib4 bot (Jan 22 2025 at 12:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (97bce08481d96a1eacfba45ffe14f4e05709c36b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 22 2025 at 15:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (72bf52f21e463ed123c31426cecc3ba6a5878092).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 22 2025 at 18:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bd502a40fb334f8d7007d830793db6509680c886).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 22 2025 at 21:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3226828897ffb337c36a3f486aaf2b0e6c0e9e6c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 23 2025 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3dc2beffa4849b995f5bf41d58cf25a47ef9ed44).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 23 2025 at 05:43):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9bfb7cd4e59c6c6d16d745f27e2370d1d8a4d638)

github mathlib4 bot (Jan 23 2025 at 09:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (681a0a09c81894fb47870c2d9b318360716f0b04)

github mathlib4 bot (Jan 24 2025 at 09:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ffaf9758753e7e58dfb0b5d60d531a72d6fe6413).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 24 2025 at 10:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1cbfe61c57846329c6daec86f44706ce589f9477).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 24 2025 at 13:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e1f9f040625dc9473eade841874dfea86c33dd60).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 24 2025 at 13:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3e696a8a9edeb0fca0e1a9df552c7e91d2aca018)

github mathlib4 bot (Jan 25 2025 at 10:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (578b8b9c0de205ff68df2d66f6c20828122e4242)

github mathlib4 bot (Jan 26 2025 at 09:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b36f8b22a2bdf77d064996493768f6f780d5f4c2)

github mathlib4 bot (Jan 27 2025 at 09:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (413249c638b4c9453166d2b94c9a7f13f6238b14).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 27 2025 at 10:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5011e4754518f50f90c05ead57ff20f753d60c98)

github mathlib4 bot (Jan 28 2025 at 10:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (94b2ff5a02d742d2b90bc22e5a0da8f4bef2c68c)

Ruben Van de Velde (Jan 28 2025 at 16:25):

I extracted the changes that already work on master (which was most of them) into #21184, quick review appreciated

github mathlib4 bot (Jan 28 2025 at 18:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2fc44e9c4aa0b14de7885879e499fb00c1b8e093).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 28 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (edd636fc612442a540d77efd4fdbc9308de8c222).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Jan 28 2025 at 21:58):

I broke it, I fix it

github mathlib4 bot (Jan 28 2025 at 22:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (090d323e8ca9c45ee4cb6e4bcbd28dd58eeab426).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Jan 28 2025 at 22:34):

And so did Kim, apparently

Kim Morrison (Jan 28 2025 at 22:52):

Oops, sorry, are we at cross purposes here?

Ruben Van de Velde (Jan 28 2025 at 22:53):

I think we made exactly the same changes, so no worries

github mathlib4 bot (Jan 28 2025 at 23:04):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (94b2ff5a02d742d2b90bc22e5a0da8f4bef2c68c)

github mathlib4 bot (Jan 29 2025 at 11:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5ff0a4782ee8ac78210032b135f7037e8c895153).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 29 2025 at 13:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (23e223e4cbe6f55c49ca01f8a94496ba84981f9c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 29 2025 at 15:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3cbf001210ddcf4c05ca37bb6c33bd4769616089).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Jan 29 2025 at 16:11):

(simpnf warnings)

github mathlib4 bot (Jan 29 2025 at 18:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b7ce26aaad6985218edd7cc8caa517846e25be1f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 29 2025 at 22:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (323ed6b5ce297555377a927ac5d0f38b73b825e8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 29 2025 at 23:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b0e2db2f53338ae6bc3506cfc201840f090332c3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jan 29 2025 at 23:56):

Just needs a shake

github mathlib4 bot (Jan 30 2025 at 00:40):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7b2d9ab953bba5cceb441b1641eae8ee62fe03fd)

github mathlib4 bot (Jan 30 2025 at 04:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (16e417ea1db9867753f0618a2a4446ebe6f7583a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 30 2025 at 07:06):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7b2d9ab953bba5cceb441b1641eae8ee62fe03fd)

github mathlib4 bot (Jan 30 2025 at 08:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (132efc702f743d24550d2b85b029ea64ffafbcab).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jan 30 2025 at 09:32):

Because of some bad timing for the cut of the nightly, I had to "downstream" a bunch of lemmas into Batteries that will land in nightly-2025-01-31, and then can be removed again. If it wasn't the end of the month and on the verge of cutting a release, I would have waited a day instead.

github mathlib4 bot (Jan 30 2025 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (132efc702f743d24550d2b85b029ea64ffafbcab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 30 2025 at 10:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9571e4aeb3689e34e89f18bba35fda5ae7a1fcd5).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jan 30 2025 at 10:52):

Just a heads up that I have outright deleted MathlibTest/CountHeartbeats.lean. It's currently not fit for purpose, as it relies on checking exact heartbeat counts.

github mathlib4 bot (Jan 30 2025 at 11:05):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e36c2b838cb650a07a6b95ae8eb96dc39b7468b2)

github mathlib4 bot (Jan 31 2025 at 08:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (01a1707b7dff363729b99ba566d378bc77c0df9d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 31 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4e87722e4b41edb65206954e7debb2152c919fde).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jan 31 2025 at 11:59):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (432e7f81b666b3821733768a4e87bd2a77dda052)

github mathlib4 bot (Feb 01 2025 at 09:31):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ee185c77453acccd00a506f01cd01692a7e55a5c)

github mathlib4 bot (Feb 02 2025 at 11:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b9329078bf12b90531207e8efd16c6ad543ee0d5)

github mathlib4 bot (Feb 03 2025 at 08:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e6775eae2c7970308672a1674b9dcadb042047ab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 03 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (347a323db691f7dccd175ebc3d6fab8d0c8b1d82).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 03 2025 at 10:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a94c6d1c3e86987f507443d7464a2c802c2e39ac)

github mathlib4 bot (Feb 03 2025 at 16:31):

:warning: Warning: The lean-toolchain file in the latest bump branch does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.
Current content: leanprover/lean4:v4.17.0-rc1

This needs to be fixed for the nightly testing process to work correctly.

Yaël Dillies (Feb 03 2025 at 17:34):

Ooh, exciting new message

github mathlib4 bot (Feb 03 2025 at 19:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a94c6d1c3e86987f507443d7464a2c802c2e39ac)

github mathlib4 bot (Feb 03 2025 at 19:27):

:warning: Warning: The lean-toolchain file in the latest bump branch does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.
Current content: leanprover/lean4:v4.17.0-rc1

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Feb 03 2025 at 22:18):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a94c6d1c3e86987f507443d7464a2c802c2e39ac)

github mathlib4 bot (Feb 03 2025 at 22:18):

:warning: Warning: The lean-toolchain file in the latest bump branch does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.
Current content: leanprover/lean4:v4.17.0-rc1

This needs to be fixed for the nightly testing process to work correctly.

Kim Morrison (Feb 03 2025 at 23:34):

I've added a step to Lean's release_checklist.py to check for this problem. Johan will fix it tomorrow when he finishes the checklist.

Johan Commelin (Feb 04 2025 at 05:07):

Should be fixed now.

github mathlib4 bot (Feb 04 2025 at 07:03):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a94c6d1c3e86987f507443d7464a2c802c2e39ac)

github mathlib4 bot (Feb 04 2025 at 09:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2dd5bb2d33e82377b2cc4e347e2317a4ec0603bc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 04 2025 at 10:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (79ad6ef36345d2b2b3f7c340017c0738e69d6dd3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 04 2025 at 10:55):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9bdd95bdc7906447e1aea509cf21c8d39633183f)

github mathlib4 bot (Feb 05 2025 at 09:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0642034a4e45d5b21dbf5d4cdd8141ef7c0c686a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 05 2025 at 10:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (435383539c55f501dedaa2ae9462bcef3d5f8882).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 05 2025 at 12:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ad7930c3f767a589b1fc696529af28a97f714308).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 05 2025 at 16:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3eb0ff709449ce0401b0032e17d61dd0f5d51b46).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 05 2025 at 19:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (24c597596e1eab32ef9047e2ca944e099df3d294).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 05 2025 at 21:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a68f922664ee0046150089fb421964c89575c08f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 06 2025 at 00:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f6895b222238ccf2027d2885ff9900a801b0f853).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 06 2025 at 00:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f6895b222238ccf2027d2885ff9900a801b0f853).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 06 2025 at 01:33):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8a2d338ba77347504a3a5a57fe4401d9ddf05d01)

github mathlib4 bot (Feb 06 2025 at 10:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (fdd759714b98d9c371a832e842643255a385e9e9)

github mathlib4 bot (Feb 06 2025 at 22:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c7a2a04be15f08bc892687f61b11059b43c8cb3b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 07 2025 at 00:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c7a2a04be15f08bc892687f61b11059b43c8cb3b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 07 2025 at 02:47):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (fdd759714b98d9c371a832e842643255a385e9e9)

github mathlib4 bot (Feb 07 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bbbf03a57847e7b7d06615da69c4d712f68f854f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 07 2025 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bbbf03a57847e7b7d06615da69c4d712f68f854f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 07 2025 at 12:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3492e1786adc9f37c7a0bb0da1f6fe84f7d01cb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 07 2025 at 16:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (feff2b7a3b3f7e4351993a12e2d8aa400b7a88a4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 07 2025 at 18:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1d666be8e3702cea5a68f7c5927ecccbb4e58b91).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 07 2025 at 22:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a71c1cefd363a33ecb382055c5823e7a63cd72bf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 08 2025 at 01:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (53d1998f8b520572d0b7bbb5d795b83a68439f0d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 08 2025 at 04:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (440c3d5524efacb02f3897055bb04260cdb9019d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 08 2025 at 09:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (82c447bebd3786d983de04212b2714e7bb011f66).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 08 2025 at 10:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (82c447bebd3786d983de04212b2714e7bb011f66).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 08 2025 at 12:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5b94d7fda9269ed8a9ea84625c7934b8994b4d48).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 08 2025 at 19:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (caef0374c9c8787d807ec54773fc90ed871d5ffd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 08 2025 at 21:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1c6671052038c292997d391b8ab6272f75288120).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 01:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4ba7257a1a92242e9e8f2307f0b7d4bb70420ab5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 07:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0868356db19999db4ce0bea593f6fd3b4f19e07a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 09:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e05e225065104b31833e1dad5cb06b0862b2fa6d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 10:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e05e225065104b31833e1dad5cb06b0862b2fa6d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 13:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (50c9a9bd433367a722e0b109c04b3514e0eb2ea7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 16:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a04abe9b91cca2a2275a46fe5277a863d721e611).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 18:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c1d47161522b8d5e570c10245776cc33c69ae085).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 21:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3d193da9516cf6a8ae8dd7a0f7fe1b7747b9250b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 09 2025 at 22:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a443ebbe967fa2bc8dd707a948e31458d320d21a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 10 2025 at 01:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (58238a71a42926206ac79f587c43eccdaafc8a4a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 10 2025 at 03:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (418896cb01a8109b3298660b41fb8656e8a0234b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 10 2025 at 03:30):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (370e197c3682b1b952160e58965fbb734bc23c26)

github mathlib4 bot (Feb 10 2025 at 10:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e2649ed629bd663355c3cb6ac5535151fa7e47b3)

github mathlib4 bot (Feb 11 2025 at 09:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (751f9504e84e892212aa23308aa4091c20e98651).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 11 2025 at 09:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ff73b3ec03f79ed0d9dc228ee801ab47497156b4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 11 2025 at 11:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (619a1ebba2f05fe0d3c1147e9628ec361175bea6)

github mathlib4 bot (Feb 12 2025 at 13:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (58fa94d32c170d0de37ff67508fb9da530c98bba).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 12 2025 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e2ee0aa168e5568a22aaf90668359f87b4d60af9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 12 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1c5e1606e6c91adeae43d9d5897c8ef108e9dcc4).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Feb 12 2025 at 22:29):

This is a Batteries problem, but unfortunately the Batteries bot has not reported...

Kim Morrison (Feb 12 2025 at 22:31):

Oh, it's just that the nightly was delayed, and Batteries only attempts to bump once a day.

github mathlib4 bot (Feb 12 2025 at 22:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bdd34c370f2466b303c232fc320ddd7dfaca7c64).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 12 2025 at 23:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3b1a275d7417006ca5848ae48adf420134ff6944).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 13 2025 at 00:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5eae4dcb283ac0db0f41f06df2ae8bb0761add4b)

github mathlib4 bot (Feb 13 2025 at 09:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ea429a57f1d4efb65e26f4310ccb93d796878cf1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 13 2025 at 09:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4083b7d96b03db1ae474536012e2cb629f010422).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 13 2025 at 12:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b942da74f8bf8d8577e9ecc3ab706343c958d876).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 13 2025 at 13:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5c7de27570615977f1d1a584a0f695487198d86e)

github mathlib4 bot (Feb 13 2025 at 20:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a3bb69909ae946c3659866533005907fbd78eeae).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 13 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (12ceac2a5f46d84622214815f6e7e7643a2649d8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 14 2025 at 00:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (70d69e0b142c8d47d3c2f136ca660b909550cd97).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 14 2025 at 02:54):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5c7de27570615977f1d1a584a0f695487198d86e)

github mathlib4 bot (Feb 14 2025 at 10:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (75b995cefa6ef6c574af7d822b6ea0ce80975512).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 14 2025 at 13:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6b28ba204395930a138b9e9151ba8c473ac7d811).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 14 2025 at 16:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (adf649c0c29e0cd6e16cb77b76c47b4a8a527d07).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 14 2025 at 19:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5f7473608e12b27d4243ad79486918027c7082dd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 14 2025 at 22:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (33db31ba3c2834d1dfd1c8df81a5b75532bb6de3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 01:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ba17ac8ca5e15fcb115dff6cee13bd19cd08a6ec).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 04:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1d3ab40c18504d15b3513643a59b45173464ea3b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 07:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e26b4fff7a0f6cf71e6ca0b6e1acbfe09b96dcfa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e26b4fff7a0f6cf71e6ca0b6e1acbfe09b96dcfa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 10:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fc1556c1688753a0a34cf52a5754dac4f8fce3ca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 13:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab7cf6ecf4c4d8fbb3516e9c6142607095d95169).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 16:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0e2ee7f1d8259a7d551213325a07196d54583b6c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 19:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3e03c00e7fe7144abcb9c63a66961732e3d57f19).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 15 2025 at 22:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (74e8a3ebaa0145c600a1d1004633c964f535aa47).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 16 2025 at 01:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (502b60c32babe32cb62f862d4c88b84c192b20e7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 16 2025 at 04:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (41fdb023ec82ce52ac3d4201e709b5c8586dc4ca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 16 2025 at 07:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (282ec35e38db97ec473e5f3dc9d512ee3ae9e712).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 16 2025 at 10:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1d9f57a81f6167795d4b62f5ef18954e2c2e156b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 16 2025 at 13:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab024bba09a1433dacf9d56ddb167a5ce0de0e70).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 16 2025 at 16:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6df878a61a0077cdfd6d1f0c80c7eec1ef6b39df).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 16 2025 at 19:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bad4a1ac9f9da887aa78225c295fb2dfa9d3ce20).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 16 2025 at 22:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (171be8eee8b950b004bcdd12645180e9fd19b972).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Feb 16 2025 at 22:38):

@Mac Malone this appears to have been broken by your plugins PR lean4#7001. Could you please take a look on Monday?

I may try reverting lean4#7001 this afternoon to see if that fixes the problem.

Mac Malone (Feb 16 2025 at 22:47):

@Kim Morrison I think I might know what the issue is. I will make a quick PR.

Mac Malone (Feb 16 2025 at 22:55):

mathlib4#21967

github mathlib4 bot (Feb 16 2025 at 23:50):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ca6d4da0ff6cfe9c3e200119dca942a302da5521)

Kim Morrison (Feb 16 2025 at 23:51):

Thanks @Mac Malone, that seems to have done it!

github mathlib4 bot (Feb 17 2025 at 01:43):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ca6d4da0ff6cfe9c3e200119dca942a302da5521)

github mathlib4 bot (Feb 17 2025 at 08:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (981a86e7f2342cd84acac36c2ec4016f87ae54b6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 17 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (981a86e7f2342cd84acac36c2ec4016f87ae54b6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 17 2025 at 11:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1c17407c1e9b10702cd31fec793352ec0ed9ee20).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Feb 17 2025 at 11:22):

Okay, the next failure report should be the issue described at #nightly-testing > breakages from leanprover/lean4#7059 , i.e. the expected failures of Mathlib.Computability.PartrecCode and Mathlib.Computability.Tape.

Kim Morrison (Feb 17 2025 at 11:23):

I would like to just comment out those files until such time as someone has time for Mathlib/Computability, but our current CI setup makes it awkward to do so.

Commenting out the entire files (using /- ... -/: -- produces long lines) means that the style linter checking that everything imports Mathlib.Init fails.

Kim Morrison (Feb 17 2025 at 11:23):

Is there anything better than comment everything below the copyright header out, and then adding import Mathlib.Init?

Kim Morrison (Feb 17 2025 at 11:24):

I worry that this is confusing to undo for whoever subsequently fixes the files.

Damiano Testa (Feb 17 2025 at 11:28):

Some of the linters ignore "import-only files". I thought that the linter that checks for import Mathlib.Init did it as well.

Damiano Testa (Feb 17 2025 at 11:28):

If not, as seems to be the case, then maybe it should?

Damiano Testa (Feb 17 2025 at 11:30):

Alternatively, renaming to file to not have lean as an extension and then lake exe mk_all is "too aggressive"?

Kim Morrison (Feb 17 2025 at 11:38):

Definitely, that would be painful (and confusing) for the maintainers or contributors kindly coming in to help out with nightly-testing!

Kim Morrison (Feb 17 2025 at 11:40):

I've modified the affected files by adding:

import Mathlib.Init
/-
Broken by https://github.com/leanprover/lean4/pull/7059
Commenting out until a fix is available.
See https://leanprover.zulipchat.com/#narrow/channel/428973-nightly-testing/topic/breakages.20from.20leanprover.2Flean4.237059

below the existing copyright header. Hopefully that is clear enough? (And adding a -/ at the end of the file, except TMToPartrec, which still needs the set_option linter.longFile ... command after the closing -/, sigh.)

Damiano Testa (Feb 17 2025 at 11:45):

Ok, maybe the longFile linter singles out Mathlib.lean and does not look at it, not because it is import-only, but because it is hard-coded.

Damiano Testa (Feb 17 2025 at 11:58):

After Kyle fixed the weird interaction between linters and guard_msgs, I have not tried to see if #guard_msgs in #exit actually exits or not. If it does, maybe it is a possible alternative?

github mathlib4 bot (Feb 17 2025 at 12:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8a202d031663be948ea8dee0d7669ff6454f4df1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 17 2025 at 12:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8a202d031663be948ea8dee0d7669ff6454f4df1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 17 2025 at 13:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1027a18fb029a2d22e0ca36800e9da75d75fd883)

Kim Morrison (Feb 17 2025 at 14:37):

(Noting that this is cheating, and ~8 files are commented out still.)

github mathlib4 bot (Feb 17 2025 at 15:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1027a18fb029a2d22e0ca36800e9da75d75fd883)

github mathlib4 bot (Feb 17 2025 at 19:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (447722b3aa730f510a09beea582a6e6ec1b2bd63).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 17 2025 at 22:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (17ac720528e61e7aadd2b929f415c7bf22419399).
You can git fetch; git checkout nightly-testing and push a fix.

Mario Carneiro (Feb 17 2025 at 22:56):

Kim Morrison said:

I've modified the affected files by adding:

import Mathlib.Init
/-
Broken by https://github.com/leanprover/lean4/pull/7059
Commenting out until a fix is available.
See https://leanprover.zulipchat.com/#narrow/channel/428973-nightly-testing/topic/breakages.20from.20leanprover.2Flean4.237059

below the existing copyright header. Hopefully that is clear enough? (And adding a -/ at the end of the file, except TMToPartrec, which still needs the set_option linter.longFile ... command after the closing -/, sigh.)

I assume it is sufficient to revert this commit? Or did you comment or stub out other things in other commits

Mario Carneiro (Feb 17 2025 at 22:56):

One of the reasons I don't really like this kind of thing is because it makes it hard to find the damage later since all the linter stuff that would notice it is being made to look the other way

github mathlib4 bot (Feb 18 2025 at 01:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a221dba44ae741ff77b01747a9eb0b8a09101bbc).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Feb 18 2025 at 01:56):

Mario Carneiro said:

One of the reasons I don't really like this kind of thing is because it makes it hard to find the damage later since all the linter stuff that would notice it is being made to look the other way

No, it was multiple commits as I worked out how to satisfy the linters. In future, I can try to produce cleaner history.

github mathlib4 bot (Feb 18 2025 at 08:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6f90ebd99f9b2de8cbaa9784d6767412e91d804b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 18 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (03b816eb74b0af467c721e14fd1524bddb78aa98).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 18 2025 at 12:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (971ebb0f1bdf5bbee750b354df153b5430bc4dd7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 18 2025 at 13:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c5db03bc3823a4bb1c5982e179bf6bcd51cb8d33)

Mario Carneiro (Feb 18 2025 at 15:46):

@Kim Morrison ping me when the defeq issue is fixed on nightly and I'll return to fixing this

Mario Carneiro (Feb 18 2025 at 15:47):

oh, I guess this is fixed already with no need for my intervention

github mathlib4 bot (Feb 18 2025 at 16:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c5db03bc3823a4bb1c5982e179bf6bcd51cb8d33)

Kim Morrison (Feb 19 2025 at 08:52):

I suspect I have broken many things with lean#7132, which had stage0 conflicts so I merged before getting a Mathlib test.

github mathlib4 bot (Feb 19 2025 at 09:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (661276889ab41f2e9ce59c23cf96133f7ed9e462).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 19 2025 at 10:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9d75f595b5f562ce236ec76bd176ea7554966cec).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 19 2025 at 12:06):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7c50f8ced4c4698d6b5fff06a9a3bbad0918687e)

github mathlib4 bot (Feb 20 2025 at 10:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (022c5bb1b68fd03195eb7cc2743469be89e2d0aa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 20 2025 at 11:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (11dafdf912525bd451817754e52808e9d905b629)

github mathlib4 bot (Feb 21 2025 at 08:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dee71704df89691e3e217c29e9998bca08e19f10).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 21 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e48664a7a29f363d1eed2bbc6989f5b486dd01b1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 21 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f4084b19bfc93dfa43f54a16be771f883239b9ee).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 21 2025 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (82253b6d3ca0b8d565ab45e1a9a10afddb75e18d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 21 2025 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5b1b3d74cdcf3c68e5898413e35b03a896fe55e9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 21 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (31af98b7f5d0adb5681821dc909e9aae757fd312).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 22 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8d0660f3c507e19b8e729894cd0be53c2b1c73f5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 22 2025 at 08:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8d0660f3c507e19b8e729894cd0be53c2b1c73f5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 22 2025 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5c838de4ceea51b70e2fc7837fd69f113229cf84).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 22 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eb486ffca6a2439b15a8aa1e56dea3eaf0302563).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 22 2025 at 15:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (abeb840f4a76fa4764d076825b201238d83a20f7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 23 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (745dc1a50a9a1a4d8a07ff604cf0ef6c107b78a4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 23 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0c390854787ae3a35f9334440bcbf06131a42e79).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 23 2025 at 18:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f864d0937aa6cd687a7f635b6b9782b9deab69a3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 23 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d077be489541992fc5ce3bbe772033719b5fa64d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 23 2025 at 23:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9751f4aa21122d4cea52d2d67c0b74a8efc4ecf0).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Feb 23 2025 at 23:45):

I fixed the ProofWidgets problem by merging https://github.com/leanprover-community/ProofWidgets4/pull/106 and cutting v0.0.52-pre3. There are still some problems because I changed the statement of Nat.succ_div when upstreaming (actually, accidentally rewrote from scratch). I'll change the statement back as I prefer the Mathlib version anyway, but this will leave nightly-testing broken until this evening.

Kim Morrison (Feb 24 2025 at 00:45):

lean#7199 should resolve the problem.

github mathlib4 bot (Feb 24 2025 at 00:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f9a634b06186b59526875873596c5b3002ed1f47).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 24 2025 at 03:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5e2e7342a4a0ce726951b40d00a9a4311ba5e447).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 24 2025 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15d6896f929dd73f6c67f73a70bf2d8501bfe201).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Feb 24 2025 at 11:04):

Unfortunately nightly-2024-02-24 wasn't cut due to some bad Windows/Lake interaction, so this will stay broken for another day.

github mathlib4 bot (Feb 24 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f410b48e6f56b9943f4be4c116e130a301d5b4d2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 24 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (42e56d74539f652e619ef870f2f518d51eb8342c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 24 2025 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e7eb04a071d0a80ce155864cdc72483b6e7c345e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 24 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3c36ad8d9c291fd21e8846430561a796f48058ea).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 24 2025 at 23:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab84c0ea2b6847abd0ab4b91e0703c8dfb4d48e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 00:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab84c0ea2b6847abd0ab4b91e0703c8dfb4d48e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 00:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab84c0ea2b6847abd0ab4b91e0703c8dfb4d48e1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Feb 25 2025 at 00:36):

@Pim Otte would you be available to fix the problem in Mathlib.Combinatorics.SimpleGraph.Connectivity.WalkDecomp on the branch nightly-testing? Your PR from #21250 has broken it.

I'll look later if you're not available, but hopefully you're familiar and can fix it quickly.

Kim Morrison (Feb 25 2025 at 00:50):

Oh, actually, it's relatively easy to fix. Slight change in number of arguments needed in the induction cases, and a minor failure of aesop that I'm just going to turn into an #adaptation_note.

Kim Morrison (Feb 25 2025 at 00:50):

@Jannis Limperg, if you wanted to look into why aesop is failing in that file on nightly-testing, that might be interesting? But not urgent.

github mathlib4 bot (Feb 25 2025 at 00:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab84c0ea2b6847abd0ab4b91e0703c8dfb4d48e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 01:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab84c0ea2b6847abd0ab4b91e0703c8dfb4d48e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 03:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b75d09c3757f634b666e4b51874054483aa6bf56).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 03:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b75d09c3757f634b666e4b51874054483aa6bf56).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 04:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (2bfa3eb705b0fe9d6cdc11f91f728f66b1720dd5)

github mathlib4 bot (Feb 25 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (86a0f0103e5c950ac0393a7afebd5f1399fc7f55).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 10:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6d33eaf659620a8f914d9c9489dad0d27be88610).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 13:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c67469e39b41cc74773da68a763c281f17ef99d2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 16:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6760fb9ea118f04f766dea26e5f61f90fcc38cd9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (babf9a897ee32554a8aeb3d3cef39103ecfbf6eb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 25 2025 at 21:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aee605ae2774b6eff7380605c8d1deeb97f50e52).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Feb 25 2025 at 21:44):

Big merge conflict on Mathlib/Data/Multiset/Basic.lean, I'll just reset it to master and try to reconstruct fixes.

github mathlib4 bot (Feb 25 2025 at 22:30):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a429f616174b54dc85e0154c84bb2d46879e70ab)

github mathlib4 bot (Feb 26 2025 at 08:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d6d30b237e057d99c7287ff67fbe7dfa629f17b1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 26 2025 at 10:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (514991a14eea12ccac3a18f4d7bce8f8d4a4ee75).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 26 2025 at 13:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (215e9c6293496e3cccee65b4f66ebdc22c8ad728).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 26 2025 at 15:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ae7f5ae7147da1bc1fa7c7ad714ba0bb69edfe3f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 26 2025 at 19:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b4e9bce0fef2e8ca5f6bd605fd7286b0eed93782).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 26 2025 at 22:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5909c29b9f0edc1481ee81468643960fd939de01).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 26 2025 at 22:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5909c29b9f0edc1481ee81468643960fd939de01).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 26 2025 at 22:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (aaaee1505b7ad5fa5afb79aeb30a7d71d4f9c7f5)

github mathlib4 bot (Feb 27 2025 at 09:36):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (945c66e068c4e874261a90232fe9e5e35975c258)

github mathlib4 bot (Feb 28 2025 at 09:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2dccc4bdfd7c8a2eb1d6d00e154c6504cb1158d4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 28 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2dccc4bdfd7c8a2eb1d6d00e154c6504cb1158d4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 28 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c79faca1f2a068da579ab761d17f06fa19e8173e).
You can git fetch; git checkout nightly-testing and push a fix.

Jannis Limperg (Feb 28 2025 at 12:51):

Kim Morrison said:

Jannis Limperg, if you wanted to look into why aesop is failing in that file on nightly-testing, that might be interesting? But not urgent.

What's the relevant file here (if the issue is still current)?

Kevin Buzzard (Feb 28 2025 at 13:00):

I think this was #22334 and the issue was explicitly raised here and you've already seen it.

github mathlib4 bot (Feb 28 2025 at 15:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7b186b7632d2dfa423646963e7227a68871a23c8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 28 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11100128fea213a315f2b4a4bd98e9b8ff1b2057).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Feb 28 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (75362b3987c7c0019db82c9ed145f47d23ab9800).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 01 2025 at 00:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5aee0a154d404a5a1aa14f3687c1a1d0d7cb9a46)

github mathlib4 bot (Mar 01 2025 at 08:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fb85dc4d9b1b2228454595ca243ef3314098035a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 01 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2626910042c837ed53e1a8080cbcbdb514b7a2fb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 01 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f4f685a6111f1bb8a4489ccef4202b17b99fe1fd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 01 2025 at 15:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7fd64f5286d24f19faea943e8d19625ff38a645c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 01 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b5719fa2d64079a651f93b3784977a297a618478).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 02 2025 at 01:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (05c75f88e308a9835e4b8b41e3228c1af58c9ae2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 02 2025 at 10:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (05c75f88e308a9835e4b8b41e3228c1af58c9ae2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 02 2025 at 10:38):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f77cdc2ac5bc49894441dc437e08ae4d40f3271a)

github mathlib4 bot (Mar 02 2025 at 11:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3f72c0fe935cdf098015a701e7373b47ba8f044a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 02 2025 at 13:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (39688c3aef0cbc145c18a63cade521e336acbe67).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 02 2025 at 15:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cf215ba599681bc3777bbe0f61a7d61bd3b5a327).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 02 2025 at 19:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5ac57f40bfaa4629b7f8dff4c18f2a40340745b5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 02 2025 at 21:53):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f77cdc2ac5bc49894441dc437e08ae4d40f3271a)

github mathlib4 bot (Mar 03 2025 at 08:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (95c78f355f66ad3bdc174500d7b9824dd73cf14b).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 03 2025 at 09:35):

Okay, this is looking good locally, so once CI catches up nightly-2025-03-03 will become v4.18.0-rc1

github mathlib4 bot (Mar 03 2025 at 10:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (25e831ed30f19e534c0e14ca2ba8c5a785e7711f)

github mathlib4 bot (Mar 04 2025 at 09:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b6520862beeef981cf659ed2ed11192dff0d9ad8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 04 2025 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b6520862beeef981cf659ed2ed11192dff0d9ad8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 04 2025 at 09:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b6520862beeef981cf659ed2ed11192dff0d9ad8).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 04 2025 at 10:07):

Uhuh, nightly-testing is borked, and I don't immediately see what caused it.

There are lots of errors, e.g. on lines like

variable {C : Type u} [Category.{v} C] {X Y Z : C}

we get

invalid binder annotation, type is not a class instance
  Category C

that ... maybe ... are due to @Kyle Miller's structure elaboration changes?

But there are also consequences of parallelism changes landing, e.g.

(kernel) constant has already been declared 'Mathlib.Order.Disjoint._auxLemma.1'

all over the place.

Kim Morrison (Mar 04 2025 at 10:07):

@Sebastian Ullrich

Kim Morrison (Mar 04 2025 at 10:08):

We may need to revert some commits and proceed more slowly with them, working out the Mathlib adaptations as we go.

github mathlib4 bot (Mar 04 2025 at 10:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b6520862beeef981cf659ed2ed11192dff0d9ad8).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 04 2025 at 10:13):

@Kim Morrison Thanks for tagging me. Let me see if I can disable the problematic behavior with an option for now.

Sebastian Ullrich (Mar 04 2025 at 10:15):

All prior changes somehow not breaking mathlib must have made me too complacent!

Sebastian Ullrich (Mar 04 2025 at 10:41):

Here is a minimization of the first issue (same root cause), likely caused by Aesop using Replay, which I assumed was used only in lean4checker :grimacing:

import Aesop

class Bifunctor where

theorem t : True := by aesop

open Bifunctor  -- unknown namespace 'Bifunctor'

Kim Morrison (Mar 04 2025 at 10:46):

Yes, I'd forgotten Aesop used it too... :-(

Sebastian Ullrich (Mar 04 2025 at 11:43):

lean#7327 is the minimal revert that fixes Mathlib for me locally. I'm actually not sure how I'd convince the bot to run Mathlib CI on it... I guess I can do it manually once the toolchain exists.

github mathlib4 bot (Mar 04 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f1bcadd1f2bb82972b0557969f08e5f77b247161).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 04 2025 at 13:14):

https://github.com/leanprover-community/mathlib4/actions/runs/13653728073/job/38167927946 has passed except for the deprecation warning in Aesop. @Kim Morrison @Johan Commelin What should we do here, revert the deprecation, add an ignore to Aesop, do this before or after merging this PR, ...?

Johan Commelin (Mar 04 2025 at 13:19):

I guess the easiest thing is to briefly revert the deprecation

Johan Commelin (Mar 04 2025 at 13:20):

Then, once we have everything up and running again, we proceed via the usual nightly-testing update cycles.

Sebastian Ullrich (Mar 04 2025 at 13:20):

And this after I manually unreverted the deprecation from the revert commit :grinning: ... (I didn't think about it making the build fail). SGTM!

Sebastian Ullrich (Mar 04 2025 at 13:21):

I faintly remember some prior discussion that warnings in dependencies shouldn't be fatal...?

Sebastian Ullrich (Mar 04 2025 at 13:22):

Also while we're at it, could we get a lean4 label "please just run Mathlib on this PR's toolchain even though it's not based on nightly-with-mathlib, I accept that failures may come from changes landed in between"?

Sebastian Ullrich (Mar 04 2025 at 13:25):

I've queued lean#7327 with the full revert

github mathlib4 bot (Mar 04 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cdc8210ed5af5de9a751a9cd68417c6b66f73016).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 04 2025 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (82bee845872d75a660b2c236ce38f9b8ba348932).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 04 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (66201572ec628f40851f0e7a66b8b37a0114bd20).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 04 2025 at 22:04):

Sebastian Ullrich said:

Also while we're at it, could we get a lean4 label "please just run Mathlib on this PR's toolchain even though it's not based on nightly-with-mathlib, I accept that failures may come from changes landed in between"?

This is done (untested!) in

feat: force-mathlib-ci label lean#7337

github mathlib4 bot (Mar 05 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3ec11919dafdb1e387d179bb32443f304894b14e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 05 2025 at 03:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6cd25d22eb5167aadcfc5b3ba983d8145751abad).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 05 2025 at 07:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c8c1429f3c89e3a9c1a01dfe9a839884f41aebad).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 05 2025 at 07:16):

Not my fault!

Sebastian Ullrich (Mar 05 2025 at 08:34):

Kim Morrison said:

Sebastian Ullrich said:

Also while we're at it, could we get a lean4 label "please just run Mathlib on this PR's toolchain even though it's not based on nightly-with-mathlib, I accept that failures may come from changes landed in between"?

This is done (untested!) in

feat: force-mathlib-ci label lean#7337

Small follow-up: lean#7342

github mathlib4 bot (Mar 05 2025 at 09:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a69bc35b7028de551fb3c101d72f5ddbef2a6b2d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 05 2025 at 09:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a69bc35b7028de551fb3c101d72f5ddbef2a6b2d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 05 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (19e565f28586cfabfa4b33ac0960048ab95497d8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 05 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (47782bc260a0a7b85099d1aaaabd290aa9e8c5e1).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Mar 05 2025 at 18:31):

I've almost fixed it, but interrupted by meeting

github mathlib4 bot (Mar 05 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1fb7412a49749178a1aa78376901054bc7b7d5b4).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Mar 05 2025 at 20:09):

Pushed a fix, hopefully we get a :check: soon

github mathlib4 bot (Mar 05 2025 at 20:40):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dc26fc02df4023439f1359ce63a1b7c2ed6cc79d)

Sebastian Ullrich (Mar 06 2025 at 09:54):

@Johan Commelin I'm still a bit confused about the setup, what's left here for nightly-with-mathlib to advance?

github mathlib4 bot (Mar 06 2025 at 10:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (769e5739ce63a2ec8970b115f09c02cdf8255cda)

Kim Morrison (Mar 06 2025 at 21:57):

@Sebastian Ullrich, nightly-with-mathlib should update automatically at about the same time one of these :check: messages appears. At least right now it all looks correct (nightly-with-mathlib = nightly-2025-03-06).

github mathlib4 bot (Mar 07 2025 at 01:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (769e5739ce63a2ec8970b115f09c02cdf8255cda)

github mathlib4 bot (Mar 07 2025 at 08:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (708ea06c33feeced7befb2cc175aa048852df2ab).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 07 2025 at 08:55):

(fix on lean-pr-testing-7261)

github mathlib4 bot (Mar 07 2025 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6fcd9b0336604518bd58d639039886e58cbbe5a2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 07 2025 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (47faa13049950bc302bfdccb6bf0eff3dee0b589).
You can git fetch; git checkout nightly-testing and push a fix.

Joachim Breitner (Mar 07 2025 at 12:13):

Still getting

  [4011/6321] Building Mathlib.Data.Nat.ModEq
trace: .> LEAN_PATH=././.lake/packages/Cli/.lake/build/lib/lean:././.lake/packages/batteries/.lake/build/lib/lean:././.lake/packages/Qq/.lake/build/lib/lean:././.lake/packages/aesop/.lake/build/lib/lean:././.lake/packages/proofwidgets/.lake/build/lib/lean:././.lake/packages/importGraph/.lake/build/lib/lean:././.lake/packages/LeanSearchClient/.lake/build/lib/lean:././.lake/packages/plausible/.lake/build/lib/lean:././.lake/build/lib/lean /home/lean/.elan/toolchains/leanprover--lean4---nightly-2025-03-07/bin/lean -Dpp.unicode.fun=true -DautoImplicit=false -DmaxSynthPendingDepth=3 -Dweak.linter.docPrime=false -Dweak.linter.hashCommand=true -Dweak.linter.oldObtain=true -Dweak.linter.refine=true -Dweak.linter.style.cdot=true -Dweak.linter.style.dollarSyntax=true -Dweak.linter.style.header=true -Dweak.linter.style.lambdaSyntax=true -Dweak.linter.style.longLine=true -Dweak.linter.style.longFile=1500 -Dweak.linter.style.missingEnd=true -Dweak.linter.style.multiGoal=true -Dweak.linter.style.setOption=true ././././Mathlib/Data/Nat/ModEq.lean -R ./././. -o ././.lake/build/lib/lean/Mathlib/Data/Nat/ModEq.olean -i ././.lake/build/lib/lean/Mathlib/Data/Nat/ModEq.ilean -c ././.lake/build/ir/Mathlib/Data/Nat/ModEq.c --json
error: ././././Mathlib/Data/Nat/ModEq.lean:388:14: unknown identifier 'add_div'
error: ././././Mathlib/Data/Nat/ModEq.lean:388:7: unsolved goals
a b c : 
hc : a % c + b % c < c
hc0 : ¬c = 0
 (a + b) / c = a / c + b / c
error: ././././Mathlib/Data/Nat/ModEq.lean:402:46: unknown identifier 'add_div'
error: ././././Mathlib/Data/Nat/ModEq.lean:402:39: unsolved goals
a b c : 
hc : c  a % c + b % c
hc0 : 0 < c
 (a + b) / c = a / c + b / c + 1
error: Lean exited with code 1
Some required builds logged failures:
- Mathlib.Data.Nat.ModEq

Pushed a possible fix.

github mathlib4 bot (Mar 07 2025 at 12:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (062d4014b715b18f58ad03a61aac66fa9b2e0c8a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 07 2025 at 13:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (062d4014b715b18f58ad03a61aac66fa9b2e0c8a).
You can git fetch; git checkout nightly-testing and push a fix.

Joachim Breitner (Mar 07 2025 at 13:30):

error: ././././Mathlib/RingTheory/Etale/Kaehler.lean:260:9: tactic 'simp' failed, nested error:
(deterministic) timeout at `isDefEq`, maximum number of heartbeats (200000) has been reached
Use `set_option maxHeartbeats <num>` to set the limit.

:-(. I'll let someone else investigate.

github mathlib4 bot (Mar 07 2025 at 16:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (71c053b52b54091905c34735bff35f3ea1952ec8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 07 2025 at 18:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7b4a09d2102c2eae2457af54dfcb57a51e99c5e0).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 07 2025 at 21:08):

I had this failure before, in the second-to-last Mathlib run of #7306. I was in fact missing a significant optimization there that then fixed the timeout but we may already have been very close to the heartbeat limit.

github mathlib4 bot (Mar 07 2025 at 21:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7b4a09d2102c2eae2457af54dfcb57a51e99c5e0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 08 2025 at 01:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7590675dfaa93de9844d39fe9c13106c327456e0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 08 2025 at 06:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b764a7e13144f807222716ea4e59bdcfecbdd5e9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 08 2025 at 09:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1a7567c33383f8e9615432a71764b63e75bedcd3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 08 2025 at 10:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1a7567c33383f8e9615432a71764b63e75bedcd3).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 08 2025 at 10:55):

Error: ././././Mathlib/RingTheory/LocalRing/ResidueField/Ideal.lean:52:1: error: @Ideal.algebraMap_residueField_eq_zero LINTER FAILED:
simplify fails on left-hand side:
failed to synthesize
  FaithfulSMul R I.ResidueField
(deterministic) timeout at `typeclass`, maximum number of heartbeats (20000) has been reached

How concerning is that error, how easy is it to extract so I can debug it, how easy is it to work around it? I am currently very interested in steady nightly-with-mathlib bumps :)

Sebastian Ullrich (Mar 08 2025 at 11:22):

(but also as it happens very late, I'm happy to move forward by manually checking I don't introduce any earlier errors)

Kevin Buzzard (Mar 08 2025 at 11:22):

Did you try just bumping the heartbeats? This might just be something that was tipped over a timeout limit

Sebastian Ullrich (Mar 08 2025 at 11:23):

I don't know how to do that in that linter

Kevin Buzzard (Mar 08 2025 at 11:26):

FWIW the thing it's failing to synthesize is false

Kevin Buzzard (Mar 08 2025 at 11:42):

I guess you could just do @[simp, nolint simpNF] for now if you want a cheap workaround? (this pattern seems to occur 100 or so times in mathlib right now). It looks like a fine simp lemma to me, as you can see the linter isn't failing because it's a bad simp lemma, it's failing because typeclass inference isn't failing quickly enough for some reason. Can you or someone else remind me how to run the linter on this declaration so I can try and see what typeclass inference is doing? Linters are not usually a part of my life.

import Mathlib

#check Ideal.algebraMap_residueField_eq_zero

-- I now want to emulate what the`simpNF` linter does when checking that this declaration is OK

Kevin Buzzard (Mar 08 2025 at 12:30):

I don't understand how to see this error locally:

import Mathlib

#check Ideal.algebraMap_residueField_eq_zero

#lint only simpNF -- works for me on `nightly-testing`

github mathlib4 bot (Mar 08 2025 at 13:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b5f64a74473714468ab3eedd7c5d541aa404e6ab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 08 2025 at 16:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e57f8bcdcdcfa30a17b98943553eb60b93b86462).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 08 2025 at 18:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c30d062e171b74fc1b45e6ebb6fe2e519adc37d3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 08 2025 at 21:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (02a95579e1f4019008bc071284372d1a13f41004).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 09 2025 at 01:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f8f22d77ccc4ec01b7b8eabee793576d59838c06).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 09 2025 at 03:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f8f22d77ccc4ec01b7b8eabee793576d59838c06).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 09 2025 at 10:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fbe595fc740ee7a1789c6e6ebefa322e054a41c0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 09 2025 at 12:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e9ada999b476e5d6c145a0f81799500f20714209).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 09 2025 at 16:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (40a8beb29d3de17bd5b7c7adac652eb57fe60e52).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 09 2025 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c48e6c5e5e440e02eceaf7fba44004d0f95f97d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 09 2025 at 21:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (182acfb6bb259564c7d2b4611ea21ac5460dbb08).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 10 2025 at 01:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (63a7be57d4c98d1a8df636cc6b645c121dc5c94c).
You can git fetch; git checkout nightly-testing and push a fix.

Jovan Gerbscheid (Mar 10 2025 at 02:24):

I've added a fix for the simpNF timeout here: #22753

github mathlib4 bot (Mar 10 2025 at 07:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7bc8f1592591c2c90e8af6fecf540bbdc3c57a42).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 10 2025 at 07:24):

@Jovan Gerbscheid Thanks, I cherry-picked it

github mathlib4 bot (Mar 10 2025 at 07:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (21ebdb2ad2d0096a136ba23ec43ffa98f68f0962)

github mathlib4 bot (Mar 10 2025 at 10:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f946d24de494227fcbef6ed1a73b5f4a8bde1bb1)

Matthew Ballard (Mar 10 2025 at 12:47):

I actually got a little time to look at this timeout.

First, @Kevin Buzzard , to recreate

import Mathlib

variable {R : Type u_1}  [CommRing R]  {I : Ideal R}  [I.IsPrime]  {x : R}

example : (algebraMap R I.ResidueField) x = 0  x  I := by simp

Some more automation around this would be nice. How much information can be in simpNF or in batteries? Even just have a expand_to_example% which produces the two last lines (maybe with a sorry) and supports replacing via a code action would be nice.

While @Jovan Gerbscheid 's fix side-steps the underlying issue, you can see from timing synthesis problems like Finite R I (I deleted my scratch code so might be slightly off from memory) takes a quite a bit of time.

I did find some low-lying problems which I will PR momentarily.

github mathlib4 bot (Mar 10 2025 at 13:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f946d24de494227fcbef6ed1a73b5f4a8bde1bb1)

github mathlib4 bot (Mar 11 2025 at 01:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (00d98b7f59e62aafcf9356987d6db7d75f0d8c59).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 11 2025 at 03:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3dec5e5b2c10a00f75c5c13fbb34c8514473b3f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 11 2025 at 05:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3dec5e5b2c10a00f75c5c13fbb34c8514473b3f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 11 2025 at 07:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f946d24de494227fcbef6ed1a73b5f4a8bde1bb1)

github mathlib4 bot (Mar 11 2025 at 10:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a75783f538090ee16c118d9583f3e5576a17cd7d)

github mathlib4 bot (Mar 12 2025 at 09:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d8118779ef2b2a598d6faa29f73849521b5a3665).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 12 2025 at 09:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3f061f51a223a85156efa61ae26e11b3ba32d89a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 12 2025 at 12:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7d0d31ed071ec4b23219de57e49d24024d06e6ef).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 12 2025 at 12:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b264b11f9193bcda26faaeac5edec4d4f6aa65d5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 12 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7ec05b96a6218a15a580c2e4c7f1bf18dbb91a55).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 12 2025 at 19:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7ec05b96a6218a15a580c2e4c7f1bf18dbb91a55).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 12 2025 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bb749e53d0aee387fb458be7a348963e03f56702).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 12 2025 at 22:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bb749e53d0aee387fb458be7a348963e03f56702).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 13 2025 at 01:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (241c1c00e575745dd020c4b1dfa11ce70ac6dcfd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 13 2025 at 04:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b4514b844977cfb75bdd82655141590f2ca84146).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 13 2025 at 04:21):

@Sebastian Ullrich

 [2669/2671] Building Counterexamples.AharoniKorman
trace: .> LEAN_PATH=././.lake/packages/Cli/.lake/build/lib/lean:././.lake/packages/batteries/.lake/build/lib/lean:././.lake/packages/Qq/.lake/build/lib/lean:././.lake/packages/aesop/.lake/build/lib/lean:././.lake/packages/proofwidgets/.lake/build/lib/lean:././.lake/packages/importGraph/.lake/build/lib/lean:././.lake/packages/LeanSearchClient/.lake/build/lib/lean:././.lake/packages/plausible/.lake/build/lib/lean:././.lake/build/lib/lean /home/lean/.elan/toolchains/leanprover--lean4---nightly-2025-03-12/bin/lean -Dpp.unicode.fun=true -DautoImplicit=false -DmaxSynthPendingDepth=3 -Dweak.linter.docPrime=false -Dweak.linter.hashCommand=true -Dweak.linter.oldObtain=true -Dweak.linter.refine=true -Dweak.linter.style.cdot=true -Dweak.linter.style.docString=true -Dweak.linter.style.dollarSyntax=true -Dweak.linter.style.header=true -Dweak.linter.style.lambdaSyntax=true -Dweak.linter.style.longLine=true -Dweak.linter.style.longFile=1500 -Dweak.linter.style.missingEnd=true -Dweak.linter.style.multiGoal=true -Dweak.linter.style.setOption=true ././././Counterexamples/AharoniKorman.lean -R ./././. -o ././.lake/build/lib/lean/Counterexamples/AharoniKorman.olean -i ././.lake/build/lib/lean/Counterexamples/AharoniKorman.ilean -c ././.lake/build/ir/Counterexamples/AharoniKorman.c --json
error: ././././Counterexamples/AharoniKorman.lean:600:6: (kernel) unknown constant '_private.Counterexamples.AharoniKorman.0.aux_4'
error: ././././Counterexamples/AharoniKorman.lean:631:49: unknown identifier 'chainBetween_subset'
error: ././././Counterexamples/AharoniKorman.lean:712:12: unknown identifier 'chainBetween_subset.trans'
error: ././././Counterexamples/AharoniKorman.lean:712:42: unknown identifier 'chainBetween_subset.trans'
error: ././././Counterexamples/AharoniKorman.lean:713:4: no goals to be solved
error: ././././Counterexamples/AharoniKorman.lean:746:53: unknown identifier 'chainBetween_subset'
error: ././././Counterexamples/AharoniKorman.lean:750:61: unknown identifier 'chainBetween_subset'
error: ././././Counterexamples/AharoniKorman.lean:746:53: unknown identifier 'chainBetween_subset'
error: ././././Counterexamples/AharoniKorman.lean:750:61: unknown identifier 'chainBetween_subset'
error: ././././Counterexamples/AharoniKorman.lean:1160:66: unknown identifier 'chainBetween_subset'
error: Lean exited with code 1
Some required builds logged failures:
- Counterexamples.AharoniKorman

this looks like fallout from lean#7334.

Kim Morrison (Mar 13 2025 at 04:22):

(Noting this file was added to Mathlib since the lean-pr-testing-7334 branch. Unfortunate timing! :-)

github mathlib4 bot (Mar 13 2025 at 06:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3d3450d07cf30b50e25e716277fb3381203cc3c0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 13 2025 at 06:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0b9bf05f3a1f9ae5a35c26127cc6bd94d0692d31).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 13 2025 at 08:21):

Thanks, likely addressed by #7468. Let's see if the new awaiting-mathlib works.

Johan Commelin (Mar 13 2025 at 08:23):

lean4#7468, I guess

Kim Morrison (Mar 13 2025 at 09:48):

@Sebastian Ullrich, this doesn't seem to have fixed the problem: https://github.com/leanprover-community/mathlib4/actions/runs/13830537191/job/38693617032

Sebastian Ullrich (Mar 13 2025 at 09:51):

Yes :( . Must be some fun new aesop edge case.

Kim Morrison (Mar 13 2025 at 10:04):

This feels like one of those brain surgeries where you need the patient awake in order to be able to tell you what they experience as you poke stuff...

github mathlib4 bot (Mar 13 2025 at 10:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6bc8904b57469119759a2455637235bfde44c0db).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 13 2025 at 11:03):

@Joachim Breitner I think this is actually your bug! You taught omega to create helper decls but as aesop uses independent branches with independent environments during proof search, they all end up with the same name and clash. Oh but there's also a bug of mine in there. /cc @Jannis Limperg

Sebastian Ullrich (Mar 13 2025 at 12:05):

IOW, Aesop is incompatible with Term.mkAuxName, which does have a few users
image.png

Sebastian Ullrich (Mar 13 2025 at 12:11):

lean#7472 is my part

Sebastian Ullrich (Mar 13 2025 at 12:15):

@Kim Morrison @Johan Commelin As Joachim is traveling for the rest of the week and we wouldn't like to revert his omega optimizations anyway, can we instead (temporarily) ban uses of omega in aesop, e.g. by ignoring this file on nightly-testing?

Kim Morrison (Mar 13 2025 at 12:20):

Sounds good to me. I've commented out the file on nightly-testing, explaining why.

github mathlib4 bot (Mar 13 2025 at 12:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (759a343fcbe32736f2daf14cabc24daebc9f5a25)

Bhavik Mehta (Mar 13 2025 at 19:15):

Ah, and I felt so clever for putting omega into aesop here! Sorry about this, I can try to look into expanding the aesop proofs if it could be helpful

Kim Morrison (Mar 13 2025 at 21:23):

No, we'll work out how to support this. It's a reasonable use case.

github mathlib4 bot (Mar 13 2025 at 21:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (759a343fcbe32736f2daf14cabc24daebc9f5a25)

github mathlib4 bot (Mar 14 2025 at 01:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c9d2c019972c9e3ea71c05f73ca58509dcfeb929).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 14 2025 at 02:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c9d2c019972c9e3ea71c05f73ca58509dcfeb929).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 14 2025 at 03:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b6dd454218e8c57933f0b8d803a67f7be8dd805c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 14 2025 at 05:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (759a343fcbe32736f2daf14cabc24daebc9f5a25)

github mathlib4 bot (Mar 14 2025 at 09:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f59312e8d961ed53df84891871a33fb6dfba5b39).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 14 2025 at 09:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f59312e8d961ed53df84891871a33fb6dfba5b39).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 14 2025 at 09:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f59312e8d961ed53df84891871a33fb6dfba5b39).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 14 2025 at 10:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (561c554d22db2729782b18be032ec89b74d3aef4).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 14 2025 at 10:27):

All but ProofWidgets fixed!

github mathlib4 bot (Mar 14 2025 at 12:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8b48c43888d14d57927ca79be20c3471e1e31a3a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 14 2025 at 13:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9cb2a54e1ffd8914b9e0e46de954703a37827f9e)

github mathlib4 bot (Mar 15 2025 at 09:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3543cd86729039b24e8ac9551a954830f1b28053).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 15 2025 at 09:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3543cd86729039b24e8ac9551a954830f1b28053).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 15 2025 at 11:05):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (950e64cf316acd5865d007144850dcc4d230381c)

github mathlib4 bot (Mar 16 2025 at 15:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bce45b1a1db87943837ca86c2571d84b75b1ae59).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 16 2025 at 16:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bce45b1a1db87943837ca86c2571d84b75b1ae59).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 16 2025 at 18:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (76e119df17aeb67c2113dca4152ef5374e7525d9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 16 2025 at 22:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cf8a78f5098134de16ff6ab7cd128cd2ab3e3bca).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 17 2025 at 01:29):

Hmm... not sure what is going on here in nightly-testing. There is a universe problem in docs#Condensed.hasExactColimitsOfShape, but I don't yet see what has changed that could cause it.

Kim Morrison (Mar 17 2025 at 01:30):

Pinging @Dagur Asgeirsson in case he can see what is wrong on nightly-testing in this file?

github mathlib4 bot (Mar 17 2025 at 01:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5e56bc5f5dc2d51190c1ceb262837832e92bd8dd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 17 2025 at 04:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d27bbbade646eee4861ab995025a66c5578c8a11).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 17 2025 at 06:19):

@Kim Morrison It's the new restriction we talked about, fixed on 7485

github mathlib4 bot (Mar 17 2025 at 07:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (896c41d5344c32d8a98a043dccfd27aa7db7bc31).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 17 2025 at 07:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (896c41d5344c32d8a98a043dccfd27aa7db7bc31).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 17 2025 at 07:17):

lean#7485

Sebastian Ullrich (Mar 17 2025 at 07:35):

Oh, I guess I missed some test failures

Kim Morrison (Mar 17 2025 at 07:36):

(I've just been looking)

Kim Morrison (Mar 17 2025 at 07:36):

Two of them are just messages coming in a different order.

Kim Morrison (Mar 17 2025 at 07:36):

Okay I guess?

Sebastian Ullrich (Mar 17 2025 at 07:36):

Yeah, looks benign

Sebastian Ullrich (Mar 17 2025 at 07:37):

The ordering is deterministic at least, just different now

Kim Morrison (Mar 17 2025 at 07:37):

The error in MathlibTest.StacksAttribute disappears if we set_option Elab.async false, but I'm not sure what the right fix is. Should run_cmd do this internally?

Sebastian Ullrich (Mar 17 2025 at 07:37):

I'll take a look, on my phone atm

Kim Morrison (Mar 17 2025 at 07:38):

MathlibTest/eqns.lean ... eqns just seems scary with parallelism!

Sebastian Ullrich (Mar 17 2025 at 07:49):

Hmm, it looks like only that specific sanity check is broken. We'd have to wait on all prior tasks in order to implement it correctly, in which case it might be better to drop it?

Damiano Testa (Mar 17 2025 at 07:58):

As for Stacks, maybe the issue is that the same file adds a declaration with the stacks attribute and checks that the declaration has been added to the relevant environment extension. Maybe the check that the declaration is in the extension happens before the declaration has had a chance of being added to the environment?

github mathlib4 bot (Mar 17 2025 at 08:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aeb47dbc742b827ac76eeb129024164fb0a3eaf5).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 17 2025 at 08:03):

I pushed a fix for the stacks attribute

Sebastian Ullrich (Mar 17 2025 at 08:04):

@Kim Morrison You were right, eqns is totally borked now! Equation generation for n is now more deterministic because it only considers the environment just after n was declared. But of course it is not possible to have a custom equation theorem for n ready at that point

Dagur Asgeirsson (Mar 17 2025 at 08:06):

I see you have fixed (worked around?) the errors in the condensed files. Is the issue that the universes of two terms of type Type*are unified in the proof? Is it better to declare their universes explicitly if they're supposed to be different?

Sebastian Ullrich (Mar 17 2025 at 08:10):

Yes, that would be ideal I think!

Sebastian Ullrich (Mar 17 2025 at 08:20):

Note: the equation theorem in the test file must have been broken for a while on nightly-testing. It turns out the test still passes with it commented out.

Sebastian Ullrich (Mar 17 2025 at 08:39):

I've committed the broken test output for now to move forward /cc @Eric Wieser

github mathlib4 bot (Mar 17 2025 at 09:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (69eb24d5020265f3fc2048e69137faa1b368ee67)

Kevin Buzzard (Mar 17 2025 at 09:05):

Elab.async one step closer!

github mathlib4 bot (Mar 17 2025 at 09:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bdf308ca17a6c2fae2c96b97393cadae10dbaae9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 17 2025 at 09:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cd5cafa0792571c24db04050f3cadbd9bfcaab4c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 17 2025 at 13:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (74fcac18838c8908e392d6ec7e898422afba88dc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 17 2025 at 14:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (0b0ab2589bbb44452061502e9cb849837c9c25d2)

github mathlib4 bot (Mar 17 2025 at 16:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eab98761167237d45662033394ebd5ee28613aac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 17 2025 at 16:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eab98761167237d45662033394ebd5ee28613aac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 17 2025 at 19:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8deb89281cb9880d8b820a009446ca9a3a58bdcb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 17 2025 at 22:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (db4c8abb9243cf1b6c77c8e544c7c851495af16a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 01:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6bdd998c78a3415946ead62bacb83dd271fd8a73).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 01:54):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (0b0ab2589bbb44452061502e9cb849837c9c25d2)

github mathlib4 bot (Mar 18 2025 at 04:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (53ec0b449760780e476e03e813e080c79b36313c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 07:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (96f29be0737b9f7d8c6bf45d2fc555098fdfd743).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 11:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d22bd4f990c36ec29867ef381dc67f43c3d40520).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 13:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4d4e085b7b6dc6611a76abfaf1a670768d43e500).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 15:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f1a5be535d23e5ecdf7ea79c2b992b0a885c6568).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 17:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ccef7686f4018a0b3b2ff152eafc7847a339d542).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 19:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (609bae754789c3d933632e304f217bbdd6ef1efb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 18 2025 at 22:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (345037212607a4b992e19bd7ab8c753387b57f2d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 19 2025 at 04:10):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b266c88eaaff9448445982628b6814ef2f94a7df)

github mathlib4 bot (Mar 19 2025 at 09:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (67019e0bbfaccd3af41e6f73024551c6e80ad2d4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 19 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (67019e0bbfaccd3af41e6f73024551c6e80ad2d4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 19 2025 at 13:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (bfb212af9d68914d3bcc24b863982969d89d861b)

github mathlib4 bot (Mar 20 2025 at 11:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2ad02e6d6419f8abdafcaffafada59cb54f5175b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 20 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (88f302b1740f7ff57d9037e7f02b45049bcff58c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 20 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bcaf02fadadb12180d9e38bc13b4036230c2f8c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 20 2025 at 18:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (61c8f96c19c529532f1650e255558d75561c7d28).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 20 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1809290af1237825991a63be10682cc327aec7d5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 20 2025 at 23:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (390f4edd30d68d493e6b38527f2a73646aa30293)

github mathlib4 bot (Mar 21 2025 at 10:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d7c024f0292e801365f36c1ab2ba2ee2da009e32).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 21 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6925c7e1b5932ad33cf868822fa25d048b2d2d9e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 21 2025 at 14:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9bbdf45da08425e91c080c63920b48533fe2f594).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 21 2025 at 15:38):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7c56b4c877c1b368d8b76a9bafa5ecbcaf0a43b2)

github mathlib4 bot (Mar 22 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a1bb21e46be5808a61489d472fcf6538d297e7c9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 22 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (20c260b92867bf530bb611360824ea31b6906d02).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 22 2025 at 15:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eb9b70720b0adbffd6a55010f2bed3ef593bef3c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 22 2025 at 19:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a4da278bf7e2eb4701117e21a87c2a16007e656b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 22 2025 at 22:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (61d602d9afcf8ce50f9ad0426f52b3f13ec9fe5c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 23 2025 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ae6fafc73f476ce66d1d3257d04f758fa1e25a93).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 23 2025 at 04:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eab25444d0e0876a8a80fede02da98a761266d48).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 23 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (40de6ff425a9b85795171505195c7d547fbaecb8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 23 2025 at 13:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (195ac92a5ce4656318c1e78ca1bd39da30bd1715).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 23 2025 at 15:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (df882075248003a227363d639e2fb53b5a3c658d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 23 2025 at 18:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ff7c9298d1d2633e5104a9c3577b14437f526039).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 23 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ff7c9298d1d2633e5104a9c3577b14437f526039).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 23 2025 at 19:55):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (0336b0207f74597b520457c4de723c3bad571a2c)

github mathlib4 bot (Mar 24 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c441f7b6964d8337ba5a736403f696aa24afe072).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 24 2025 at 13:47):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (0336b0207f74597b520457c4de723c3bad571a2c)

github mathlib4 bot (Mar 24 2025 at 14:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d499abdf5a10c078627f8bd4fd58f0c680d64019).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 24 2025 at 15:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d499abdf5a10c078627f8bd4fd58f0c680d64019).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 24 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f3baa493991af10fc9896c8ac834e9a484da3da7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 24 2025 at 15:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f3baa493991af10fc9896c8ac834e9a484da3da7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 24 2025 at 16:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6995c4c3b4ab7565955e9e9bc202ca07a3ed7f7a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 24 2025 at 16:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (689ff66332639ec77b017dc0c24c5c8721c91d79).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Mar 24 2025 at 17:29):

Was https://github.com/leanprover-community/mathlib4/commit/6027e36a6252bf64cd76df86c50dda184e7d31d4#diff-eee30c5d524ebf27d1bd42a6128196f01b7eee44d8286e352d885c5a1afc5209L315 a by exact? fix @Kim Morrison ? That ended up changing the signature and making an impossible instance. Pushed a fix.

github mathlib4 bot (Mar 24 2025 at 18:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1ebd64f226d2bbb857698fc31efaeb9b72a2b1d1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 24 2025 at 19:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (98c6231f61d24a768245c3a0719e3d617c198f13).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 24 2025 at 20:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e7f18a305a91a997d0b68d407e433b78ea51d60a)

Kim Morrison (Mar 24 2025 at 23:40):

Kyle Miller said:

Was https://github.com/leanprover-community/mathlib4/commit/6027e36a6252bf64cd76df86c50dda184e7d31d4#diff-eee30c5d524ebf27d1bd42a6128196f01b7eee44d8286e352d885c5a1afc5209L315 a by exact? fix Kim Morrison ? That ended up changing the signature and making an impossible instance. Pushed a fix.

Oops, my fault, but I don't remember what I was doing. Thanks for catching this one.

github mathlib4 bot (Mar 25 2025 at 00:35):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e7f18a305a91a997d0b68d407e433b78ea51d60a)

github mathlib4 bot (Mar 25 2025 at 10:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5aab19e80b3649cc8fe899f46cbacafa341877ac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 25 2025 at 13:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6e04344033ed5a6b2eb4582fa713e56c473994de).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 25 2025 at 16:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f832b4494a6dfb53a644216142b0a0eea21d2d66).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 25 2025 at 19:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2ff7d06e7a6789eef7a2c1e755ec7ce70f0107bc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 25 2025 at 21:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3cd8962b3f158a8f957d8d2e81662ee09e5cd286).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Mar 25 2025 at 21:20):

It seems to be some simp/aesop timeouts. One timeout I fixed by adding in a dsimp only. (I think we'll be able to remove that one in one of the next nightlies.)

Concerningly, one of the failing cases causes dsimp only to time out if I try adding it.

github mathlib4 bot (Mar 25 2025 at 22:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b3fa3dd1f39fbef29e5ebbe0271df54005c1bbc3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 25 2025 at 23:28):

I've just added maxHeartbeats 400000 to the three places still failing, for now.

Kim Morrison (Mar 25 2025 at 23:29):

@Yaël Dillies, but you be able to look at ChevalleyThm.PolynomialC.induction_aux in your newly added ChevallyComplexity.lean file, on nightly-testing, and see if you can either just get it back down under the heartbeats limit, or localize to any extent what has slowed down?

github mathlib4 bot (Mar 25 2025 at 23:41):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ed4fcfffeca0d59158ff44e2aa842d4709ff446b)

github mathlib4 bot (Mar 26 2025 at 09:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8c625a214da99ac4a231481ea7e15d224345407c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 26 2025 at 09:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8c625a214da99ac4a231481ea7e15d224345407c).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 26 2025 at 09:23):

Batteries and Aesop needed some fixes for lean#7679.

github mathlib4 bot (Mar 26 2025 at 10:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b97db3eddf5a50dd47937cfd4018ba7661ce9cf1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 26 2025 at 10:33):

Sad, more maxHeartbeats on nightly-2025-03-26, it seems. :-(

github mathlib4 bot (Mar 26 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (80bca22cca4fab91f21d7b53b9185b61b4244da7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 26 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cc40bfec1047f8c40fb3856921406f69431a735e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 26 2025 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (97f8d3677882d02cebb2af67bb45c31a501f6b3a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 26 2025 at 23:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b6525099e2a2ec55700b17e01012ff7c1c95de7).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 26 2025 at 23:58):

Separately from this issue, there are a number of new slow-downs on nightly-testing under nightly-2025-03-26. All of them seem to be aesop calls. You can find these by looking for /-- Requires more heartbeats after nightly-2025-03-26. -/ on nightly-testing.

The relevant change in Aesop is:

% git diff 30671eb0eca7678572c74fd0c798e443b00dc259
diff --git a/Aesop/Util/Tactic/Unfold.lean b/Aesop/Util/Tactic/Unfold.lean
index 2183355..a32f44d 100644
--- a/Aesop/Util/Tactic/Unfold.lean
+++ b/Aesop/Util/Tactic/Unfold.lean
@@ -50,7 +50,7 @@ where
         Simp.tryTheorem? e
           { origin := .decl unfoldThm
             proof := mkConst unfoldThm
-            rfl :=  isRflTheorem unfoldThm }
+            rflTask :=  isRflTheorem unfoldThm }
       match result? with
       | none   => return .continue
       | some r =>
diff --git a/lean-toolchain b/lean-toolchain
index ab5f1f6..5b70d13 100644
--- a/lean-toolchain
+++ b/lean-toolchain
@@ -1 +1 @@
-leanprover/lean4:nightly-2025-03-25
+leanprover/lean4:nightly-2025-03-26

which is adapting (possibly incorrectly) to @Sebastian Ullrich's lean#7679.

Pinging also @Jannis Limperg.

github mathlib4 bot (Mar 27 2025 at 00:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c66c94d8c525d7da0f6c199ffc6968b7c992029c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c66c94d8c525d7da0f6c199ffc6968b7c992029c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 03:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f67208eb8713418887cd9e6e9e0a342a6c50ba98).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 06:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4e2055c27e7a1c05925f7a89b58e758750ea0e84).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Mar 27 2025 at 07:05):

For the slowdowns it would be good to know if these are purely heartbeats or wall clock as well

github mathlib4 bot (Mar 27 2025 at 09:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0d97ff349103148789c8d8c9d8793852f5c475bd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 09:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0d97ff349103148789c8d8c9d8793852f5c475bd).
You can git fetch; git checkout nightly-testing and push a fix.

Yaël Dillies (Mar 27 2025 at 09:50):

Kim Morrison said:

Yaël Dillies, but you be able to look at ChevalleyThm.PolynomialC.induction_aux in your newly added ChevallyComplexity.lean file, on nightly-testing, and see if you can either just get it back down under the heartbeats limit, or localize to any extent what has slowed down?

I will try looking today but no promise I'll get to it

github mathlib4 bot (Mar 27 2025 at 09:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e50e0918c715bdd03e268b42428b4415db151c19).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 27 2025 at 10:22):

Kim Morrison said:

Separately from this issue, there are a number of new slow-downs on nightly-testing under nightly-2025-03-26. All of them seem to be aesop calls. You can find these by looking for /-- Requires more heartbeats after nightly-2025-03-26. -/ on nightly-testing.

and unfortunately there are even more, and more severe, slow-downs on nightly-2025-03-27. Sebastian and I are starting to profile the worst of these now.

github mathlib4 bot (Mar 27 2025 at 10:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (eff9da572aaa6b532c82a3994deceb722cd92cb5).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 27 2025 at 10:40):

Here are before and after profiler results from docs#CommRingCat.monoidAlgebraAdj.

simps use of isDefEq has hugely blown out.

Sebastian Ullrich (Mar 27 2025 at 12:16):

attribute [-simp]
  Std.DTreeMap.Const.compare_maxKey_modify_eq
  Std.DTreeMap.Const.compare_maxKey!_modify_eq
  Std.DTreeMap.Const.compare_minKey_modify_eq
  Std.DTreeMap.Const.compare_minKey!_modify_eq
  Std.DTreeMap.Const.compare_minKeyD_modify_eq
  Std.TreeMap.compare_minKey_modify_eq
  Std.TreeMap.compare_minKey!_modify_eq
  Std.TreeMap.compare_minKeyD_modify_eq
  Std.TreeMap.compare_maxKey_modify_eq
  Std.TreeMap.compare_maxKey!_modify_eq

makes it fast again /cc @Paul Reichert

Kim Morrison (Mar 27 2025 at 12:22):

Was just about to report that reverting lean#7679 hasn't helped.

Kim Morrison (Mar 27 2025 at 12:23):

Oops, metavariables in the head of the LHS, that'll do it. Past time for the linter...

Paul Reichert (Mar 27 2025 at 12:45):

Thanks for the hint and sorry, I'll create a PR to remove these simps and will come up with a PR in a few minutes. Perhaps I'll need to find a good way to state these such that they have a better discrimination pattern (perhaps by providing separate Ord-based lemmas).

Paul Reichert (Mar 27 2025 at 13:01):

Update: It's https://github.com/leanprover/lean4/pull/7695.

github mathlib4 bot (Mar 27 2025 at 13:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (da234f8458226fa9e16cc2ae348dcdc2b30e87db).
You can git fetch; git checkout nightly-testing and push a fix.

Notification Bot (Mar 27 2025 at 13:27):

A message was moved from this topic to #nightly-testing > 2025-3-27: segfaults in leangz by Mario Carneiro.

github mathlib4 bot (Mar 27 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d6403f93fe8f0ab25df87ce14052b4f9e8c3bd02).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 17:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6068fa5b912ad07be32404d398eca17cc7b31c32).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 18:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6068fa5b912ad07be32404d398eca17cc7b31c32).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 18:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6068fa5b912ad07be32404d398eca17cc7b31c32).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0beb5de959a3105ab2704176357b3022586321e6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f1c3d6132e587183ea9ac44e4c529dfff1e24e36).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 27 2025 at 23:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f1c3d6132e587183ea9ac44e4c529dfff1e24e36).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 28 2025 at 00:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (90f577e8a58c5dfb106c4657e4d34df71dfbe84c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 28 2025 at 02:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (90f577e8a58c5dfb106c4657e4d34df71dfbe84c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 28 2025 at 02:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (90f577e8a58c5dfb106c4657e4d34df71dfbe84c).
You can git fetch; git checkout nightly-testing and push a fix.

Mario Carneiro (Mar 28 2025 at 02:14):

cache success!

Mario Carneiro (Mar 28 2025 at 02:15):

the remaining issues have been left as an exercise for the reader

github mathlib4 bot (Mar 28 2025 at 03:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (96e12f2dcc230d69e167e93a9e12a909887f9c9e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 28 2025 at 06:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (de25915c5fb885ce202ae2914aec995ffb41102a).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Mar 28 2025 at 08:31):

Mario Carneiro said:

the remaining issues have been left as an exercise for the reader

I'm working on those exercises now (-;

Johan Commelin (Mar 28 2025 at 08:39):

Looks like it will be a 1-line fix.

github mathlib4 bot (Mar 28 2025 at 08:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fbcec6386d71e9e7406cb3572b197786bc5b741f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 28 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fbcec6386d71e9e7406cb3572b197786bc5b741f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 28 2025 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fbcec6386d71e9e7406cb3572b197786bc5b741f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Mar 28 2025 at 10:14):

I've just confirmed locally that we can remove all the new maxHeartbeats, now that the bad simp lemmas have been removed, and hopefully nightly-testing should come green soon. :fingers_crossed:

Yaël Dillies (Mar 28 2025 at 10:20):

Does that mean I don't need to look at Chevalley anymore?

Kim Morrison (Mar 28 2025 at 10:51):

Ah, yes, you don't need to look at that anymore! Thanks for asking!

github mathlib4 bot (Mar 28 2025 at 11:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (07234560b588005c159bd00a0e81e7546f924ce4)

github mathlib4 bot (Mar 29 2025 at 04:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8bd5208c5bee1a2aceb7dc0c921a209382b64404).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 29 2025 at 10:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b4e2ffb295eb3110e852499f3318c9ffc0d0271d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 29 2025 at 13:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a1b8d7845467111b2d9206691d54947917deaac9)

github mathlib4 bot (Mar 30 2025 at 10:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ab98a3ffaa98586009f793bbdd18d80d6ecc5d79)

github mathlib4 bot (Mar 31 2025 at 02:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4be83ef567b3cdbe4fe940b36e6ada3d2ffb4410).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 31 2025 at 02:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ab98a3ffaa98586009f793bbdd18d80d6ecc5d79)

github mathlib4 bot (Mar 31 2025 at 10:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ca1ee28af09a31031159dcade8cd94f3a35492f2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 31 2025 at 11:59):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (44a2fd5edc38e4760b008956991d62cb65917977)

github mathlib4 bot (Mar 31 2025 at 13:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c65306321c59fbef0e1fda26a32e66347a0ceef5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 31 2025 at 14:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (44a2fd5edc38e4760b008956991d62cb65917977)

github mathlib4 bot (Mar 31 2025 at 15:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c6cd01be658269b6fd759048bd9758eed9b1e5fa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Mar 31 2025 at 19:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (44a2fd5edc38e4760b008956991d62cb65917977)

github mathlib4 bot (Apr 01 2025 at 09:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5e033aa736bd1620df982693b3bb17f19ffd6c21).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4a16cda1817b69e8bfcc7c97c83361909c3a9ba4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 11:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4e545b9c44359e6c23aa6e7ee9f103da9617715c).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 01 2025 at 11:27):

I'm fairly sure these failures are coming from lean#7762, which unfortunately wasn't tested against Mathlib.

Kim Morrison (Apr 01 2025 at 11:28):

@Sebastian Ullrich, it's late here for me, so I haven't really looked to see if there is an easy fix in @[to_additive] to cope with this. We may have to revert lean#7762, and then try again with tomorrow's nightly as v4.19.0-rc1?

github mathlib4 bot (Apr 01 2025 at 11:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7440afbbbd59b13a3ecc2bacdc67e4cbf8368584).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 12:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (343fba15a3f027f69535af9650a3f19cb75dfc19).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 15:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7c822cd27ad6abd08a0ab8012897468b1e037c61).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 17:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f18d5e7643f61459ce65a745f8faf75a51479cfb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 17:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (388a6d19f8c4b74c27371be43657e9bf7a14119b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 19:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7a941131c430d136257a88f45b13a9fcff282906).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 20:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1e7f890bd4cdc5001302eb24f84e8f53ee997055).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 01 2025 at 22:20):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (aed9d747c0fa0a811af70c98c323f2d54a4e74ac)

Kim Morrison (Apr 01 2025 at 22:23):

Thanks Kyle and Sebastian for the work overnight!

github mathlib4 bot (Apr 01 2025 at 22:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c5de4f36ecce65a95981a34fa3687504674674a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 01 2025 at 22:50):

This was me dealing with merge conflicts...

github mathlib4 bot (Apr 01 2025 at 23:11):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (aed9d747c0fa0a811af70c98c323f2d54a4e74ac)

github mathlib4 bot (Apr 02 2025 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab457a502f6711335814c0f7d4517c71691e4923).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 10:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab457a502f6711335814c0f7d4517c71691e4923).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 10:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (aed9d747c0fa0a811af70c98c323f2d54a4e74ac)

github mathlib4 bot (Apr 02 2025 at 10:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b4fe96d7aa76c0a139cb2940a722c7782962009).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 12:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2d11cab8f878c31c2d4dbda995272f5fcc6be361).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 13:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7a4b93882bf21abd156eee5f6fee2815a5651564).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 16:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c314845010566d6913d1f0422a1c248f59efc97e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 19:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ccb2aeb2b4d6a1fca132003f45050ca740013ea4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 22:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f2a23fd338cc2440cc93cdb3a2422e346924babf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 22:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (858062724f8532d95b7e03e1f724ac4523ba16ce).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 02 2025 at 23:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d66f383244a70111a71e348e40aff03745c4ac02)

github mathlib4 bot (Apr 03 2025 at 00:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ecdddd70b8ae8c08b0dfa7a918598d871f1c44bc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 03 2025 at 01:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d66f383244a70111a71e348e40aff03745c4ac02)

github mathlib4 bot (Apr 03 2025 at 14:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3b689fd4b5bcdb0643e8cc59e6f9368e2fb51840).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 03 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b7e7d34b02961cba8f71180be18cefb670cf046d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 03 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (99717f89ba48894a8d2b102aec4aa6e05bba6833).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 03 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (37f686cf27093bcbde5a9eb2f1519ef730de1828).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 04 2025 at 00:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (81295dfbd8dc35fc1d1f399b7b61dd6cf6e05cb2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 04 2025 at 01:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (81295dfbd8dc35fc1d1f399b7b61dd6cf6e05cb2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 04 2025 at 03:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (81295dfbd8dc35fc1d1f399b7b61dd6cf6e05cb2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 04 2025 at 03:40):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b4d11241f700b09f70f513e2f5ebec8863113059)

github mathlib4 bot (Apr 04 2025 at 07:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3ab550b8004bcb8520bffb0b8e1c8bd2bc94a8f4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 04 2025 at 10:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7e3ec380a557ceb5c51f157aea6f72c3f14bc317)

github mathlib4 bot (Apr 04 2025 at 19:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7508a9e2525fc667fb6c44af1ab9f3e49a364560).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 04 2025 at 21:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (91a7291e877a8ddbb9e95f32875b3470f3ff3dfe).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 05 2025 at 01:37):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7e3ec380a557ceb5c51f157aea6f72c3f14bc317)

github mathlib4 bot (Apr 05 2025 at 09:27):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0cc1f970691e01afdf9d8bb9f8307cd7b6aca12a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 05 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0cc1f970691e01afdf9d8bb9f8307cd7b6aca12a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 05 2025 at 12:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bdc275fd75f9b2cbdada233ee1a5adde99cf16eb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 05 2025 at 15:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (801a63fdcbd7b0164e4c410e4c9ac92092b712bb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 05 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (28f8afefce5a97f78bba2ae08b72fb322ed5b443).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 05 2025 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (895b1f3655a411757b15089a01eeaf8c6d200df8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 06 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (020da59ce271c24bb642a4c5b3646095447927f4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 06 2025 at 06:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0e1917eb24641cebfd8cbfd91c1cf7eee7e1f9d7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 06 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2aa907ab8a1f690d97ef4a00f589d3e8ab1cb2c0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 06 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2aa907ab8a1f690d97ef4a00f589d3e8ab1cb2c0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 06 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (32a0a63fe26b39faa3d1f6055e7f9086095640f9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 06 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3a141dd224751a2343052a30b3e9a563f8d43687).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 06 2025 at 23:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dbd5552b9e1679ba690cc279e32cbaec5b48f171).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 06 2025 at 23:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dbd5552b9e1679ba690cc279e32cbaec5b48f171).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 00:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15b1cdd7990bc6cd7c1cfab6268595090b91fb29).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 07 2025 at 01:37):

Oh dear, lake exe cache get on the current nightly-testing (d4ab2e5cf588ba671ea265bf16ed1b4b2b3e67bf) results in many /Users/kim/.cache/mathlib/57bc8e5d7a5be2fe.ltar: Operation not supported (os error 45) errors.

github mathlib4 bot (Apr 07 2025 at 01:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dadb75c188fcaf0397e9b223a066b87ba735946d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 07 2025 at 01:38):

CI is also failing in the "check the cache" step, although without printing such error messages, just failing with exit code 3.

Kim Morrison (Apr 07 2025 at 03:33):

@Mario Carneiro, @Mac Malone, unless someone has an idea in the meantime, could we use tonight's meeting spot to try to diagnose this?

github mathlib4 bot (Apr 07 2025 at 04:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bdd987365c7adf9adb82a0baa6ac79f05be2777d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 07:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (95556a99a0c8276d46dc33dfa666da6e4d832eca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7874e38f7476c0cb054152aaee30d3555ddf001b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 09:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0b2ee1e4f1b09613f2a001f52648bf14d239b01d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 07 2025 at 12:49):

Kim Morrison said:

Oh dear, lake exe cache get on the current nightly-testing (d4ab2e5cf588ba671ea265bf16ed1b4b2b3e67bf) results in many /Users/kim/.cache/mathlib/57bc8e5d7a5be2fe.ltar: Operation not supported (os error 45) errors.

@Mario Carneiro, I am guessing this is a change to the olean format breaking leangz, although I don't see anything in the recent commits that looks like this.

Might you be able to take a look?

Kim Morrison (Apr 07 2025 at 12:53):

Some of the latest failures (separately from the olean problem) are likely from lean#7824, as its seems we need further noncomputable modifiers.

Mario Carneiro (Apr 07 2025 at 12:54):

That doesn't sound like a olean issue, it sounds like a disk/IO issue. But I will take a look

Kim Morrison (Apr 07 2025 at 12:54):

There's also some breakage from my lean#7847, fortunately apparently contained in already deprecated proofs which are close to being deleted, and I'll just delete a bit early.

github mathlib4 bot (Apr 07 2025 at 12:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0bd203b35e20df4361729d6f6921070cc356e11f).
You can git fetch; git checkout nightly-testing and push a fix.

Mario Carneiro (Apr 07 2025 at 13:12):

I get a different error:

/home/mario/.cache/mathlib/16566a083771a79f.ltar: Permission denied (os error 13)

(repeated a few hundred times)

Mario Carneiro (Apr 07 2025 at 13:16):

running it through strace, I see it is attempting to call mkdir -p /home/lean/actions-runner/_work/mathlib4/mathlib4/.lake/build/lib/lean/Mathlib/Data/SetLike which fails at the point of trying to create the /home/lean directory on my computer

Mario Carneiro (Apr 07 2025 at 13:16):

so apparently these LTAR files have acquired file paths from the GHA runners

Mario Carneiro (Apr 07 2025 at 13:21):

LTAR files contain records of a file path and compressed data for it, with the file path looking like this normally:

./.lake/build/lib/Mathlib/MeasureTheory/Constructions/Polish/Basic.trace

On the newly generated files they look like this:

/home/lean/actions-runner/_work/mathlib4/mathlib4/.lake/build/lib/lean/Mathlib/Data/SetLike/Basic.trace

Kim Morrison (Apr 07 2025 at 13:25):

@Mac Malone, this is your change from lean#7822

Mario Carneiro (Apr 07 2025 at 13:27):

it looks like this will need changes to cache, not leangz

Mario Carneiro (Apr 07 2025 at 13:27):

(or lake)

Mario Carneiro (Apr 07 2025 at 13:31):

there doesn't seem to be a function in FilePath for relativizing an absolute path

Kim Morrison (Apr 07 2025 at 13:37):

@Mac Malone, could you weigh in with your opinion on whether the correct solution is to relativize, or to go back to, in this circumstance, emitting a relative path to begin with (as lake used to)?

Kim Morrison (Apr 07 2025 at 13:38):

If we need a relativization function in FilePath on short notice ... @Henrik Böving, you probably know better than me who is best placed to implement it?

Kim Morrison (Apr 07 2025 at 13:38):

(I'm going to bed now. :-)

Mario Carneiro (Apr 07 2025 at 13:39):

I can write one in cache if needed, the one the runners use can be quite specialized

Mario Carneiro (Apr 07 2025 at 13:39):

i.e. just stripPrefix

Kim Morrison (Apr 07 2025 at 13:39):

That would be lovely as a stopgap, thank you.

Mario Carneiro (Apr 07 2025 at 13:45):

the part which is confusing me is that cache doesn't use lake at all -- there are no Lake.* imports in cache, so I don't see how mac's changes could have propagated to cache

Mario Carneiro (Apr 07 2025 at 13:49):

aha, it's via lake exe - it now sets the LEAN_SRC_PATH to be full of absolute paths instead of relative paths

Mario Carneiro (Apr 07 2025 at 14:05):

pushed a very basic relativization step in cache. It might need a cache refresh though

github mathlib4 bot (Apr 07 2025 at 14:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7548d2a74910571f1d423e85d6d0e803d8f8997f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 15:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (21001c8dd6171db6b4fbfa6b6da749e66ebf009f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 16:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e37082f608ffd1ef0cc7cfe5ba34eb7bec578ca5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 16:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e37082f608ffd1ef0cc7cfe5ba34eb7bec578ca5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5d515d8437cdc1f0ab2f13825c6e768225f99a75).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 19:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (abd344e43d9dffb162c7370488b86c6e8188db0b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 07 2025 at 22:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d2f6311adec2ea11cbeec4f8ca4a959c98620ea1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 08 2025 at 01:20):

Mario Carneiro said:

pushed a very basic relativization step in cache. It might need a cache refresh though

I'm unfortunately still experiencing /Users/kim/.cache/mathlib/1a8bf81714581847.ltar: Operation not supported (os error 45) on running lake exe cache get on nightly-testing, although CI itself seems happy. Can anyone else reproduce?

Mario Carneiro (Apr 08 2025 at 01:23):

confirmed

Mario Carneiro (Apr 08 2025 at 01:30):

fixed better this time

Mario Carneiro (Apr 08 2025 at 01:31):

(missed an edge case which meant that only files in mathlib dependencies were fixed)

github mathlib4 bot (Apr 08 2025 at 02:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b7aab63cacec62673c58dccf1a1e167ecc495f0f)

Mario Carneiro (Apr 08 2025 at 02:40):

and unpacking worked this time too

Johan Commelin (Apr 08 2025 at 03:42):

Hooray! Thanks for your valiant efforts (-;

github mathlib4 bot (Apr 08 2025 at 04:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b7aab63cacec62673c58dccf1a1e167ecc495f0f)

github mathlib4 bot (Apr 08 2025 at 10:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c6bbaddd6b31ff0b28693a7afdd270d05186ca55)

github mathlib4 bot (Apr 09 2025 at 10:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6c7393e439bdc19b55044ff3fd636b969a9a1393).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 09 2025 at 12:38):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (157a68078c492a194022e1d97461507e6ce59c71)

github mathlib4 bot (Apr 10 2025 at 04:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (21a70379f01ce05319d4890a9ead392094c8ba27).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 07:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (89ce5442a7ea1de25a645e07ebcf712ddcabd063).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 08:33):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (157a68078c492a194022e1d97461507e6ce59c71)

github mathlib4 bot (Apr 10 2025 at 08:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b759d2040f9f64e0baf40f45c384630e6f9d2abb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 08:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f87b82356399f67765a092ba1cec3b84dd072db7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 08:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f87b82356399f67765a092ba1cec3b84dd072db7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 10:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6cd6e917ded15d3d8fc11ee3e6d415cb772252e2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 11:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8c16e6e1cc131f0021a9efe1aa5f56046cba612f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 12:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b4367811d208c50064e5d6cbfe20b601e72e675a)

github mathlib4 bot (Apr 10 2025 at 18:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (af8d2825cf30e68f54daf4a93388165015b349eb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (89ff66b3f0763a2b2d3888b48e538faac06983aa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 10 2025 at 23:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b4367811d208c50064e5d6cbfe20b601e72e675a)

github mathlib4 bot (Apr 14 2025 at 08:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (360bf0d2fd4b3f63857df76bdd9b2d0929e5ebe5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 14 2025 at 09:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b247dc2064294f92d05eed8ec10b7105ebad259c).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 14 2025 at 10:40):

One breakage tonight is that I changed the Pow instance on UIntX in lean#7886, and Mathlib/Data/BitVec.lean is broken. My proposal is to delete everything that is broken in this file, without replacement. The material there is only to set up UIntX so it can be used with Mathlib's ring tactic. As far as I am aware there are no users of this besides perhaps @Tobias Grosser's group. It won't be too long before grind and simp in Lean supersede the ring tactic for these users (we hope).

Let's wait to see if Tobias (or someone he asks to look at this) sounds anguished about ring not working with UIntX in the meantime. If so, we can work out who will fix it, and otherwise we'll hope it simply doesn't need fixing.

Kim Morrison (Apr 14 2025 at 10:41):

A problem I don't understand yet is Mathlib/FieldTheory/IsAlgClosed, where several simp lemmas appear to not be firing, and I don't see what change in Lean could explain this.

Kim Morrison (Apr 14 2025 at 10:44):

Another as yet unexplained problem is Mathlib/Analysis/Distribution/SchwartzSpace.lean, where a gcongr call is producing quite different results that previously.

Perhaps here I can ping @Moritz Doll and/or @Sébastien Gouëzel to see if they can see what has changed?

github mathlib4 bot (Apr 14 2025 at 10:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dcefb86ae959b9ea61c7cb7976ce83c3646e3fa8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 14 2025 at 10:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dcefb86ae959b9ea61c7cb7976ce83c3646e3fa8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 14 2025 at 13:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ece17b308fd0bb27dfd7608ad78d9dc3f384adf9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 14 2025 at 16:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5cc5bd99d13e664296018320f964cdb6f2b25a12).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 14 2025 at 19:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7860ff0f071e852af922555e045f9034c97e9221).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 14 2025 at 22:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (791b0c0760b875bc35046948fb593c7f4e9c4a81).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 15 2025 at 01:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d8e8ad3a0fb1dbe7704c23bfe36200bd3f311712).
You can git fetch; git checkout nightly-testing and push a fix.

Tobias Grosser (Apr 15 2025 at 04:09):

@Kim Morrison, thank you for considering me. I am traveling this week, so won't be around to fix this this week. Nothing bad will happen if the ring instance is dropped for now. I can look into this next week and either carry it out-of-mathlib or immediately switch to grind, ...

Tobias Grosser (Apr 15 2025 at 04:09):

Please do not feel blocked on this by me.

Kim Morrison (Apr 15 2025 at 04:33):

Great, thanks Tobias. grind isn't quite ready for you, but we'll make sure things work in time. :-)

Kim Morrison (Apr 15 2025 at 04:34):

Back to the other problems:

The problem in SchwartzSpace.lean is actually due to a change in behaviour in move_mul.

Kim Morrison (Apr 15 2025 at 04:34):

I've annotated the changed goal states, but haven't investigated.

Kim Morrison (Apr 15 2025 at 04:34):

Could I ping @Arthur Paulino and @Damiano Testa to take a look?

Kim Morrison (Apr 15 2025 at 04:35):

(I suspect this may actually reflect a bug where some upstream function has changed behaviour ... we'll see.)

github mathlib4 bot (Apr 15 2025 at 04:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d8e8ad3a0fb1dbe7704c23bfe36200bd3f311712).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Apr 15 2025 at 05:11):

Pushed temporary fixes.

I wrote the rws to fix Mathlib/Analysis/Distribution/SchwartzSpace.lean and left an adaptation note. It's the only #adaptation_note in the file @Arthur Paulino and @Damiano Testa.

Stranger are those failing simpas in Mathlib/Analysis/Normed/Algebra/Spectrum.lean and Mathlib/FieldTheory/IsAlgClosed/Spectrum.lean @Kim Morrison. Moving the using clauses into haves fixes them. I didn't investigate. Random guess: are there some typeclasses that have changed? Potentially there are instances that don't synthesize soon enough with Tactic.elabTerm stx none (mayPostpone := true).

github mathlib4 bot (Apr 15 2025 at 05:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d8e8ad3a0fb1dbe7704c23bfe36200bd3f311712).
You can git fetch; git checkout nightly-testing and push a fix.

Damiano Testa (Apr 15 2025 at 05:24):

I'll take a look at move_mul, but it'll be in a few hours.

github mathlib4 bot (Apr 15 2025 at 05:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7daf90f27b24d887938ccfda31b0ef510ebfe469).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 15 2025 at 07:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (05e06d9e47a29b8eef909151f6ce935f459fb3d7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 15 2025 at 09:09):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (502763ce50606727068031da926036ac415b9944)

Damiano Testa (Apr 15 2025 at 09:44):

I am slowly understanding what happens. There are two (1 + ‖x‖) ^ l in the goal

The first has expr

@HPow.hPow    Lean.Grind.CommRing.toHPow (1 + x) l : 

while the second one has expr

@HPow.hPow    instHPow (1 + x) l : 

and move_mul does not consider them the same. This means that writing move_mul [(_ + ‖_‖) ^ _] matches the first, on the LHS, and moves it, but does not perform the analogous movement for the other one, on the RHS.

However, using move_mul [(_ + ‖_‖) ^ _, (_ + ‖_‖) ^ _] would work: the first matches the LHS factor, the second one matches the RHS factor and they then both move.

github mathlib4 bot (Apr 15 2025 at 10:05):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (502763ce50606727068031da926036ac415b9944)

Damiano Testa (Apr 15 2025 at 11:12):

Here is a #mwe showing the issue (only works in branch#nightly-testing).

import Mathlib.Tactic.MoveAdd
import Mathlib.Algebra.Ring.Basic

example {R} [CommRing R] {z w : R} : z ^ 1 * w = z ^ 1 * w := by
  -- if you comment the next line, then `move_mul` succeeds
  show (HPow.hPow (self := Lean.Grind.CommRing.toHPow)  _ _) * _ = _
  move_mul [z ^ 1]
  rfl

With the show line in, the first power becomes "different" from the second one and move_mul only moves the first match. Without it, both powers are "equal", so move_mul moves both.

Damiano Testa (Apr 15 2025 at 11:13):

What I still need to understand is why the match is not up to defeq, even though move_mul seems to use isDefEq and not exact matching on the expressions.

Arthur Paulino (Apr 15 2025 at 11:41):

So isDefEq is not returning true for entities that are defeq? Or is there still doubt whether those are defeq or not?

(I'm catching up with the thread)

Damiano Testa (Apr 15 2025 at 11:42):

No, I think that there is a bug in move_add: there is a first defeq check which (I assume) does the right thing.

Damiano Testa (Apr 15 2025 at 11:42):

However, later I use exact matching on expressions, but these are now different-but-defeq.

Damiano Testa (Apr 15 2025 at 11:43):

If you are curious, docs#Mathlib.MoveAdd.reorderUsing does exact matching on expressions (it is used later with \alpha being an Expr.

Damiano Testa (Apr 15 2025 at 11:44):

The defeq check is at docs#Mathlib.MoveAdd.pairUp, but the information about this is not propagated to the later "pure" function.

Damiano Testa (Apr 15 2025 at 11:46):

I am tempted to leave the small hack in nightly-testing that uses either the rws that Kyle used, or using the "double" move_mul call and refactor move_mul later, when I can try to do a better job at it.

Arthur Paulino (Apr 15 2025 at 11:48):

Minor thing: there's a typo in the docstring of pairUp

let R := [mkNatLit 0, mkNatLit 0,                                 mkNatLit 1] -- i.e. [0, 1]

Should be

let R := [mkNatLit 0, mkNatLit 0,                                 mkNatLit 1] -- i.e. [0, 0, 1]

Damiano Testa (Apr 15 2025 at 11:49):

Thanks! I picked that up, I also think that the first R in

At the end, it returns the sublist of `R` of the elements that were matched to some element of `R`,

is an L.

Arthur Paulino (Apr 15 2025 at 11:52):

My first impression is that instance resolution is getting in the way. Has anything changed recently on that regard?

Damiano Testa (Apr 15 2025 at 11:53):

On master, the grind stuff is non-existent.

Arthur Paulino (Apr 15 2025 at 12:16):

I'm surprised this is the only failure point of move_mul, considering the hypothesis that its behavior has changed

Kim Morrison (Apr 15 2025 at 12:16):

It's terrible that Lean.Grind.CommRing.toHPow is showing up anywhere, and I'm surprised that it didn't break more!

github mathlib4 bot (Apr 15 2025 at 12:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (091be7a837765bc72eae216dd63b8412fbeece62).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 15 2025 at 13:21):

Okay, reducing the priority of the parent projections for Lean.Grind.CommRing resolves the problem in SchwartzSpace.lean.

Kim Morrison (Apr 15 2025 at 13:22):

and similarly the other adaptation notes for 2025-04-14!

Kim Morrison (Apr 15 2025 at 13:22):

I will get that into the next nightly.

Damiano Testa (Apr 15 2025 at 13:22):

I now wonder whether move_mul should not be "fixed" and act as a check that similar such changes do not happen in the future. :lol:

Damiano Testa (Apr 15 2025 at 13:23):

I am going to delay revamping move_mul for now: although I think that it would probably benefit from a revamp, I do not have the capacity to do it now.

Kim Morrison (Apr 15 2025 at 13:24):

lean#7975

Damiano Testa (Apr 15 2025 at 13:26):

Should the PR come with a test that makes sure that the grind instance is not picked up? Maybe even in mathlib?

github mathlib4 bot (Apr 15 2025 at 13:35):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (502763ce50606727068031da926036ac415b9944)

github mathlib4 bot (Apr 16 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1a64c90d1b3d20cdeabc6fd9900e9cdd9b0a9bbf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 16 2025 at 10:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (908d1720cb6a97f2f9118da71465af28855a3eea)

github mathlib4 bot (Apr 17 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d4fc0372201cb277506d362c74ce239678d648bb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 17 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d4fc0372201cb277506d362c74ce239678d648bb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 17 2025 at 11:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d4fc0372201cb277506d362c74ce239678d648bb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 17 2025 at 11:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6fb295ce6674766a959e9d3cad4daf750bfdf2bf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 17 2025 at 13:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6fb295ce6674766a959e9d3cad4daf750bfdf2bf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 17 2025 at 16:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (446b459fb17e024ec88cdfd27021cd8b177e5e58).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 17 2025 at 19:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (579c35b7ad7fe1b2351c2be08caa6412a02fd1aa).
You can git fetch; git checkout nightly-testing and push a fix.

Bhavik Mehta (Apr 17 2025 at 23:32):

Kim Morrison said:

No, we'll work out how to support this. It's a reasonable use case.

Have there been updates on this? The commented out version has been in master for a little while now

github mathlib4 bot (Apr 18 2025 at 01:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5cffd1624a0c74eed2fb4edf9a760065f09b9f25).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 18 2025 at 04:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5cffd1624a0c74eed2fb4edf9a760065f09b9f25).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 18 2025 at 09:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (535376f6425a5498089d5db02838ef847d3799b5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 18 2025 at 10:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c7e8bc78d14e27f9e33f83c772ee82775ede357e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 18 2025 at 16:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (06187a42401e4125bc9adbe513290e624a7edb72).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 18 2025 at 16:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (06187a42401e4125bc9adbe513290e624a7edb72).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 18 2025 at 19:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (46ea5ea53c733e376d4637d978ffe179c8e6d1de).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 18 2025 at 21:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fc7ec703b36bc6ddf510ff84b58265318091f439).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 19 2025 at 01:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5724abfc5ed6140c8e66fc85ac4d0743135e8775).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 19 2025 at 03:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (323f78124522dbc2f87ecf16bd21c378ff82c462).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 19 2025 at 10:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f8ab29495610ed1f1e7aef5878396a2987609b53).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 19 2025 at 13:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f8ab29495610ed1f1e7aef5878396a2987609b53).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 19 2025 at 15:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0d9eafd4f7a081106570e2e053e8fcc9de5b57b4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 19 2025 at 17:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6a858d8eb60af16817a32cf642a5bc67a2ec52b5).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Apr 19 2025 at 17:28):

There's a problem here. Mathlib.Algebra.CharP.Basic defines

instance (α : Type*) [CommRing α] (n : ) [CharP α n] : Lean.Grind.IsCharP α n

The Grid.IsCharP class has n as an outparam, but CharP does not have n as an outparam, so the synth order checker fails.

I'm turning off the checker for this instance and leaving an adaptation note.

github mathlib4 bot (Apr 19 2025 at 17:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6a858d8eb60af16817a32cf642a5bc67a2ec52b5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 19 2025 at 19:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a97f34f9002eea29dac71f0b294678d702511e2c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 19 2025 at 20:31):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (7e1178d897c64fca384e902ea5298d99491f4e16)

github mathlib4 bot (Apr 20 2025 at 09:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (04cea2442cb64efe013904b87cae551507694c23)

github mathlib4 bot (Apr 21 2025 at 10:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2002920645c1f9223ac9557c2251c7d5f2744a5a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 21 2025 at 13:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9da3d905bbbfbf8acdc5c95aecbe86ae234dfdcc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 21 2025 at 15:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0c3e3bc3f49047238a49c2b40eac6ae65cf03cdc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 21 2025 at 18:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (32998106f5c17a8b3e9ed1142b0fd8d10308d301).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 21 2025 at 23:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (baf884f022743fe2d457d778610456a718bc471f)

github mathlib4 bot (Apr 22 2025 at 08:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15c5f504a7f2bea1cc172e9b925c5263bff6f1e2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 22 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b438301d5c57ed978f64f7d2f0ae865443faf50).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 22 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0205af1a3f3bf24456b24eff09f9027b5336a989).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 22 2025 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c6fb6f0bace9c91471161ad102fa2236081e4be6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 22 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a29b84dc5791a6674cacb955f0b91282e998476f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 22 2025 at 19:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (673d2deeb899c29f763413a77d2a802c3e610eb7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 22 2025 at 20:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (673d2deeb899c29f763413a77d2a802c3e610eb7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 22 2025 at 22:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (04c82c164d0b74dbfe3fcd0d7e174938d1112399).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 23 2025 at 01:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a5abec925c22ff12ab61d8c9f42d443ce6ee8008).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 23 2025 at 07:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (80bf3eaeb13d9d6f55b62656b60c8c24be15a55c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 23 2025 at 10:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4790a8f38cb6c3851e047216eb5274d1584d5919).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 23 2025 at 11:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b3692fdf0b4e4ac8d6d2355d52ea0c97640b863d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 23 2025 at 12:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e218a97a46ace3af6eaee464e89926011811242f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 23 2025 at 15:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (deb75d65c1b697b286e4c4d7871e618a720ba0bb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 23 2025 at 18:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5eed989e6db5c84e7df50fff5efaf55aea0b8b93).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 23 2025 at 21:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b000f0cba825173fbea70867165ea6ec82378494).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 24 2025 at 03:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0b45b3cb4ae9ef0d9abc6fe8deabed9b4a509656).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 24 2025 at 06:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a6a1efc4b1e46844f4ac443f6ad575e71017b82b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 24 2025 at 09:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (44efe04055fba9a1387f320d39c6ec9d6a609aa1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 24 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (44efe04055fba9a1387f320d39c6ec9d6a609aa1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 24 2025 at 12:52):

Sorry, these breakages are on me, from Lean.Grind.CommRing changes. I will just comment out these instances until I have a chance to fix them.

github mathlib4 bot (Apr 24 2025 at 13:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3c53374d33845762c7987c8c5f2b09d1fa16ea1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 24 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9062fa84b18ca99b0a1faabab8922de665ea91cc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 24 2025 at 18:54):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (156e74538449f643a8fd5db493849c10ddcdd093).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 24 2025 at 21:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3804f24fdae894f4e2dcac649545982149f3ef85).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 25 2025 at 01:00):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c2e31189d9dc2cd707ba1f07bf3df408d0dc30ed).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 25 2025 at 03:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c2e31189d9dc2cd707ba1f07bf3df408d0dc30ed).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 25 2025 at 06:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (50ab41a8bcfd26dedf33cb74c31229b86dc2b4ef).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 25 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11cedf3d2f9d57a855f824465f347d349d3cd5f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 25 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11cedf3d2f9d57a855f824465f347d349d3cd5f1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 25 2025 at 10:48):

I'm hoping this will come good shortly, apologies for the long time spent broken here...

Kim Morrison (Apr 25 2025 at 10:51):

@Joël Riou, I'm wondering if I could ask you to have a look at a change I had to make in Mathlib.Algebra.Homology.Embedding.Connect, in lemma d_comp_d, where I added the note

    #adaptation_note /-- Prior to nightly-2025-04-25 this was just `simp`. -/
    -- Previously, `simp` would use `d_ofNat`,
    -- but now it uses `Int.natCast_add` and goes in a different direction and gets stuck.
    simp_rw [Int.ofNat_eq_coe, X_ofNat, d_ofNat, HomologicalComplex.d_comp_d]

on branch#nightly-testing.

If you'd have a chance to take a look at this, and investigate if there are additional @[simp] lemmas we can add to restore the correct behaviour, that would be very helpful. (Alternatively, we can investigate why Int.natCast_add it now firing, and try to undo that change.)

I can look into this again next week if no one else has got to it by then.

Bhavik Mehta (Apr 25 2025 at 10:52):

Sebastian Ullrich said:

can we instead (temporarily) ban uses of omega in aesop, e.g. by ignoring this file on nightly-testing?

Is there a tracking issue for this? It seems that omega is banned in aesop now, and the file is ignored in mathlib master. It would be nice to have some idea of when this file is coming back!

Kim Morrison (Apr 25 2025 at 10:53):

This is an question for @Jannis Limperg, right?

github mathlib4 bot (Apr 25 2025 at 11:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aaf7807033ea98abbd591b7bfd0fecb9182eef7d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 25 2025 at 11:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aaf7807033ea98abbd591b7bfd0fecb9182eef7d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 25 2025 at 13:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (aaf7807033ea98abbd591b7bfd0fecb9182eef7d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 25 2025 at 13:21):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b7a687535bfa626b79c5554e6f7e2a6dfd15339a)

Joël Riou (Apr 25 2025 at 15:19):

Kim Morrison said:

Joël Riou, I'm wondering if I could ask you to have a look at a change I had to make in Mathlib.Algebra.Homology.Embedding.Connect, in lemma d_comp_d, where I added the note

I would think that Int.natCast_add is a good simp lemma in general, so that we just need to prevent it being triggered in this particular case. I have pushed a "fix" consisting in squeezing simp? [-Int.natCast_add].

github mathlib4 bot (Apr 25 2025 at 15:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b7a687535bfa626b79c5554e6f7e2a6dfd15339a)

github mathlib4 bot (Apr 26 2025 at 09:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a91fc5caa16bc82b9ba3eeb55ba4268223553f17).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 26 2025 at 11:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a0dbca2092519754c44c7409a9988b943cbb9ee3).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Apr 26 2025 at 14:17):

Almost there in lean#8114! @Kim Morrison I think we can wait for the next nightly but I'm curious - would there be any negative consequences of bumping nightly-testing to a PR release?

github mathlib4 bot (Apr 26 2025 at 14:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a0dbca2092519754c44c7409a9988b943cbb9ee3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 26 2025 at 15:34):

Sebastian Ullrich said:

Almost there in lean#8114! Kim Morrison I think we can wait for the next nightly but I'm curious - would there be any negative consequences of bumping nightly-testing to a PR release?

We've done it occasionally, it should work, and CI will clobber the toolchain tomorrow.

github mathlib4 bot (Apr 26 2025 at 16:53):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (637398a215a1ec7aadc4de0138c5bd4527296279)

Sebastian Ullrich (Apr 26 2025 at 17:53):

Indeed, only the discover-lean-pr-testing check yelled at me :) .

I'm not quite sure yet whether my deprecation of ConstantInfo.isTheorem, or its attached message, is appropriate. In core, all of its users really cared about whether the constant was originally declared as a theorem, thus the deprecation message. But here the two users really only cared about what constructor it was at that point in time, so I changed them to direct matches.

github mathlib4 bot (Apr 26 2025 at 18:47):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (637398a215a1ec7aadc4de0138c5bd4527296279)

github mathlib4 bot (Apr 27 2025 at 09:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (44f760b7eedc79bdbd0aade893d545d16a2c58cf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 27 2025 at 12:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (44f760b7eedc79bdbd0aade893d545d16a2c58cf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 27 2025 at 13:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (44f760b7eedc79bdbd0aade893d545d16a2c58cf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 27 2025 at 16:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a569d4850c7a997eb018903d0f4d3d27589b7b77).
You can git fetch; git checkout nightly-testing and push a fix.

Bhavik Mehta (Apr 27 2025 at 16:31):

Kim Morrison said:

This is an question for Jannis Limperg, right?

The discussion here #lean4 > aesop and bv_decide @ 💬 suggests that it's a problem with replay, rather than with aesop

Ruben Van de Velde (Apr 27 2025 at 18:42):

Quick r? #24417

Kim Morrison (Apr 27 2025 at 18:54):

Bhavik Mehta said:

Kim Morrison said:

This is an question for Jannis Limperg, right?

The discussion here #lean4 > aesop and bv_decide @ 💬 suggests that it's a problem with replay, rather than with aesop

@Jannis Limperg, do you know what change is needed? Ideally aesop would just take over whatever replay functionality it needs.

github mathlib4 bot (Apr 27 2025 at 19:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (04fc112dc64638d572c795b5515dbc1eeadc1e29).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 27 2025 at 21:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (26e8de2dfae04438c9cd6da1fa9df74d89f70e6b)

github mathlib4 bot (Apr 27 2025 at 22:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fed914b4469dc74c7ff6cf8e3a681a38a1b5e672).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 28 2025 at 00:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b8e91f6731db01e801d19a5c068fad31a64d38b5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 28 2025 at 03:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (70fb092b5fbe862f4116a3a722a128228328ba4b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 28 2025 at 07:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f77211db8b7a134d5eaa8131e63fab3ff0e80a70).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 28 2025 at 07:40):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (26e8de2dfae04438c9cd6da1fa9df74d89f70e6b)

github mathlib4 bot (Apr 28 2025 at 09:48):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (91ba50b9ac2717983d780a776d2a36d7eb989509)

github mathlib4 bot (Apr 28 2025 at 19:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (12e7ef97c27845977c4f82e86db3e93dd851f71b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 28 2025 at 20:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab000e4c8ffacfdc42e08b5467fb89c7d6888184).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 28 2025 at 22:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ab000e4c8ffacfdc42e08b5467fb89c7d6888184).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 28 2025 at 22:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (91ba50b9ac2717983d780a776d2a36d7eb989509)

github mathlib4 bot (Apr 29 2025 at 09:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (072b045dc0d12adc22df3d516bba40d3990db0ce).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 29 2025 at 09:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c00c2f88f546a022ea12486c0a890110c0b5a7f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 29 2025 at 12:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (61ea3c01210efd193bb5a6a71be4a75cc956b797).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Apr 29 2025 at 13:25):

Looks like someone has already fixed this one, thanks. :-)

Johan Commelin (Apr 29 2025 at 13:30):

I'm working on it

Ruben Van de Velde (Apr 29 2025 at 13:41):

Another quick review at #24449

Johan Commelin (Apr 29 2025 at 13:42):

@Ruben Van de Velde can you please explain the reason for that PR?

Johan Commelin (Apr 29 2025 at 13:43):

Are these changes that are backported from bump/v4.20.0?

Ruben Van de Velde (Apr 29 2025 at 13:46):

From nightly-testing, but same thing, yeah

Johan Commelin (Apr 29 2025 at 13:48):

But these change are already being reviewed when they get merged into bump/v4.20.0 through the adaptation PRs. So, while I appreciate the effort, I don't think it's really necessary.

github mathlib4 bot (Apr 29 2025 at 14:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (61ea3c01210efd193bb5a6a71be4a75cc956b797).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Apr 29 2025 at 14:50):

I think it's beneficial to limit the monthly bump PR to just the changes that need to happen all at once, otherwise you get massive commits on master

Johan Commelin (Apr 29 2025 at 14:52):

That's true.

Johan Commelin (Apr 29 2025 at 14:53):

In that case. Is there a way to auto-generate PRs like yours?

Johan Commelin (Apr 29 2025 at 14:53):

And independently, to ask git whether the patch is contained in stuff that has already been reviewed, to avoid double-reviewing?

Johan Commelin (Apr 29 2025 at 15:01):

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (61ea3c01210efd193bb5a6a71be4a75cc956b797).
You can git fetch; git checkout nightly-testing and push a fix.

I'm confused. Locally it builds, tests, and lints fine...

Johan Commelin (Apr 29 2025 at 15:02):

Never mind, the issue is shake

Johan Commelin (Apr 29 2025 at 15:04):

$ lake exe shake --fix
The following changes will be made automatically:
/home/jmc/repos/nightly-testing-bumps/Mathlib/Data/Stream/Init.lean:
  remove #[Mathlib.Data.List.Defs]
Successfully applied 1 suggestions.

except... no? The import is still there.

Removed it manually.

github mathlib4 bot (Apr 29 2025 at 15:16):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (5afdea540abf6226b130896e2c1ae3e06de1c3bb)

github mathlib4 bot (Apr 30 2025 at 09:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (819ba93940a13dad156bbb33138035f9e763aab0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 30 2025 at 12:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d31099deb6401127888aa31e2724ba8594769f18).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 30 2025 at 13:43):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4dd235e6045ca31c51dace4dcff464a16170359c)

github mathlib4 bot (Apr 30 2025 at 19:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2c6431a7fae9ba16e92fefbebd3648bdeb0bb5c3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Apr 30 2025 at 21:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3f501c89f185e585c5be27b36857b9cbd7bdde88).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 01 2025 at 00:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ffa0da468b56742dac6d108dff59ad4ee1ddfc6a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 01 2025 at 04:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9bd9792ac67f684040ebb58a609f48f10ff10bc6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 01 2025 at 06:59):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (4dd235e6045ca31c51dace4dcff464a16170359c)

github mathlib4 bot (May 01 2025 at 10:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (429a671bb6b2694fe09ad32e728a85df69a542d9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 01 2025 at 13:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f4adaa2f478c30c5f520e2571a2b668f6c6f592e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 01 2025 at 16:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d21cb887c766740060152de7c03960739c851ed7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 01 2025 at 16:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (701d7503190076933232fbffd40efc333cae8490)

github mathlib4 bot (May 02 2025 at 09:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (9609f78734850b7dd8482688323908633e77fa4a)

github mathlib4 bot (May 03 2025 at 10:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (af3f7e59787eba900eb6489ddf6631eb87099d3f)

github mathlib4 bot (May 04 2025 at 08:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cf60aac646306fe4e74f6d112edc8754cf50927a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 04 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9c5455a132e91d6101121aa2e7a1342862352dda).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 04 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ce872d984ce45ccb7baddd49a913fd450733a709).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 04 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (529c13b5da1ff47aef41dbebd4d004fdf353aaf7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 05 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (03bc870a1a65cfea41eecb05a8599288a601629b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 05 2025 at 06:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (19855c0801d3dfaf2874823db6190d43df6cb4f9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 05 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a3652388e0853e5215b14d437feff567f9258f8e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 05 2025 at 09:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a3652388e0853e5215b14d437feff567f9258f8e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 05 2025 at 12:29):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dafa7119eaad16a20c041afb508c337464b6b316)

github mathlib4 bot (May 05 2025 at 21:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6870b869fd0a1a4bb0334893dd78183c76580b83).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 06 2025 at 04:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dafa7119eaad16a20c041afb508c337464b6b316)

github mathlib4 bot (May 06 2025 at 10:05):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a19d1649383d65a9c4aa006b1f896f003c61a160)

github mathlib4 bot (May 06 2025 at 10:05):

:warning: Warning: The lean-toolchain file in the latest bump branch does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.
Current content:
This needs to be fixed for the nightly testing process to work correctly.

Damiano Testa (May 06 2025 at 11:27):

:warning: exotic message!

github mathlib4 bot (May 06 2025 at 13:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a19d1649383d65a9c4aa006b1f896f003c61a160)

github mathlib4 bot (May 06 2025 at 13:34):

:warning: Warning: The lean-toolchain file in the latest bump branch does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.
Current content:
This needs to be fixed for the nightly testing process to work correctly.

Kim Morrison (May 06 2025 at 13:52):

Strange message, because it's false...

Kim Morrison (May 06 2025 at 13:53):

(But we are exploring a corner of CI that has never successfully run before, so I guess this is to be expected.)

Kim Morrison (May 06 2025 at 13:57):

Let's see if #24635 helps.

github mathlib4 bot (May 06 2025 at 16:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a19d1649383d65a9c4aa006b1f896f003c61a160)

github mathlib4 bot (May 06 2025 at 16:28):

:warning: Warning: The lean-toolchain file in the latest bump branch does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.
Current content:
This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (May 06 2025 at 19:04):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a19d1649383d65a9c4aa006b1f896f003c61a160)

github mathlib4 bot (May 07 2025 at 10:27):

:warning: Warning: The lean-toolchain file in the latest bump branch does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.
Current content:
This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (May 07 2025 at 13:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (aa0e73cf2d3ddd03282752c311ea8ff9771f6bc0)

github mathlib4 bot (May 08 2025 at 09:49):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (d892bde274dc0b200161339bc4fb901f7e1be0d1)

github mathlib4 bot (May 09 2025 at 10:26):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (33217e9878a8466b793bad6b09c35070fb55741a)

github mathlib4 bot (May 10 2025 at 09:55):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (dd0898a0fb2ffee28c2dac88edad44a1c10d0116)

github mathlib4 bot (May 11 2025 at 10:12):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (8869f89d6f5b19b3c41bdbcaaac5d38c06434caa)

github mathlib4 bot (May 12 2025 at 10:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (c3e0c0c39b94e1825953e547abef20a534faf46e)

github mathlib4 bot (May 13 2025 at 10:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f167e8ddbde220d1a70abd905821e6bf83828935).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 13 2025 at 11:51):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f167e8ddbde220d1a70abd905821e6bf83828935).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 13 2025 at 12:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b9ded787281c489758b033d759e03098a786b1af).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 13 2025 at 13:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b3c5820c69d5c33c515f20d76e34874e5f742020).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 13 2025 at 16:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (33308ffdc0dc62f1437e76c5ce0857f52b7b3bfa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 13 2025 at 19:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e9db98beeec1b415e419a3a8f0d96ed55b0f29ab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 13 2025 at 21:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (87a50461a7f908301812ff4292c6826365e458c0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 13 2025 at 22:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (da11a5fe442e11ece25a34f3aef63411fdf7e64a)

github mathlib4 bot (May 14 2025 at 08:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c53aaa6730188e4f26ead9ab05029673b3fcea3b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 14 2025 at 10:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bdbaaec4586199137d0c4b8de97c1ececfb8f05d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (May 14 2025 at 11:10):

Ouch:

error: /Users/kim/projects/lean/mathlib4/Mathlib.lean:1:0:
import Batteries.Data.String.Lemmas failed,
environment already contains 'String.instTransOrd' from Std.Classes.Ord.String

Kim Morrison (May 14 2025 at 11:46):

(I fixed this by simply importing Std.Classes.Ord.String in Batteries.Data.String.Lemmas, to ensure that Lean could see the potential for conflict and automatically choose better names.)

github mathlib4 bot (May 14 2025 at 12:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f55ac5ea0e76acb6f46d12182c7008f46995c424).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 14 2025 at 12:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (624a35316bda9df5ef3649d2fbf2c975f51124cf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 14 2025 at 13:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (88c664917b2ae535a983bff73d77c23e3d667f8c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 14 2025 at 16:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c61b9b01b5cb518d61dfd95afe1253bd92a147ad).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 14 2025 at 19:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (73a7031ff90f2cee74ed18883bba867790593600).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 14 2025 at 22:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (909e37908d7a2df03f0d43c5d9e9dda31bbf6cd3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 15 2025 at 01:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d6c3a2d285e461d43a0bed7d7a2aa51fce4de3d9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 15 2025 at 07:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4009f934785d750afe7a58f05496bf7c5227b4a2).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (May 15 2025 at 07:26):

I already fixed that! (shake --fix) Not sure what went wrong, trying again

Ruben Van de Velde (May 15 2025 at 07:27):

Maybe https://github.com/leanprover-community/mathlib4/issues/24743?

Kim Morrison (May 15 2025 at 07:28):

@Mario Carneiro, the fix for this is in your #24807, which is marked awaiting-author. Will you have a chance to look soon? If not we'll just merge anyway, I guess.

github mathlib4 bot (May 15 2025 at 08:00):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ca03b453d5de520856682af67fa7afbdfca8ea17)

github mathlib4 bot (May 15 2025 at 09:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (590a7b8322f33874b3b570bc1f2dc09f92c11d2b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 15 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (590a7b8322f33874b3b570bc1f2dc09f92c11d2b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 15 2025 at 09:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (58bea692477a193f887dc52f966400f66c14d0b0).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (May 15 2025 at 10:14):

Hmm, I seem to have broken something badly by moving the notation class Inv up to the Lean repository in lean#8345.

Kim Morrison (May 15 2025 at 10:15):

We're now getting lots of errors like

(-1 + u⁻¹ : R) -- failed to synthesize Inv R

for u : Rˣ.

Kim Morrison (May 15 2025 at 10:15):

@Kyle Miller, perhaps you have a hint?

Kim Morrison (May 15 2025 at 10:18):

Ah, maybe I see a whitespace typo that may have broken the unop% elaboration helper.

github mathlib4 bot (May 15 2025 at 10:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9e7d035eaa9148e5aa81d80aabcf12c1c1b84004).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (May 15 2025 at 11:04):

Ah, sorted. One must not use unop% for Inv.inv!

I'll move nightly-testing over to the lean-pr-testing-8351 toolchain shortly.

Kim Morrison (May 15 2025 at 11:19):

There were also quite a few changes that had accumulated that were incompatible (i.e. had superfluous dsimps) with Jovan's recent changes. Probably we will have some more of these before the end of the month.

github mathlib4 bot (May 15 2025 at 11:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (951d0a1e08447c2fe2f4d5062837c2428ded4fc6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 15 2025 at 12:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (125bc590062e108313bdc113f8d6341664bd4d11).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 15 2025 at 13:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (de9c99925b9978fe63320cdf17e99000f347bdff).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (May 15 2025 at 13:22):

Ah, okay, the bot sets the toolchain back to nightly automatically. This will remain broken until tomorrow.

github mathlib4 bot (May 15 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f3d9e0c630b3de5bb65b2a87074e440677fa8d48).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 15 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2ddde4f3126db03aeeff243a6a2fae1e0f0ea698).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (May 15 2025 at 18:51):

Kim Morrison said:

Ah, sorted. One must not use unop% for Inv.inv!

That's unfortunate... Is using Inv.inv in this heterogenous way the most common? Not adding unop% means types in arithmetic expressions won't be able to propagate through Inv.inv in the same way as other arithmetic operations.

Using the unop% helper, you'd have to write (-1 + (u⁻¹ : Rˣ) : R) (maybe (-1 + (u⁻¹ :) : R) works too). Not very pleasant.

github mathlib4 bot (May 15 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4551f5664b69a6e16aaad2ade073c9c0cd1b8639).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 16 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7e5e1e6ae45b5aa96299cf330b2df9016b4c542a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 16 2025 at 03:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c4a97f5f275b2d5e70c42bd711299840cb192c36).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 16 2025 at 06:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (64f23d2ee4fa8bd912b4450c2e9691e80e0a7222).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 16 2025 at 09:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (52e9c62bb1c948ac7d8c8c23f21ef9fa7e775c41).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 16 2025 at 10:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4d4b317a9ccafdb62206c78711b29d43bccf7ea3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 16 2025 at 11:14):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (00be6377c3a1cfd3d70f6b2d3b18409bafbc8f7e)

github mathlib4 bot (May 17 2025 at 09:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (49a23c600d5abe180e30a5c6fed3cc708b7e1de2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 17 2025 at 11:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (77454ed02f4703ee3f9fb9c57d7554501ffd605b)

github mathlib4 bot (May 19 2025 at 10:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f27355c1aed94df0bcbaf74b72d86c1daebfda6e)

github mathlib4 bot (May 19 2025 at 11:08):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (19337f2bd8ff53570f7b5095f6d8b4ea9f724b8f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 19 2025 at 13:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (82b03c0d5781998b03f097733b384f711d03fffa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 19 2025 at 13:50):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (f27355c1aed94df0bcbaf74b72d86c1daebfda6e)

github mathlib4 bot (May 20 2025 at 08:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a91df8da4ca1c8e0a80c0807f2c1e8a9ea9011e2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 20 2025 at 13:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a228b7f6ef14afc0fbaabcbd70945f65a7fcd6ef).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 20 2025 at 15:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0d2d0d7c62b4aa30ac89a4ce98117733a5e0fa65).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 20 2025 at 18:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2193fd84b62b242dbeea388727568c3d23e5e251).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 20 2025 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9564192722ac6bcb396a8ef68f176092b87b0e10).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 00:09):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (83f3832c6cfeecbc8d16b0248c98346956a7f0e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 00:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (83f3832c6cfeecbc8d16b0248c98346956a7f0e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 00:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (83f3832c6cfeecbc8d16b0248c98346956a7f0e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 01:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (83f3832c6cfeecbc8d16b0248c98346956a7f0e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 02:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (83f3832c6cfeecbc8d16b0248c98346956a7f0e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 02:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (83f3832c6cfeecbc8d16b0248c98346956a7f0e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 06:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (83f3832c6cfeecbc8d16b0248c98346956a7f0e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 07:49):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (6f0aafa2a2f76b744f66db7ae846ceaee38974e5)

github mathlib4 bot (May 21 2025 at 10:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4f17adebb3ea7e6d095ded0d8897bd5a47bfe07d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 21 2025 at 11:11):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (136d4927370922d50f5b36654f71eec43784c6c5)

github mathlib4 bot (May 22 2025 at 08:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (69245187dc435125749c5cc16759da1508b6e0af).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 22 2025 at 10:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (136d4927370922d50f5b36654f71eec43784c6c5)

github mathlib4 bot (May 22 2025 at 12:17):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b1993479392f304ab4e33947612d512d43b90d2d)

github mathlib4 bot (May 22 2025 at 16:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (537a98e0c053976429d5fe61d843c5c8ac2c892e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 22 2025 at 18:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f34c1f584077f008f706f4fa12fc8881ad722e31).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 22 2025 at 21:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3ee28f8c6f81ffe85729e2c3c62656b11b45aa85).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 22 2025 at 23:50):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b1993479392f304ab4e33947612d512d43b90d2d)

github mathlib4 bot (May 23 2025 at 09:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (484320504fe5f8b2ff564b8ca8319a43d4695b2b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 23 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (484320504fe5f8b2ff564b8ca8319a43d4695b2b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 23 2025 at 12:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3ffff9ede0b0dcb00ff651e58baa0754c0968dcc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 23 2025 at 15:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4db29a97d5f4c276a1a883ccbcd44113e3070c2b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 23 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (06d29195366303f117ff51400f7544b1cfeec3d0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 24 2025 at 00:53):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (de0f1e8317fc7bb31981dfc149f13b739253f09a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 24 2025 at 03:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (30ae5addc4aba5803b38de4777e03f3a720a9dea).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 24 2025 at 10:44):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d4d6fed9ec6df46db12fbc9ebed2d86ab66fbf29).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 24 2025 at 11:04):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (1db1f04b7a88cd75102b70ac6befc4b18d08727c)

github mathlib4 bot (May 25 2025 at 10:04):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (e8511a836bcc06fe4f35d6b5eae5770cf0a06e60)

github mathlib4 bot (May 26 2025 at 12:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8386af85095c985aa33ed448aa9890a40cc5fa00).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 26 2025 at 13:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2f24c6a54108fa0a30015d289b78f7de11931b8e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 26 2025 at 16:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (cdf00c3262877ba8a9c34e58215d2a31dee64adb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 26 2025 at 19:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1671a6800555ca3012b379b59af87b2d0e23750c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 26 2025 at 21:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (61de43dfb330ba44bc6ac5603a46cedc2583b583).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 26 2025 at 23:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (78204fd6d53e7401f71e97facae181abcef6c875)

github mathlib4 bot (May 27 2025 at 09:23):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1f5342720a7869e4ff8c2f890acad3818fefc82c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 27 2025 at 10:24):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (fafc2d8bb4f2384bc2852e88e420e6d041b596c3)

github mathlib4 bot (May 28 2025 at 09:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (97bc5f6d896e1593618d0b57beca4f9de618a50b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 28 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (97bc5f6d896e1593618d0b57beca4f9de618a50b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 28 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b7922f25621402041cfbf49370324e43d5366d2f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 28 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fc190a53670152feca8698a35180a7d4bc08de07).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 28 2025 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a8e1f8267d4cbabac2f3ec3efd0611eabf8d0fbe).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 28 2025 at 21:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (282cd80104881fe7981f70f2482bf3a2d1ee93b3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 29 2025 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b5423b71cf1e1bd16c3668e70af3f1568f5dc221).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 29 2025 at 05:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a8f4f9af9a747169f9bf2a10c29894bc29c8af64).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 29 2025 at 05:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a8f4f9af9a747169f9bf2a10c29894bc29c8af64).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 29 2025 at 06:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a8f4f9af9a747169f9bf2a10c29894bc29c8af64).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (May 29 2025 at 09:18):

@Michael Rothgang, @Anne Baanen would you be available to look at this failing test?

It is an interaction between the directory dependence linter and the new linterOption framework.

Anne Baanen (May 29 2025 at 09:19):

Ok, I'll take a look.

Kim Morrison (May 29 2025 at 09:20):

I've just pushed 3a34736f599 which temporarily comments out the failing test, as I would like to ensure we get to green for Lean testing purposes before the weekend.

Kim Morrison (May 29 2025 at 09:20):

But this commit can be reverted.

Anne Baanen (May 29 2025 at 09:33):

Fixed! The header linter checks whether it's running in Mathlib or a test file, and disables itself otherwise, but did not recognize the test file. Not sure why that isn't an issue on the master branch.

github mathlib4 bot (May 29 2025 at 09:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (3a34736f5995ef991ce09ffd0439fe995f49f7dc)

Anne Baanen (May 29 2025 at 09:40):

Ah, seems a merge went wrong. Copied over the exact code now, which should do exactly the same thing.

github mathlib4 bot (May 29 2025 at 11:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e88e619b06606c36e542cefe2af9b382112a0348).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 29 2025 at 13:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2b2788e7a1259d491770fb9660b58375774f816c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 29 2025 at 16:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ec35a548acb922c0093155ec2d73d1e618454872).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 29 2025 at 19:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (520939fab5fa0944e628b5f3870b23cda61639d5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 29 2025 at 22:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1a9b964b92509b9a757fd24bae6b6b9812443163).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 30 2025 at 00:30):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (59c607936721f4ccb5c7c3cd3ca9f6039a6d82be)

github mathlib4 bot (May 30 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1a9b964b92509b9a757fd24bae6b6b9812443163).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 30 2025 at 13:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (00898110647ec3168fdea4081af13d2621a95354).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 30 2025 at 15:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4459088658417ad4ec82b194da3184cbe638b7e0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 31 2025 at 09:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3f45597c0f418ed651130f877e2a89186ea3abcc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 31 2025 at 13:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bc40dcfb1a99949bd4985ec93613f008124148a5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (May 31 2025 at 19:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9265da5cb8f95b4210a510f861fe8a6cdb16bb16).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 01 2025 at 01:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (644a2302b0210c65cac2ba7497eba7f90a3cb803).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 01 2025 at 04:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6ea68a87c1a3887fc0a9150cec021206d5a0d024).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 01 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6ea68a87c1a3887fc0a9150cec021206d5a0d024).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 01 2025 at 16:17):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7aca00c01d2ab15e53c9a04ae59200aca42b80d2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 01 2025 at 22:04):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a3cf05e12e284f915874efc4a0131c41a6e23532).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 02 2025 at 00:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ac7d8cf03db685fb9230d273bbe09ace3cc370df).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 02 2025 at 04:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1414404d0a57f58a3cd748ac7b9060349b37dfbc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 02 2025 at 06:56):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a55b97615cc094e3aa31a004f9069130f269daae).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 02 2025 at 07:13):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (347b2efa08a0a3cefd676315c3bdb64cf11fbe3c)

github mathlib4 bot (Jun 02 2025 at 10:23):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (59d029368a02341d0ddb123a1d9f5a4d6737935c)

github mathlib4 bot (Jun 03 2025 at 08:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bdc2b05443e4b288467636946059666bc4eef292).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 03 2025 at 10:27):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (595ac3cad016af3480984a4f0972e1808a3a8bc5)

github mathlib4 bot (Jun 04 2025 at 09:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d1cba2e8f07d95dbae8fb527d66769ba28c68ee3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 04 2025 at 09:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d1cba2e8f07d95dbae8fb527d66769ba28c68ee3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 04 2025 at 10:17):

Looks like we need a ProofWidgets patch for lean#8105.

Kim Morrison (Jun 04 2025 at 10:21):

Done in v0.0.63-pre.

Kim Morrison (Jun 04 2025 at 10:23):

Does anyone know why to_additive is broken on nightly-testing?

Kim Morrison (Jun 04 2025 at 10:34):

lean#8584 was the answer. Unfortunately the bot didn't automatically merge, or even report, lean-pr-testing-8584, but that's done now.

github mathlib4 bot (Jun 04 2025 at 11:21):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (03daea22daa097731dd0f3d8f870e36086671b88)

Sebastian Ullrich (Jun 04 2025 at 14:35):

Kim Morrison said:

lean#8584 was the answer. Unfortunately the bot didn't automatically merge, or even report, lean-pr-testing-8584, but that's done now.

My bad, that's likely because I pushed it directly to master. Unfortunately there is still this GitHub bug that prevents us from merging these PRs ourselves but I'm planning to ask someone else next time.

github mathlib4 bot (Jun 04 2025 at 16:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (a0370507e2922f0a329a2d8cc17e9f9148cd168d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 04 2025 at 16:39):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (03daea22daa097731dd0f3d8f870e36086671b88)

github mathlib4 bot (Jun 05 2025 at 07:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b71e8543f488392e9cac2e5fef9511f787562a1f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 05 2025 at 09:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d2867d7b07c7f3edf4dd93cba6d7499615267a6f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 05 2025 at 10:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c7f51d87683fe8f4567263bab492016c5ff4b54e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 05 2025 at 11:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c7f51d87683fe8f4567263bab492016c5ff4b54e).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 05 2025 at 11:06):

Merged batteries-pr-testing-1220

github mathlib4 bot (Jun 05 2025 at 11:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c7f51d87683fe8f4567263bab492016c5ff4b54e).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 05 2025 at 11:47):

@Mario Carneiro:

info: Shake/Main.lean:644:0: #[Name.anonymous]
error: Shake/Main.lean:643:0: ❌️ Docstring on `#guard_msgs` does not match generated message:

info: #[Name.anonymous]
error: Lean exited with code 1
Some required builds logged failures:
- Shake.Main
error: build failed

Kim Morrison (Jun 05 2025 at 11:49):

Kim Morrison said:

Merged batteries-pr-testing-1220

I've reverted this, as it needs further review. Let's get #25478 in master asap, and then that will flow into nightly-testing.

github mathlib4 bot (Jun 05 2025 at 11:55):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0a7d1791fb0a41960ca4624a38f492896c5941ac).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jun 05 2025 at 12:16):

Is that meta fallout on Shake? Any idea why it succeeded on the PR itself?

Sebastian Ullrich (Jun 05 2025 at 12:23):

Upgraded to syntax quotation. I did not allow for module system modifiers yet as it's unlikely Shake will do something sensible with them without further changes.

github mathlib4 bot (Jun 05 2025 at 12:29):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7d5bdba1cb8d07d9818165c7be4509ab757ad7f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 05 2025 at 13:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7d5bdba1cb8d07d9818165c7be4509ab757ad7f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 05 2025 at 14:47):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (673dbbdb126ec2f903efa5baec90a60b50b10a30)

Mario Carneiro (Jun 05 2025 at 23:08):

Sebastian Ullrich said:

Is that meta fallout on Shake? Any idea why it succeeded on the PR itself?

As foretold: #general > lake exe shake --fix is broken @ 💬

Mario Carneiro (Jun 05 2025 at 23:11):

As to why it succeeded: it didn't. So the question is why this failed build is reported as a success here

github mathlib4 bot (Jun 05 2025 at 23:34):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (673dbbdb126ec2f903efa5baec90a60b50b10a30)

github mathlib4 bot (Jun 06 2025 at 04:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (05d5f260d39c47f48e3618aefa768ccfb9a88465).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 06 2025 at 05:38):

This is failing, I think, as a side effect of our recent deployment of landrun.

Kim Morrison (Jun 06 2025 at 05:38):

Unfortunately, I won't be able to fix this until Monday, so if anyone would like to investigate that would be great.

Kim Morrison (Jun 06 2025 at 05:40):

The actual error is:

https://github.com/leanprover-community/mathlib4/actions/runs/15482344387/job/43590344569#step:17:13

so almost surely we are just running with the wrong toolchain when CI is handling nightly-testing.

Kim Morrison (Jun 06 2025 at 05:40):

Oh!

Kim Morrison (Jun 06 2025 at 05:41):

We are running mk_all from the master branch, against files on nightly-testing...

Kim Morrison (Jun 06 2025 at 05:43):

@Johan Commelin, what do you think? I think we're going to have to set up a lower security CI setup for nightly-testing, that just runs the scripts from nightly-testing itself.

I think we're going to have a similar issue for any version bumps on master too. We're going to have to have a separate CI process that simply uses the branch's scripts.

Kim Morrison (Jun 06 2025 at 05:43):

More if statements in mk_build_yml.sh?

github mathlib4 bot (Jun 06 2025 at 07:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (480a4cbf195d7ce802babd92cffe1f626a567588).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 06 2025 at 10:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (57ed0a13e76418c4b9322b3e23c5f3d5cd9e8445).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 06 2025 at 13:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fda802e34e3e8ff584b5c38764679611c606ccef).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 06 2025 at 15:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (742c6cc0769cf57b985f7cd7970bbb687eb002a7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 06 2025 at 18:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (48cebe313b2cc4203ff3f01ccaa171dc6197a528).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 06 2025 at 21:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2b5cc7dbf7b9acc716eb70f1fc593f77ffc5c984).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 07 2025 at 01:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (abbdd1252138b5a815e9bbc91df8c31c37f5928b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 07 2025 at 03:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (994033ef9c4b418ad19747aa3589495b60728067).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Jun 07 2025 at 08:39):

Kim Morrison said:

We are running mk_all from the master branch, against files on nightly-testing...

Sorry... why is that an issue?

github mathlib4 bot (Jun 07 2025 at 09:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bd7f0d6243fa265cd3251a5046111248e07ed421).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 07 2025 at 09:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bd7f0d6243fa265cd3251a5046111248e07ed421).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 07 2025 at 13:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bf1171271afab2055ee6dd577146d47ccfc087f9).
You can git fetch; git checkout nightly-testing and push a fix.

Bryan Gin-ge Chen (Jun 07 2025 at 14:19):

Johan Commelin said:

Kim Morrison said:

We are running mk_all from the master branch, against files on nightly-testing...

Sorry... why is that an issue?

So I haven't read scripts/mk_all.lean, but my best guess from the error that Kim linked earlier is that mk_all requires that the package it's running in has the same toolchain, and here they are different?

Johan Commelin (Jun 07 2025 at 14:23):

Hmmm... That's unfortunate. From what I understand about what mk_all is doing, I would think it could be pretty toolchain agnostic. Back when it was a bash/python script, it certainly was!

github mathlib4 bot (Jun 07 2025 at 16:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6c6e0180f0d3dc9f47f85532f48d268d8656789a).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Jun 07 2025 at 18:01):

Yeah, that's a disadvantage of writing our tooling in lean

github mathlib4 bot (Jun 07 2025 at 19:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (006201f19d874255716a8a2365a2a630984b1dc9).
You can git fetch; git checkout nightly-testing and push a fix.

Damiano Testa (Jun 07 2025 at 21:08):

mk_all goes through some effort of determining the dependencies automatically, so that it works on a "generic" project, not just in mathlib. This has its disadvantages, though, especially now that there are so many meanings for mathlib when dealing with PRs from forks.

github mathlib4 bot (Jun 07 2025 at 22:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bb076f5f2d39b534b917755b0338314b6714304b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 08 2025 at 01:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bb076f5f2d39b534b917755b0338314b6714304b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 08 2025 at 06:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c38c7fde32656c7fa1b2471ed1ae0d50a600f089).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 08 2025 at 09:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3bb3ee2af45a24bd1533f8e1803c06a5035a7070).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 08 2025 at 13:24):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (284e9184e3c66df8c1ab46e85f2cbf4e6b6c3e68).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 08 2025 at 16:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d1c754c26e7bb83ba1f88f9a51e3c536722c769f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 08 2025 at 19:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8b8fe2fa631658e55895b284747a997a249d3599).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 08 2025 at 21:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8b8fe2fa631658e55895b284747a997a249d3599).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 09 2025 at 04:31):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (18fc2693a603f23ffda0e45a2983ccf374aa1323).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 09 2025 at 07:16):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7deb334c5f5104f4edad1a6396dd02a8cddefb86).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 09 2025 at 10:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (fe653fb930c0c9c876267b109287322a055e12a0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 09 2025 at 12:19):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c9a191be40d6f147aa466f25016fdcd251242aab).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 10 2025 at 01:43):

Anne, this is failing both in the build step (because of our recent CI changes), and in the style lint step. Could you look at the style lint step? I think this is fallout from your changes around mathlibLeanOptions.

Kim Morrison (Jun 10 2025 at 02:16):

Sorry, I misdiagnosed this.

@Mac Malone, it seems that after lean#8447 I have to add open Lean in the Mathlib lakefile, because LeanOption has moved from the Lake namespace to the Lean namespace.

Was this intentional?

If so, could you please add a deprecation?

Kim Morrison (Jun 10 2025 at 02:21):

Also, @Mac Malone, on nightly-2025-06-09 in the nightly-testing branch, from lake build I am seeing output like

 [860/6820] Running mathlib/Mathlib:default

where the number keeps counting up, but without ever showing a change in what is being built. (While Aesop was building I was seeing individual files.)

github mathlib4 bot (Jun 10 2025 at 03:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (30b4d6e87eaaa93450a25e8ad795bf3596275589).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 10 2025 at 03:13):

@Mac Malone, the Lean.Options API seems to have changed quite a bit. Could you confirm that adfa721e97b on the nightly-testing branch is in accordance with your intentions?

Mac Malone (Jun 10 2025 at 03:21):

@Kim Morrison LGTM! Sorry for not catching this myself. I overlooked the fact that despite it succesfully triggering the mathlib testing bot, it never actually completing and posted a comment. I will add an export in Lake for LeanOption.

Mac Malone (Jun 10 2025 at 03:31):

Done in lean4#8701.

github mathlib4 bot (Jun 10 2025 at 04:18):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (30b4d6e87eaaa93450a25e8ad795bf3596275589).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Jun 10 2025 at 04:42):

Hmmmzz, progress I guess. But now something's wrong with the cache of Archive and Counterexamples.

github mathlib4 bot (Jun 10 2025 at 07:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0e832cb41d406dc3c36bccead1fb0f1015f53ca7).
You can git fetch; git checkout nightly-testing and push a fix.

Damiano Testa (Jun 10 2025 at 07:17):

Johan Commelin said:

Hmmmzz, progress I guess. But now something's wrong with the cache of Archive and Counterexamples.

This looks like the same error reported at #mathlib4 > Post-Build Step failing.

github mathlib4 bot (Jun 10 2025 at 07:54):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ec6233852527a58479b0ff9fbe8335e1a8f221f5)

Johan Commelin (Jun 10 2025 at 07:56):

Marvelous!

github mathlib4 bot (Jun 10 2025 at 10:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5db2d4df25746b0b19b588e0d6be79ed4da95278).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jun 10 2025 at 11:02):

The nightly failed to be released because of a network issue: https://github.com/leanprover/lean4/actions/runs/15552859159/job/43793596273. And this part of the workflow does not work when retriggered.

Johan Commelin (Jun 10 2025 at 11:06):

@Sebastian Ullrich Do you have a suggestion how to get this back on track? Or do we just wait it out for one day?

Kim Morrison (Jun 10 2025 at 11:18):

The same issue is now occurring in the pr-release.yml action: https://github.com/leanprover/lean4/actions/runs/15557339238/job/43801116160

Kim Morrison (Jun 10 2025 at 11:20):

Claude suggests chainging to use ncipollo/release-action@v1, or just run a shell script:

  run: |  # <-- Raw shell commands, not using any action
    gh release create pr-release-${{ steps.workflow-info.outputs.pullRequestNumber }} \
      --repo ${{ github.repository_owner }}/lean4-pr-releases \
      --title "Release for PR ${{ steps.workflow-info.outputs.pullRequestNumber }}" \
      artifacts/*/*
  env:
    GH_TOKEN: ${{ secrets.PR_RELEASES_TOKEN }}

I'm having trouble guessing the underlying cause... I can take a look in about 45 minutes if no one gets there first. :-)

Sebastian Ullrich (Jun 10 2025 at 15:23):

Apparently they simply broke it: https://github.com/softprops/action-gh-release/issues/628. Could someone pin our version?

github mathlib4 bot (Jun 10 2025 at 16:28):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ec6233852527a58479b0ff9fbe8335e1a8f221f5)

Johan Commelin (Jun 10 2025 at 17:01):

@Sebastian Ullrich voila: https://github.com/leanprover/lean4/pull/8710

github mathlib4 bot (Jun 10 2025 at 19:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ec6233852527a58479b0ff9fbe8335e1a8f221f5)

Kim Morrison (Jun 11 2025 at 00:30):

Kim Morrison said:

Also, Mac Malone, on nightly-2025-06-09 in the nightly-testing branch, from lake build I am seeing output like

 [860/6820] Running mathlib/Mathlib:default

where the number keeps counting up, but without ever showing a change in what is being built. (While Aesop was building I was seeing individual files.)

:ping_pong: @Mac Malone, not sure if you saw this, you replied to one of the three messages.

Kim Morrison (Jun 11 2025 at 00:30):

Kim Morrison said:

Mac Malone, the Lean.Options API seems to have changed quite a bit. Could you confirm that adfa721e97b on the nightly-testing branch is in accordance with your intentions?

@Mac Malone similarly here.

Mac Malone (Jun 11 2025 at 00:35):

@Kim MorrisonOh, sorry, I did see them! As you noted, I replied to the later one (about the Options API. However, I entirely forgot about the former (the progress) in the process. Thanks for reminding me! I will take a look into the progresss issue soonish (probably tomorrow).

Kim Morrison (Jun 11 2025 at 00:37):

@Mac Malone, you replied to the problem about the missing export, but never said anything about the changes in adfa721e97b. Could you confirm on that one?

Mac Malone (Jun 11 2025 at 00:40):

@Kim Morrison The changes seem fine to me. (That's what the "LGTM!" from the reply was referring to. I probably should have quote replied and worded things better to make that more obvious. :sweat_smile:)

Kim Morrison (Jun 11 2025 at 00:40):

All good. Just wasn't sure which subset of things you were responding to. :-)

github mathlib4 bot (Jun 11 2025 at 01:51):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ec6233852527a58479b0ff9fbe8335e1a8f221f5)

github mathlib4 bot (Jun 11 2025 at 08:44):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (507556cae9ed2b8419fe8a42dad90c7f63c512ae)

Kim Morrison (Jun 12 2025 at 03:43):

Uh oh... On nightly-testing now, lake build --no-build takes several minutes (instead of several seconds) to complete.

Mac Malone (Jun 12 2025 at 03:44):

@Kim Morrison Is this new today?

Kim Morrison (Jun 12 2025 at 03:44):

Seems to be. I will check a few previous nightlies now.

Kim Morrison (Jun 12 2025 at 03:44):

I don't see anything particularly scary: perhaps lean4#8654?

Kim Morrison (Jun 12 2025 at 03:45):

Nope, the problem is present on nightly-testing-2025-06-09 as well.

Mac Malone (Jun 12 2025 at 03:46):

There was a performance regression in Lake's lean --setup integration that I am currently investigating.

Mac Malone (Jun 12 2025 at 03:46):

If that is this, I am suprised this did not come up in our previous discussion.

Kim Morrison (Jun 12 2025 at 03:47):

I haven't been building nightly-testing locally the last few days.

Kim Morrison (Jun 12 2025 at 03:47):

And we don't have any CI that would detect this. (We should!)

Kim Morrison (Jun 12 2025 at 03:47):

(i.e. just set a maximum time in the existing --no-build check)

Mac Malone (Jun 12 2025 at 03:48):

Ah, okay, then I am currently working on that. Hopefully I will have a fix tomorrow.

Kim Morrison (Jun 12 2025 at 03:48):

nightly-testing-2025-06-05 is fine, so it is somewhere in between those

Kim Morrison (Jun 12 2025 at 03:49):

Okay. If you won't have a fix before the nightly is cut, could you revert it for now? nightly-testing is unusable right now.

Mac Malone (Jun 12 2025 at 03:51):

If necessary, sure. Just to make sure this is the issue, how did you encounter the progress issue on nightly-testing without running into this?

Kim Morrison (Jun 12 2025 at 03:53):

Good question. I assume that I'd actually made changes, and so expected it to be slow because it was actually building. It's only today that I realised it was slow even without changes.

Mac Malone (Jun 12 2025 at 03:56):

That woould fit with what I understand of the issue. It appears to be a fixed startup cost, so any signficant build work will outpace it.

github mathlib4 bot (Jun 12 2025 at 04:08):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (507556cae9ed2b8419fe8a42dad90c7f63c512ae)

Mac Malone (Jun 12 2025 at 04:46):

Reversion of the main change that should be causing this is at lean4#8736. I am benching it now to verify that this fixes the performance.

github mathlib4 bot (Jun 12 2025 at 07:45):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (507556cae9ed2b8419fe8a42dad90c7f63c512ae)

github mathlib4 bot (Jun 12 2025 at 10:25):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0665576140e9230df6e2705ab13a40e1f97e1e75).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 12 2025 at 12:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dd1b855f6545ac5892b13fe6c80ff6098ebc7fa6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 12 2025 at 14:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (6763a6b949fef28608b5924d78e64443b00a4de5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 12 2025 at 16:20):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (41813ea0472a1e7b0b67e059628141ddaffd08c6).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 12 2025 at 16:46):

I've added an adaptation note. The simpNF linter is saying:

/- The `simpNF` linter reports:
SOME SIMP LEMMAS ARE NOT IN SIMP-NORMAL FORM.
see note [simp-normal form] for tips how to debug this.
https://leanprover-community.github.io/mathlib_docs/notes.html#simp-normal%20form -/
-- Mathlib.Analysis.Normed.Operator.Banach
Error: /home/lean/actions-runner/_work/mathlib4/mathlib4/pr-branch/Mathlib/Analysis/Normed/Operator/Banach.lean:366:1: error: @ContinuousLinearMap.equivRange_symm_toLinearEquiv Left-hand side simplifies from
  (ContinuousLinearMap.equivRange hinj hclo).symm.toLinearEquiv
to
  (ContinuousLinearMap.equivRange hinj hclo).symm
using
  dsimp only [*, @ContinuousLinearEquiv.toLinearEquiv_symm]

but making that change doesn't typecheck.

@Johan Commelin, any ideas there?

Johan Commelin (Jun 12 2025 at 16:47):

Hmmz, shall we remove @[simp] and leave an adaptation note that it should be restored?

Kim Morrison (Jun 12 2025 at 16:48):

For now I added nolint simpNF. I think either is fine?

github mathlib4 bot (Jun 12 2025 at 16:59):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e90c049dd73c386a1fd3aedc82ac15728986b8ba).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 12 2025 at 17:31):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ff8c43ce37dd0f416618df7d95c8a7d497efa4ba)

Sébastien Gouëzel (Jun 12 2025 at 18:16):

I've pushed a fix: since #25604, the normal form has symm to the end, so I have replaced (ContinuousLinearMap.equivRange hinj hclo).symm.toLinearEquiv with (ContinuousLinearMap.equivRange hinj hclo).toLinearEquiv.symm.

github mathlib4 bot (Jun 12 2025 at 18:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (079d907947d1f6e81eb9578652c34da168a0d886).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 12 2025 at 19:32):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ff8c43ce37dd0f416618df7d95c8a7d497efa4ba)

github mathlib4 bot (Jun 13 2025 at 00:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (04defa097355b5354bc614e78d62381915de05c3).
You can git fetch; git checkout nightly-testing and push a fix.

Kyle Miller (Jun 13 2025 at 07:08):

Heads up: I thought I saw that lean4#7395 had a clean mathlib build and merged, but I forgot that the bot shows :check: when there are linter warnings. It's just a handful of discretionary shows. I figure at this point @Robin Arnez or someone else can follow up with this discussion and change the unused tactic linter, or otherwise comment these shows out with adaptation notes.

github mathlib4 bot (Jun 13 2025 at 07:22):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (ff8c43ce37dd0f416618df7d95c8a7d497efa4ba)

github mathlib4 bot (Jun 13 2025 at 09:07):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8bbb5cb82be152d13e59d682bb718b170227693d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 13 2025 at 09:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8bbb5cb82be152d13e59d682bb718b170227693d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 13 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3117eecd5f446dcb117140921e74e5f123cd6c31).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 13 2025 at 15:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (dfb6ce9dacf6008f7e8605573b93834bb4f64388).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jun 13 2025 at 15:53):

There seems to have been some miscommunication, I'm sorry; but I maybe wanted to wait a bit with #25749 until there was clear consensus about whether we want to lint show (but now we don't have an adaptation for the original PR!). Now I feel like the best way to go is to make batteries build (batteries#1273) and then just fix the unused tactic linter for the nightly builds. #25749 would then go towards master and can be merged (or closed) when there is clear consensus whether this linter should or should not exist.

github mathlib4 bot (Jun 13 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8e87a39073921d284b41aa374f987d1cb8389034).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 13 2025 at 21:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8e87a39073921d284b41aa374f987d1cb8389034).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 13 2025 at 22:57):

A small fix was required for lean#8660.

Kim Morrison (Jun 13 2025 at 23:14):

@Sebastian Ullrich, I suspect this one is for you:

info: Mathlib/LinearAlgebra/Reflection.lean:238:0: PANIC at Lean.EnvExtension.modifyState Lean.Environment:1354:13: environment extension is marked as `mainOnly` but used in async context 'Module.reflection_mul_reflection_zpow_apply'

Kim Morrison (Jun 13 2025 at 23:24):

I have removed all the no-op show statements on nightly-testing. If we decide we want to revert this later, it is all contained in f076c124d254e3396ad236f987b1920803416674.

github mathlib4 bot (Jun 14 2025 at 00:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (500dfe433a366d409a53a24ac6d8707b1fad58df).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 14 2025 at 04:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (121a02334ffc8d465d6b417b157ba649f37504ec).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 14 2025 at 09:32):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b91260d8f8793f387f404608e5e069acebafd127).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 14 2025 at 10:02):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b91260d8f8793f387f404608e5e069acebafd127).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jun 14 2025 at 11:10):

Kim Morrison said:

Sebastian Ullrich, I suspect this one is for you:

info: Mathlib/LinearAlgebra/Reflection.lean:238:0: PANIC at Lean.EnvExtension.modifyState Lean.Environment:1354:13: environment extension is marked as `mainOnly` but used in async context 'Module.reflection_mul_reflection_zpow_apply'

Thanks for the ping, build succeeds with #8783

github mathlib4 bot (Jun 14 2025 at 13:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9c220e68f000c0ef821bc446fbd62743dbe25771).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 14 2025 at 16:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (50e49dc2e9c35748e2313071052bdb6dd16a6fe5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 15 2025 at 01:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ad1b437587a1dbcc0b22624cb0ae9208d206508a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 15 2025 at 06:20):

lean#8783

github mathlib4 bot (Jun 15 2025 at 06:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9b0c6a877559b4bb45860affaeafb705cee085aa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 15 2025 at 10:01):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c1abdfac7d2c45c0b4498f4bcdb3eb326cc8dd1e).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 15 2025 at 10:09):

Unfortunately we didn't get a nightly-2025-06-15 because of an unrelated CI failure, so we're still broken because of the panic.

Sebastian Ullrich (Jun 15 2025 at 11:18):

I'll put in a workaround and retrigger

github mathlib4 bot (Jun 15 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d6898ad6d18b35cc86b820cf9e974f91464f9956).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 15 2025 at 13:49):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d6898ad6d18b35cc86b820cf9e974f91464f9956).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 15 2025 at 14:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d6898ad6d18b35cc86b820cf9e974f91464f9956).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jun 15 2025 at 14:26):

linting failures

Sebastian Ullrich (Jun 15 2025 at 14:26):

I had to push an empty commit because of #nightly-testing > bot not running CI

github mathlib4 bot (Jun 15 2025 at 15:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (0e9bcbf7a1008b0b88cad6c59abf12bed4cfe3b8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 15 2025 at 19:22):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (76bbcf04d10aa01ae77c716c8962840dc6eb708e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 15 2025 at 22:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e6f52a442b52ac7fddcb4ae4818e1751c6efd3c9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 15 2025 at 22:33):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (948d9cf87c819cd70097ea14acdd04c1e1662205)

github mathlib4 bot (Jun 16 2025 at 10:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (84e70de5507db0f1c6bcffaf2be6aa8aad81fc27).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 16 2025 at 12:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (84e70de5507db0f1c6bcffaf2be6aa8aad81fc27).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 16 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (84e70de5507db0f1c6bcffaf2be6aa8aad81fc27).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 16 2025 at 16:05):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1a83ec9d7a74f9063014411a530bdbdbb3b86a38).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 16 2025 at 18:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (db52f0992d294d2273c2eff06bc4cfac13460b0c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 16 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (953440dbe5b77d9a00996d6c216a2605a70b5560).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 16 2025 at 22:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (953440dbe5b77d9a00996d6c216a2605a70b5560).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 16 2025 at 23:18):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (442b5ff8c6f5f3422ddb2f05dc995312c0151133)

github mathlib4 bot (Jun 17 2025 at 11:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (260a59832ccf9c8e06fb1c814c7ff52904b449a3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 17 2025 at 12:52):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (2b6e3d707757364f10504dedab0ffb33151a128e).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jun 17 2025 at 14:40):

List.eraseIdx_insertIdx seems to have been removed without deprecation!

github mathlib4 bot (Jun 17 2025 at 14:43):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d9d3b4ca93885992bd5e90cea0920539876590a7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 17 2025 at 15:03):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d9d3b4ca93885992bd5e90cea0920539876590a7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 17 2025 at 16:15):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b28d99bfc16a696dbadad5aa76994b5e18077878)

github mathlib4 bot (Jun 17 2025 at 19:57):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (1e3fd2ae72c72afc312889b3be4d1e9aba69f048).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 17 2025 at 20:58):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b28d99bfc16a696dbadad5aa76994b5e18077878)

Kim Morrison (Jun 18 2025 at 00:06):

Robin Arnez said:

eraseIdx_insertIdx

@Robin Arnez, could you clarify? It seems to have been deprecated:

theorem eraseIdx_insertIdx_self {i : Nat} {xs : Array α} (h : i  xs.size) :
    (xs.insertIdx i a).eraseIdx i (by simp; omega) = xs := by
  rcases xs with xs
  simp_all

@[deprecated eraseIdx_insertIdx_self (since := "2025-06-15")]
theorem eraseIdx_insertIdx {i : Nat} {xs : Array α} (h : i  xs.size) :
    (xs.insertIdx i a).eraseIdx i (by simp; omega) = xs := by
  simp [eraseIdx_insertIdx_self]

I would like to add a new unconditional eraseIdx_insertIdx, but I ran out of time while trying to work out what the actual statement is. If anyone feels like filling that hole, much appreciated!

github mathlib4 bot (Jun 18 2025 at 01:01):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (b28d99bfc16a696dbadad5aa76994b5e18077878)

Robin Arnez (Jun 18 2025 at 07:34):

I'm referring to List.eraseIdx_insertIdx

Kim Morrison (Jun 18 2025 at 08:35):

Thanks: lean#8863.

github mathlib4 bot (Jun 18 2025 at 10:31):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (294bb3092e09c13589badb26029975a8c23bace3)

github mathlib4 bot (Jun 19 2025 at 09:33):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15948de6846fca0ff7d814eb3e5e53333f8f98d9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 19 2025 at 09:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (15948de6846fca0ff7d814eb3e5e53333f8f98d9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 19 2025 at 13:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7156927d977c9f8907dbbc26c03343d9ca0e8ebc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 19 2025 at 14:21):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a764cea413f461f95d178ff2b45603eb23325c9f)

github mathlib4 bot (Jun 19 2025 at 14:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4516ade29687c518f78674687cbe5054dff0b6de).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 19 2025 at 15:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8fea0ef4f2fb3e534fb87a0bb0b54ef0b3e2b1ca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 19 2025 at 21:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11c6fbd61e7ad45f5b09ec03688b1faebd8c6bc5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 19 2025 at 23:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (11c6fbd61e7ad45f5b09ec03688b1faebd8c6bc5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 20 2025 at 01:46):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (a764cea413f461f95d178ff2b45603eb23325c9f)

github mathlib4 bot (Jun 20 2025 at 11:42):

:check: The latest CI for Mathlib's branch#nightly-testing has succeeded! (94511d1ad61c75e054cf7e2e341c4fa856c762e3)

github mathlib4 bot (Jun 20 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (bee89f3673fb76a7d18eba011b7faf678a6f5888).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 20 2025 at 21:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (3a374b3d383130b67c070244bb80e8076a3162e8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 21 2025 at 01:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3b173fdbb090edd2cd442ffce037920b2c90c57).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 21 2025 at 03:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3b173fdbb090edd2cd442ffce037920b2c90c57).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jun 21 2025 at 08:24):

github mathlib4 bot schrieb:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3b173fdbb090edd2cd442ffce037920b2c90c57).
You can git fetch; git checkout nightly-testing and push a fix.

#26246

github mathlib4 bot (Jun 21 2025 at 09:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c3b173fdbb090edd2cd442ffce037920b2c90c57).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 21 2025 at 12:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e2f8bf7b23d89378826e81b4404891f7291233a8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 22 2025 at 02:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e2f8bf7b23d89378826e81b4404891f7291233a8).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 22 2025 at 03:27):

@Jovan Gerbscheid (or perhaps @Floris van Doorn), could you take a look at the failures in RefinedDiscrTree on nightly-testing?

If you make a PR to nightly-testing and ping me here, we will merge it asap.

Cameron Zwarich (Jun 22 2025 at 03:31):

@Kim Morrison I'm pretty sure this is fallout from lean4#8577. I can't push to the Mathlib PR branch, so I put the changes here:
https://github.com/leanprover-community/mathlib4/compare/lean-pr-testing-8577...zwarich:mathlib4:lean-pr-testing-8577
In particular, the fix for this RefinedDiscrTree issue:
https://github.com/leanprover-community/mathlib4/commit/a44064ca904086697218920bcd4231a8e0aa83a3

Kim Morrison (Jun 22 2025 at 03:48):

Thanks, I'll merge now.

github mathlib4 bot (Jun 22 2025 at 04:13):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e2f8bf7b23d89378826e81b4404891f7291233a8).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 22 2025 at 04:45):

Unfortunately these breakages are due to #8745. I've asked @Sebastian Graf to investigate.

github mathlib4 bot (Jun 22 2025 at 04:45):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e2f8bf7b23d89378826e81b4404891f7291233a8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 22 2025 at 06:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (087a0dcf4e085d7b18f0edfa58feec58455e4811).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Graf (Jun 22 2025 at 08:44):

Sorry about that! Reverted in #8926 until I debug this on Monday

github mathlib4 bot (Jun 22 2025 at 08:58):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (69f66e45f2b260a05ad7f57389dc0e26d1625209).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 22 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (98757f740ed946f6a907f8a9768bf475d7a02200).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 22 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (e004dbe1b44429f881c0052f44c5175ab3b6d774).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 22 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (27dacf7872f1687d629b4677edd14530c27f9bb3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 22 2025 at 18:41):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ffbf9db0c1b1c5d1693997bbc44633b032fa0c09).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 22 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (4f1603b00f5c3e0e43d0daf234c4199c342782db).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 04:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7585da85249b3fdfaaeced1967bcf87fa72d3526).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 06:47):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (7585da85249b3fdfaaeced1967bcf87fa72d3526).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 09:14):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (df94cc8aed24878666997fe1ea7fc2f2ffab7770).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 09:39):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8425daf3115a1d977ed66db14278891ebcd86622).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 12:48):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (f609d6347c79cace43753bbe8228ba33dc0bb4bb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 15:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ffaf539d0a3f5686921aafef32ac8b41ec5f9070).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 15:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (8910701cb7c78acaa4cabdd0e94b8bd721a4dd51).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (24c007389a7c2b221fa6214ae41c90d79a169650).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 16:12):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (9bb19c991ac039c5efcd04309b4d6cbd088a1d30).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 23 2025 at 17:26):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c5a9e9845d0661a9e75758afda16a8f92724b809).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 23 2025 at 23:54):

github mathlib4 bot said:

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (c5a9e9845d0661a9e75758afda16a8f92724b809).
You can git fetch; git checkout nightly-testing and push a fix.

Just noting that this message (correctly!) refers to a commit on the nightly-testing branch on the new mathlib4-nightly-testing fork.

Kim Morrison (Jun 23 2025 at 23:55):

Be careful for now that these branches are duplicated, and not automatically sync'd across the forks. Once we're got green and validated a few more things, we'll be deleting everything relating to nightly-testing from the main repo.

Kim Morrison (Jun 23 2025 at 23:59):

I've disabled unusedSimpArgs in Batteries for now.

Kim Morrison (Jun 23 2025 at 23:59):

If any Batteries contributors would like to re-enable it (by fixing its suggestions) that would be lovely.

Kim Morrison (Jun 24 2025 at 00:03):

I've fixed a deprecation in Aesop, and resolved the unusedSimpArgs linter results in Aesop (i.e. left that option on).

github mathlib4 bot (Jun 24 2025 at 01:30):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ddeb36463f3add2f7f51064165a94955f6a63488).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 24 2025 at 02:06):

Oof, I've fixed the grind instance problems, the one remaining one is that MathlibTest/zmod.lean is failing:

-- A Mersenne exponent, chosen so the test below takes no more than a few seconds
-- but should be enough to trigger a stack overflow from a non-tail-recursive implementation
-- of exponentiation by repeated squaring.
def k := 11213
def p := 2^k - 1

set_option exponentiation.threshold 100000 in
-- We ensure here that the `@[csimp]` attribute successfully replaces (at runtime)
-- the default value of `npowRec` for the exponentiation operation in `Monoid`
-- with a tail-recursive implementation by repeated squaring.
/-- info: 1 -/
#guard_msgs in
#eval (37 : ZMod p)^(p-1)

Any ideas which change could have triggered this?

Kim Morrison (Jun 24 2025 at 02:07):

Candidates:

  • I've messed up the typeclasses somehow in making grind changes?
  • The new compiler??

github mathlib4 bot (Jun 24 2025 at 02:50):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (d5fc04be39b3c3d14232958d6f67a4bbedb94f1b).
You can git fetch; git checkout nightly-testing and push a fix.

Cameron Zwarich (Jun 24 2025 at 03:55):

Kim Morrison said:

Oof, I've fixed the grind instance problems, the one remaining one is that MathlibTest/zmod.lean is failing:

-- A Mersenne exponent, chosen so the test below takes no more than a few seconds
-- but should be enough to trigger a stack overflow from a non-tail-recursive implementation
-- of exponentiation by repeated squaring.
def k := 11213
def p := 2^k - 1

set_option exponentiation.threshold 100000 in
-- We ensure here that the `@[csimp]` attribute successfully replaces (at runtime)
-- the default value of `npowRec` for the exponentiation operation in `Monoid`
-- with a tail-recursive implementation by repeated squaring.
/-- info: 1 -/
#guard_msgs in
#eval (37 : ZMod p)^(p-1)

Any ideas which change could have triggered this?

I went back to check and this fails on the branch where I had the new compiler. This is failing with a stack overflow in Nat.binaryRec._redArg. The comment in the test indicates that this implementation is not supposed to be used, due to csimp replacing it with a more efficient implementation. The new compiler definitely supports csimp. In this case, the actual csimp seems to be coming from a to_additive tactic, which might be part of the complication:

@[to_additive (attr := csimp)]
theorem npowRec_eq_npowBinRec : @npowRecAuto = @npowBinRecAuto := by
  funext M _ _ k m
  rw [npowBinRecAuto, npowRecAuto, npowBinRec]
  match k with
  | 0 => rw [npowRec, npowBinRec.go, Nat.binaryRec_zero]
  | k + 1 => rw [npowBinRec.go_spec, npowRec_eq]

The new compiler does csimp replacement a bit earlier than the old compiler, but I also don't immediately see how this could be contributing.

Kyle Miller (Jun 24 2025 at 04:10):

I commented out this test and added an adaptation note.

Cameron Zwarich said:

The new compiler does csimp replacement a bit earlier than the old compiler

Maybe that phase isn't seeing through the instances? (I'm kind of surprised that this sort of csimp lemma ever worked!)

github mathlib4 bot (Jun 24 2025 at 05:06):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (b47dd848b7a0be8753fcc35794ffa18f026aadd2).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 24 2025 at 05:12):

Okay, I think this may have been due to a missing secret, which I've just installed.

github mathlib4 bot (Jun 24 2025 at 05:15):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5efd73a5d3ea04fdbd9cb7622b007778ae22d47c).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 24 2025 at 05:16):

failure was apparently a transient error? an rm -rf failed with "directory not empty"!?

Cameron Zwarich (Jun 24 2025 at 05:27):

Kyle Miller said:

I commented out this test and added an adaptation note.

Cameron Zwarich said:

The new compiler does csimp replacement a bit earlier than the old compiler

Maybe that phase isn't seeing through the instances? (I'm kind of surprised that this sort of csimp lemma ever worked!)

It's calling the npowBinRecAuto version, so the csimp is being applied. The issue seems to be that the call to npowBinRecAuto in Fin.instCommRing doesn't get specialized, and thus the call to Nat.binaryRec doesn't get specialized, and it doesn't become tail recursive.

Damiano Testa (Jun 24 2025 at 05:39):

Kim Morrison said:

failure was apparently a transient error? an rm -rf failed with "directory not empty"!?

I've seen this error on Zulip before: let me find it.

Damiano Testa (Jun 24 2025 at 05:40):

#mathlib4 > CI error

Damiano Testa (Jun 24 2025 at 05:40):

I don't know if it was resolved, though.

github mathlib4 bot (Jun 24 2025 at 06:11):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (5efd73a5d3ea04fdbd9cb7622b007778ae22d47c).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 24 2025 at 06:19):

Should be resolved by #26335

github mathlib4 bot (Jun 24 2025 at 10:34):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ddfb62ceafe025db4ebea0b95b4497d54f62e602).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 24 2025 at 14:10):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (ee86d36ab1dd03463f288b0930f88dde5fc7f038).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 24 2025 at 14:21):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (352c8fe70d2d824e56b42ae4eff3d81e12b02ad9).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jun 24 2025 at 15:07):

branch#nighly-testing is a dead link; does branch#leanprover-community/mathlib4-nightly-testing:nightly-testing work?

Robin Arnez (Jun 24 2025 at 15:09):

Hmm, no, well then nighly-testing branch?

Bryan Gin-ge Chen (Jun 24 2025 at 15:09):

I guess we could introduce a linkifier that overrides the usual behavior of branch# for things starting with branch#nightly-testing?

Robin Arnez (Jun 24 2025 at 15:11):

I think [nighly-testing branch](https://github.com/leanprover-community/mathlib4-nightly-testing/tree/nightly-testing) is the simplest solution here, otherwise we'd need to account for lean-pr-testing-nnnn, batteries-pr-testing-nnnn etc.

Bryan Gin-ge Chen (Jun 24 2025 at 15:14):

Ah, in that case we won't have to touch the linkifiers and can just modify the bot.

Robin Arnez (Jun 24 2025 at 15:19):

#26363

github mathlib4 bot (Jun 24 2025 at 15:28):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (181035fc4b4f4906081d462bff8d3e8e1ed34cc8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 25 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's branch#nightly-testing has failed (952958955c177b70db52b9f0398b99c1d43b52e0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 26 2025 at 00:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fe308e4ca7d9774f565977000df41fcecd835e20).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 26 2025 at 01:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d9ca23c0c7f6327cc2535dca0237925b270876b5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 26 2025 at 02:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d9ca23c0c7f6327cc2535dca0237925b270876b5).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 26 2025 at 03:00):

This is still not retrieving oleans successfully, and I can't work out why. It looks like it is both uploading and downloading from the mathlib4-nightly-testing part of the cache.

Kim Morrison (Jun 26 2025 at 03:00):

:eyes: welcome here

github mathlib4 bot (Jun 26 2025 at 05:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8499edf0ab8fee0f1a872b09aaefaff471ea205f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 26 2025 at 06:01):

(New hypothesis; we're using expired tokens, asking for new ones now.)

github mathlib4 bot (Jun 26 2025 at 06:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (abc613d853099ef2d853d4f1d80415444f9a8e12).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jun 26 2025 at 07:09):

Yay!

% lake exe cache get
Current branch: nightly-testing
Using cache from nightly-testing remote: leanprover-community/mathlib4-nightly-testing
Attempting to download 6883 file(s) from leanprover-community/mathlib4-nightly-testing cache
Downloaded: 1358 file(s) [attempted 1358/6883 = 19%]

github mathlib4 bot (Jun 26 2025 at 07:11):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (a34e1c5f921ae3180b4b17d3e7f6dbe2fd429c64)

Kim Morrison (Jun 26 2025 at 07:15):

and lean4's nightly-with-mathlib branch has advanced to nightly-2025-06-25!

Kim Morrison (Jun 26 2025 at 07:17):

and testing integrated CI at lean#9009

Johan Commelin (Jun 26 2025 at 07:17):

Awesome!

github mathlib4 bot (Jun 26 2025 at 09:43):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (a7a22988bfc0af71de347122a1f8e6921d34341e)

Damiano Testa (Jun 26 2025 at 20:41):

I just saw lean4#8626, which is great! It may cause some issues for the commandStart linter, since it was working around the pretty-printing of comments.

Damiano Testa (Jun 26 2025 at 20:42):

I think that it will make the code easier, but it may have broken some of its internal logic.

github mathlib4 bot (Jun 27 2025 at 02:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (07cfcb45828dd2b1853c54fca7b21615710b9274).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 27 2025 at 03:44):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (a7a22988bfc0af71de347122a1f8e6921d34341e)

github mathlib4 bot (Jun 27 2025 at 09:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6732e714d6e517f95987eb9a4a534c058e5c09d4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 27 2025 at 16:31):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (ad22e744d4e452c699b7920037aaefd5c1b340a3)

github mathlib4 bot (Jun 28 2025 at 04:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (80e325d03e62156434a5ca14444ca6e62ca1ae6d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 28 2025 at 06:17):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (67ea618eaa7da522864a1af4f72d040a9a2ab001).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 28 2025 at 06:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5e3fdf53a6d5dff83adb5b845f49565174190848).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 28 2025 at 07:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d9e205156e8e5455a1cb54740a0bd2a31cf329f0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 28 2025 at 13:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4e342cc3cce123c2f650d4b0aba684b3082653aa).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jun 28 2025 at 13:08):

test failures from error message changes

github mathlib4 bot (Jun 28 2025 at 16:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (220e69382df066881c9670d59e46a8469781e95c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 29 2025 at 05:52):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (0d70a64f5c7231677f7cf3f306c00a037bc9f1a7)

github mathlib4 bot (Jun 29 2025 at 07:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (232f6019633df4c5df35823b2a3aed5e3cc9e93e).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jun 29 2025 at 07:35):

New unused simps... :)

github mathlib4 bot (Jun 29 2025 at 08:07):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (0d70a64f5c7231677f7cf3f306c00a037bc9f1a7)

github mathlib4 bot (Jun 29 2025 at 09:44):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c79d633c61f6f1f22e16f1b496b558adb7fd76c0)

github mathlib4 bot (Jun 29 2025 at 12:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (944ea7b2547e7c9b17f597ba90967f79cbf217e9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 29 2025 at 12:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b8a60b9f8f35da39b97573411ab1b45e9635dea7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 29 2025 at 20:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (72d1975dc5e9aa6978e2746c94f24d0dc7d20d56).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 29 2025 at 22:57):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c79d633c61f6f1f22e16f1b496b558adb7fd76c0)

github mathlib4 bot (Jun 30 2025 at 10:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (652ecde381fdeddf8cc064277ebeadf1d4ba8f6a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 30 2025 at 11:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4d3f9fc4f9a617e732cbc1e665c4459699c65c53).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 30 2025 at 11:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4d3f9fc4f9a617e732cbc1e665c4459699c65c53).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jun 30 2025 at 12:24):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (89823940ea0b4649c7c323bb97d582b98701710f)

github mathlib4 bot (Jun 30 2025 at 23:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7336b4823df10e3e99f011ccd84868964cf5762b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 01 2025 at 01:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (20c9066cc51942ee4e2b16102c272dd37b1c86d7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 01 2025 at 04:15):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9bb543f12cbf71b988811ffb377bc4c0afd1edd1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 01 2025 at 05:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (bbe8bf86d6e417b9a2d778249d89dbc03751cbc1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 01 2025 at 07:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6a76d664e308892f6585150fa5ae16f699c5dff4).
You can git fetch; git checkout nightly-testing and push a fix.

Matthew Ballard (Jul 01 2025 at 12:37):

I wanted to see the logs for the post-build step to see the more verbose logs and confirm some things. But it hasn't reached there since the change. So I thought I poke at fixes but after cloning leanprover-community/mathlib4-nightly-testing, I cannot get lake exe cache get to do anything useful. Is this expected? Am I missing something?

Kim Morrison (Jul 01 2025 at 12:53):

We had some severe outages on nightly-testing the last 48 hours due to some release related bugs (the bug that results in rc2!)

Kim Morrison (Jul 01 2025 at 12:53):

I think the current run at https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/15999671828 will be more informative / successful.

Matthew Ballard (Jul 01 2025 at 12:58):

What should lake exe cache get do?

github mathlib4 bot (Jul 01 2025 at 13:45):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (db224c26fed68ca7bb97062baa775cfcd1b8c329)

Kim Morrison (Jul 02 2025 at 00:29):

Matthew Ballard said:

What should lake exe cache get do?

On these nightly-testing builds, lake exe cache get ought to be putting and retrieving the cache from the leanprover-community/mathlib4-nightly-testing cache.

github mathlib4 bot (Jul 02 2025 at 00:47):

:warning: Warning: The lean-toolchain file in the latest bump branch does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.
Current content:
This needs to be fixed for the nightly testing process to work correctly.

Kim Morrison (Jul 02 2025 at 01:01):

Hmm, this message seems to be mistaken. I'll make the reporting more robust here.

Kim Morrison (Jul 02 2025 at 01:03):

#26605

github mathlib4 bot (Jul 02 2025 at 09:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (79c95d5ec83b4c065e706977a13146ee8af2b744).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 02 2025 at 10:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d2e1782f49535d6a7a965e46f4bd914d9917d24c).
You can git fetch; git checkout nightly-testing and push a fix.

Matthew Ballard (Jul 02 2025 at 12:30):

Kim Morrison said:

Matthew Ballard said:

What should lake exe cache get do?

On these nightly-testing builds, lake exe cache get ought to be putting and retrieving the cache from the leanprover-community/mathlib4-nightly-testing cache.

In CI this is achieved with the repo flag being set, if I just check out the branch on my clone of the fork, I assume it should do the same. But it does nothing. Is lake exe cache get not part of the usual workflow for fixes or am I missing something?

github mathlib4 bot (Jul 02 2025 at 13:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d2ae93ab36e184f7f5149c86f58a04f1c5d6e8f7).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jul 02 2025 at 14:44):

I think someone is missing something. The git checkout nightly-testing; lake exe cache get usually results in a successful retrieval of at least something for me.

Kim Morrison (Jul 02 2025 at 14:45):

e.g. just now:

% get nightly-testing
warning: refname 'nightly-testing' is ambiguous.
Switched to branch 'nightly-testing'
Your branch is up to date with 'nightly-testing/nightly-testing'.
remote: Enumerating objects: 3, done.
remote: Counting objects: 100% (1/1), done.
remote: Total 3 (delta 0), reused 0 (delta 0), pack-reused 2 (from 1)
Unpacking objects: 100% (3/3), 1.73 KiB | 443.00 KiB/s, done.
From github.com:leanprover-community/mathlib4-nightly-testing
   d2e1782f495..d2ae93ab36e  nightly-testing -> nightly-testing/nightly-testing
Updating d2e1782f495..d2ae93ab36e
Fast-forward
 lake-manifest.json | 2 +-
 1 file changed, 1 insertion(+), 1 deletion(-)
info: plausible: checking out revision 'fde3fc21dd68a10791dea22b6f5b53c5a5a5962d'
info: importGraph: checking out revision '856a8cb8908af109aac3ce13e2b4f866f3d75199'
info: proofwidgets: checking out revision '2d6d124aedc3023506a67e50bfd5582384d6bd17'
info: aesop: checking out revision 'a1b5d59f433c6ec2b318192bd910c257a3c62be8'
info: Qq: checking out revision '56047303fce0d07dcae7e3e91b17eef67d11f6f4'
info: batteries: checking out revision '7f8c95c59c246ae4a85315de3e536943ea22ae08'
info: Cli: checking out revision '1604206fcd0462da9a241beeac0e2df471647435'
Current branch: nightly-testing
Is nightly-testing a remote URL? false
Extracted repo from remote URL:
Using cache from nightly-testing remote: leanprover-community/mathlib4-nightly-testing
Attempting to download 6895 file(s) from leanprover-community/mathlib4-nightly-testing cache
Downloaded: 6884 file(s) [attempted 6895/6895 = 100%] (99% success)
Attempting to download 11 file(s) from leanprover-community/mathlib4 cache
Downloaded: 0 file(s) [attempted 11/11 = 100%] (0% success)
Warning: some files were not found in the cache.
This usually means that your local checkout of mathlib4 has diverged from upstream.
If you push your commits to a branch of the mathlib4 repository, CI will build the oleans and they will be available later.
Alternatively, if you already have pushed your commits to a branch, this may mean the CI build has failed part-way through building.
Decompressing 6884 file(s)

Matthew Ballard (Jul 02 2025 at 14:50):

Huh. Same behavior. Thanks. Not sure what happened before.

github mathlib4 bot (Jul 02 2025 at 15:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (748fb4bc7e253be9f444f46fca8613220c3b021d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 02 2025 at 16:00):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (ba1eddb9838ecfb4e994d061ad19a7f8cae7c2ff)

github mathlib4 bot (Jul 03 2025 at 10:13):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (cff489e0715ed8f943a2ea8b0a3bbc208170f4c8)

Kim Morrison (Jul 04 2025 at 00:11):

Just a heads up that lean-pr-testing-9168 on the leanprover-community/mathlib4-nightly-testing fork will need merging into nightly-testing this evening.

I'm not sure if the automatic merge bot will pick this one up, as the branch was created manually.

github mathlib4 bot (Jul 04 2025 at 02:06):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (cff489e0715ed8f943a2ea8b0a3bbc208170f4c8)

github mathlib4 bot (Jul 04 2025 at 09:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5c2779d74ccb0a2f3b50f5751e27428adad7ff7b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 04 2025 at 15:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cd86023575fe28099ea9d80ce23a30ac02542abf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 05 2025 at 09:20):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a3fea1ddef70d4200743be14edfc03df9cb8cd76).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 06 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b8fddd0faf04bb44ed9b787f88211c62754b2151).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 07 2025 at 09:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ded554dcebac64917b21a78470f209290e8586b4).
You can git fetch; git checkout nightly-testing and push a fix.

Cameron Zwarich (Jul 07 2025 at 22:13):

Does anyone know how to fix these grind errors? It would be nice to get this building again.

Robin Arnez (Jul 08 2025 at 07:00):

As far as I know, these were fixed on master but the merge failed (?)

Robin Arnez (Jul 08 2025 at 07:03):

For reference: 19f4ef2

Kevin Buzzard (Jul 08 2025 at 07:34):

But #26715 is merged?

github mathlib4 bot (Jul 08 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (318f85e0600205f8243c0c4e581d06ea4488dfaf).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 08 2025 at 09:26):

Yeah I mean they didn't properly merge into nightly-testing

Robin Arnez (Jul 08 2025 at 09:26):

For some reason...

Robin Arnez (Jul 08 2025 at 09:27):

Something like a git cherry-pick 19f4ef2c52b278bd96626e02d594751e6e12ac98 might be enough to get it working again

github mathlib4 bot (Jul 09 2025 at 09:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3c3a510d8046e29080581404a73830e14f4ff250).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 10 2025 at 08:56):

Could I request write access for nightly-testing? (for fixing this and for other lean PRs in the future)

github mathlib4 bot (Jul 10 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a47fcb8fbcb494f44b8d3d6fc2cf88907052e7f9).
You can git fetch; git checkout nightly-testing and push a fix.

Kevin Buzzard (Jul 10 2025 at 09:41):

@Robin Arnez you should have write access to mathlib non-master branches now

Robin Arnez (Jul 10 2025 at 09:41):

Hmm, I'm not interested in mathlib, but mathlib4-nightly-testing, if anyone could do that

Kevin Buzzard (Jul 10 2025 at 09:42):

Oh apologies, I hadn't realised that this was a different repo.

Kevin Buzzard (Jul 10 2025 at 10:02):

@Robin Arnez invitation sent!

github mathlib4 bot (Jul 10 2025 at 10:29):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7fcf4f67c8ffc416ea20d884f56a08a9d24f27e5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 10 2025 at 11:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (66a4a8e7884856f2183c6023d9b39c5483466d67).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 10 2025 at 13:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e6a92dfeea954dfe3f945764858b3952d3b36914).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 10 2025 at 14:28):

nightly#11 is building!

github mathlib4 bot (Jul 10 2025 at 15:58):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (15ebf28712be5f7c5416c9ef6f220b8c05c3d813)

github mathlib4 bot (Jul 11 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7a16afbc8072070a5089e456a34c56f666f09dde).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 11 2025 at 10:50):

This seems to be a regression of lean#9305... (universe problem..?)

Patrick Massot (Jul 11 2025 at 13:13):

This looks really mysterious. Michael and I investigated a bit, but we give up. Everybody should feel free to clone the nightly branch and create a file containing:

import Mathlib.Data.Finset.Attr
import Mathlib.Data.Finset.Dedup
import Mathlib.Data.Finset.Empty
import Mathlib.Data.Multiset.FinsetOps

open Finset Multiset

section Insert

variable [DecidableEq α] {s t : Finset α} {a b : α} {f : α  β}

/-- `insert a s` is the set `{a} ∪ s` containing `a` and the elements of `s`. -/
instance : Insert α (Finset α) :=
  fun a s => ⟨_, s.2.ndinsert a⟩⟩
@[simp]
theorem mem_insert : a  insert b s  a = b  a  s :=
  mem_ndinsert

theorem mem_insert_self (a : α) (s : Finset α) : a  insert a s :=
  mem_ndinsert_self a s.1

theorem mem_insert_of_mem (h : a  s) : a  insert b s :=
  mem_ndinsert_of_mem h

@[simps!]

def insertPiProd (f : α  Type*) (x : Π i  insert a s, f i) : f a × Π i  s, f i :=
  (x a (mem_insert_self a s), fun i hi => x i (mem_insert_of_mem hi))

/-- Combine a product with a pi type to pi of insert. -/
def prodPiInsert (f : α  Type*) {a : α} (x : f a × Π i  s, f i) : (Π i  insert a s, f i) :=
  fun i hi =>
    if h : i = a then cast (congrArg f h.symm) x.1 else x.2 i (mem_of_mem_insert_of_ne hi h)

/-- The equivalence between pi types on insert and the product. -/
def insertPiProdEquiv  {s : Finset α} (f : α  Type*) {a : α} (has : a  s) :
    (Π i  insert a s, f i)  f a × Π i  s, f i where
  toFun := insertPiProd f
  invFun := prodPiInsert f
  left_inv _ := by
    sorry
  right_inv _ := by
    refine Prod.ext ?_ sorry
    · expose_names
      clear s_1 a_1 f_1 t b β has
      simp only [insertPiProd_fst]
      sorry

theorem insertPiProdEquiv.extracted_1 {α : Type*} [inst : DecidableEq α] {s : Finset α}
  (f : α  Type*) {a : α}  (x : f a × ((i : α)  i  s  f i)) :
  (insertPiProd f (prodPiInsert f x)).1 = x.1 := by
  simp only [insertPiProd_fst]
  simp only [prodPiInsert, reduceDIte, cast_eq]

The last theorem is extracted from the previous one and works. But the previous one fails.

Patrick Massot (Jul 11 2025 at 13:14):

The goal states look identical even with pp.all

Patrick Massot (Jul 11 2025 at 13:14):

The error message is

(kernel) application type mismatch
  @prodPiInsert α inst s f a x i a
argument has type
  i  insert a s
but function has type
  i  insert a s  f i

Eric Wieser (Jul 11 2025 at 16:02):

@Robin Arnez is correct, simp -congrConsts only [insertPiProd_fst] works fine

Robin Arnez (Jul 11 2025 at 16:03):

It's not a universe problem but an instance problem

Robin Arnez (Jul 11 2025 at 16:03):

but it is because of the congr consts

Eric Wieser (Jul 11 2025 at 16:04):

Well, I mean you're correct that that PR is responsible

Eric Wieser (Jul 11 2025 at 16:06):

#check @prodPiInsert.congr_simp is enough to get the crash

github mathlib4 bot (Jul 12 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3d1bc5643ea305c9d448b373a6d849cea86ce3f8).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 12 2025 at 14:24):

lean4#9318 might be enough to fix this. The problem was that proofs could depend on Decidable instances but they weren't being rewritten:

def test {α : Type u} [DecidableEq α] {x : α} (h : (x == x) = true) : Nat := sorry

turned into

theorem test.congr_simp {α : Type u} {inst : DecidableEq α} [inst' : DecidableEq α] {x x' : α} (hx : x = x') (h : (x == x) = true) :
    @test α inst x h = @test α inst' x' h := ...

Robin Arnez (Jul 12 2025 at 14:25):

The fix was to just fix Decidable parameters if proofs depend on them:

theorem test.congr_simp {α : Type u} [DecidableEq α] {x x' : α} (hx : x = x') (h : (x == x) = true) :
    @test α inst x h = @test α inst x' h := ...

This isn't ideal (in particular in other cases) but at least works

Eric Wieser (Jul 12 2025 at 16:07):

Will we see similar trouble for other typeclasses like Fintype?

Robin Arnez (Jul 12 2025 at 18:52):

Decidable is hardcoded specifically to generate stuff like {inst : DecidableEq α} [inst' : DecidableEq α] to allow things like

def abc (p : Prop) [Decidable p] : Nat := sorry

to use

theorem abc.congr_simp {p p' : Prop} (h : p = p') {inst : Decidable p} [inst' : Decidable p'] :
    @abc p inst = @abc p' inst' := ...

Fintype could in theory get similar treatment but doesn't because the generation code specifically checks docs#Lean.Meta.ParamInfo.isDecInst

github mathlib4 bot (Jul 13 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6b84a83a77c7ad02d00f48e07f83be8554d3d3e8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 14 2025 at 09:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (18e1516b655d08e2d7b18b2f47dd73d9040ca6f9).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Jul 15 2025 at 08:36):

This is failing with several errors of the following form:

error: Mathlib/Algebra/Group/Submonoid/Operations.lean:667:2: @[to_additive] failed. Type mismatch in additive declaration. For help, see the docstring of `to_additive.attr`, section `Troubleshooting`. Failed to add declaration
AddMonoidHom.map_mrange:
unknown constant 'AddSubmonoid.map.congr_simp'
error: Lean exited with code 1

Johan Commelin (Jul 15 2025 at 08:36):

Does anyone know how to fix this?

Sebastian Ullrich (Jul 15 2025 at 08:39):

Likely related to #9305, which started introducing these constants. I'd have to refresh my memory on how to_additive is supposed to handle them; maybe AddSubmonoid.map does not exist yet at that point?

Johan Commelin (Jul 15 2025 at 08:43):

It should exist already. Because we're working on map_mrange. So {Add}Submonoid.map is from quite a bit earlier.

Sebastian Ullrich (Jul 15 2025 at 08:43):

I'll take a quick look

github mathlib4 bot (Jul 15 2025 at 08:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2185648684a1e29eea950e4ef6775d509f4f833f).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jul 15 2025 at 08:46):

A #print AddSubmonoid.map.congr_simp before fixes it :rolling_on_the_floor_laughing: ... so probably some incorrect metaprogramming API being used

Sebastian Ullrich (Jul 15 2025 at 08:55):

This might be fixed by #9300, let's test that

github mathlib4 bot (Jul 15 2025 at 10:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b69cf3b739a4a81aa130b6a9a929244fc38ff861).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jul 15 2025 at 11:04):

Sebastian Ullrich said:

This might be fixed by #9300, let's test that

It didn't, but I pushed a Mathlib-side changes that fixes at least the first occurrence

Johan Commelin (Jul 15 2025 at 11:04):

Thanks!

github mathlib4 bot (Jul 15 2025 at 11:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (feb37124118c837cd1a435044964daed952faa4b).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Jul 15 2025 at 12:54):

There's also some whacky change with simp...

error: Mathlib/Algebra/BigOperators/Ring/Finset.lean:125:6: (kernel) application type mismatch
  Pi.cons s a b f a' h
argument has type
  a'  insert a s
but function has type
  a'  insert a s  δ a'

github mathlib4 bot (Jul 15 2025 at 16:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (99ff50ea195c2751509e595d56b079dd94354e7c).
You can git fetch; git checkout nightly-testing and push a fix.

Eric Wieser (Jul 15 2025 at 16:59):

That one was identified already in another thread, it's to do with the congruence lemmas being illegal

github mathlib4 bot (Jul 15 2025 at 17:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b8f4aea6110b56abedade4d7d75aa18804f0512e).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Jul 15 2025 at 19:12):

Eric Wieser said:

That one was identified already in another thread, it's to do with the congruence lemmas being illegal

What thread?

github mathlib4 bot (Jul 15 2025 at 19:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (38f7e1292c9e93fd6f374095429b0c907a87f253).
You can git fetch; git checkout nightly-testing and push a fix.

Patrick Massot (Jul 15 2025 at 22:53):

I think Eric means #nightly-testing > Mathlib status updates @ 💬

Patrick Massot (Jul 15 2025 at 22:53):

which is the same thread but an earlier message.

Eric Wieser (Jul 15 2025 at 22:54):

And lean4#9318 was the proposed fix

Johan Commelin (Jul 16 2025 at 05:01):

And Leo just merged lean4#9395 which should also fix this

github mathlib4 bot (Jul 16 2025 at 09:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a7a7ce073039c7c472592d31dfb972b61e196efc).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Jul 16 2025 at 10:35):

$ lake exe cache get
... snip ...
If you push your commits to a branch of the mathlib4 repository, CI will build the oleans and they will be available later.

That sentence needs some updating. But grepping through the source, I didn't find it.

Johan Commelin (Jul 16 2025 at 11:32):

I'm confused by the :cross_mark: from CI. Locally nightly-testing seems to build fine.

Sebastian Ullrich (Jul 16 2025 at 11:34):

It's #nightly-testing > bot not running CI again, super confusing

github mathlib4 bot (Jul 16 2025 at 12:17):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (da62c86042859cdb68ba036dd10a1348f4563127).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Jul 16 2025 at 13:01):

Anyways, I'm still getting

error: Mathlib/Combinatorics/SimpleGraph/Turan.lean:258:35: (kernel) application type mismatch
  @IsTuranMaximal V inst✝³ G inst✝¹
argument has type
  DecidableRel G✝.Adj
but function has type
  [DecidableRel G.Adj]    Prop

on the latest nightly...

Sebastian Ullrich (Jul 16 2025 at 13:14):

I reverted my workarounds, this failure actually looks a bit different from the others. Could you check whether it is the only one? We should report it in that case.

Sebastian Ullrich (Jul 16 2025 at 13:15):

And feel free to reapply the workaround in the meantime

github mathlib4 bot (Jul 16 2025 at 13:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c1264bd85e7c6473bbf1a7a24a3ea1b056e6aa79).
You can git fetch; git checkout nightly-testing and push a fix.

Johan Commelin (Jul 16 2025 at 13:36):

@Sebastian Ullrich locally it indeed seems to be the only failure

github mathlib4 bot (Jul 17 2025 at 08:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b621bb78764633b7ae68d98f9de15ac22805f731).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 17 2025 at 09:50):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (3935d86a432f8ffe32f17ea00c12e090cf1df6de)

Johan Commelin (Jul 17 2025 at 10:03):

@Sebastian Ullrich Wait? What happened? Did you magically fix something?

Sebastian Ullrich (Jul 17 2025 at 10:03):

I only put my workarounds back in place for now

Sebastian Ullrich (Jul 17 2025 at 10:04):

That is, the ones Leo hasn't already addressed

github mathlib4 bot (Jul 17 2025 at 13:38):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (3935d86a432f8ffe32f17ea00c12e090cf1df6de)

github mathlib4 bot (Jul 18 2025 at 09:46):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (44e5df9a4f8aaaf07d6ff1be692c0cf06c1d48a6)

Robin Arnez (Jul 22 2025 at 10:06):

Did this break for some reason?

Robin Arnez (Jul 22 2025 at 10:08):

Some outdated tokens or something?

Bryan Gin-ge Chen (Jul 22 2025 at 12:28):

Uh oh, I tried to refresh one of the tokens but I may have screwed something up. Let me check.

github mathlib4 bot (Jul 22 2025 at 12:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (20145bdb2fe6ee3e430187b69b1597f83a85c49c).
You can git fetch; git checkout nightly-testing and push a fix.

Bryan Gin-ge Chen (Jul 22 2025 at 12:36):

OK, it's back now. Thanks for pointing this out, Robin!

github mathlib4 bot (Jul 23 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (34a2f348f0b09367f34a550686e38d00b17bdc37).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 00:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b420ac7884e612813bb08447834f5d1511199dad).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 01:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c318e73ffde2c0cee9c110a0f5599326a038cdcf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 04:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6f2781891be2ca1de18fd1af1f58f46f29fcb734).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 06:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6e06a7a0f91ab256b935f84de538bf5e7c5e92f7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 06:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d8dfcdd20e0372c3c9c0e9d1e4a6d359b263de34).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 07:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (98272387219f06d50f58f9b43a6e5d566e20a69f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 13:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f641e8ef65cbf0b3bb058fd2132fa0ba210c0cc0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 14:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (95e6b1288b79201efe878b13170af923f9e5049e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 18:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9bbc530f4c22f15283466d7a6f84fd2e3421dab8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 23 2025 at 21:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (04ce2295625838a375fbfe8a2048d583a9c2824a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 24 2025 at 01:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (beae12d2f599bfd9cccaa108db63eb42864cf6c8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 24 2025 at 01:46):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (08872da5eaa35fa7972f97f1f41efd1b64c0c8f4)

github mathlib4 bot (Jul 24 2025 at 04:45):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Jul 24 2025 at 07:37):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (08872da5eaa35fa7972f97f1f41efd1b64c0c8f4)

github mathlib4 bot (Jul 24 2025 at 08:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (91fc2ce00feb3e9969154d3fcb0606b6d097f5be).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 24 2025 at 12:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1f9ac127232cfd3a61b68dd853a800d3640ef3a6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 24 2025 at 15:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cab90a41d93b59b75c90e6678bd1790cb5a8e0b5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 24 2025 at 21:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6346f82037a4c5ff90909ec00dd88abec281d5ff).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 24 2025 at 23:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (de511720dc870f3c2ebed9dd41f91d964ae27dca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 25 2025 at 00:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d171db5a72b9542ade85a31277a9b02bf056720d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jul 25 2025 at 03:25):

I made a mistake in changing the definition of Lean.Grind.Field, nightly-testing will be broken until the new nightly in a few hours.

github mathlib4 bot (Jul 25 2025 at 04:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (166f090148fb24cb3c48e821f26ef576ce1fca6f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 25 2025 at 09:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5d2b55f7404a021f0ca43144d6070cb4c24fa61d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 25 2025 at 10:25):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (15c20f8e14302f8100c32c69e6dedccce114e2ac)

github mathlib4 bot (Jul 25 2025 at 13:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (33579c0836cc407d6952852c274042552084c083).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 25 2025 at 16:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e9eeaf4e7570a706db3e588f637f5a05cb637bb8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 25 2025 at 16:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5927597cca90cf9013842f783f3b73514c103700).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 25 2025 at 17:46):

Hmm cache doesn't work for nightly-testing PRs
Edit: it works but very inconsistently

github mathlib4 bot (Jul 25 2025 at 18:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a210381b8190ab77d022686ce6ce9c2cfde31f5e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 25 2025 at 21:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fd71efe621a526c826578116ae29a06544ec2ac9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 26 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d2b567f6675d5724613e1f91c4415e48361ae3b2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 26 2025 at 03:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (692c705661365aa50ec0db5fff36381f48ba36d9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 26 2025 at 06:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (20c3cefcfb32013a122512123ee853a5e73423e8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 26 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (300d6ec2fdc036898f7ca0070bf5d91909df0bb2).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 26 2025 at 09:25):

We have a lot of lost commits in nightly-testing so I'm trying to restore them in nightly#16

Robin Arnez (Jul 26 2025 at 09:26):

My plan is to start with reverting everything to upstream/master and then slowly adding back nightly-testing changes until it starts building again

Robin Arnez (Jul 26 2025 at 09:27):

I'm currently stuck at Mathlib/Geometry/Euclidean/Congruence.lean and Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean

Robin Arnez (Jul 26 2025 at 09:27):

Mathlib/Geometry/Euclidean/Congruence.lean has an internal grind failure,

Robin Arnez (Jul 26 2025 at 09:27):

Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean has a simp_all failing that should (?) work

Robin Arnez (Jul 26 2025 at 09:29):

If anybody knows which nightly adaptations I might be missing, please tell me

github mathlib4 bot (Jul 26 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3ea0bcb9098126552ff4ffe6e78d36138dd579c3).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 26 2025 at 13:21):

Update: Mathlib/Geometry/Euclidean/Congruence.lean is the only failing file now, might be a grind bug but I'm not sure

github mathlib4 bot (Jul 26 2025 at 13:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a9b5dffa2820cffd96797f9450cc47bdbc5d4591).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 26 2025 at 14:48):

Okay, managed to reduce the problem it to lean4#9562

github mathlib4 bot (Jul 26 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (33f427f4deb852e28bd134f729dd751b69a8cf32).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 26 2025 at 18:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0da1986c08bded96f8e9297161bbda37de20b496).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 26 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4187b61039f897afdf144a9c4a934ad4c74743bb).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jul 26 2025 at 22:47):

Robin Arnez said:

We have a lot of lost commits in nightly-testing so I'm trying to restore them in nightly#16

What happened?

github mathlib4 bot (Jul 26 2025 at 23:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (018899d73b30601afd3a1ea99263ecf01e89fa3e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 27 2025 at 00:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (874718b8e79f6f277d22ba29e0a54e9685998385).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 27 2025 at 02:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cbd41d9ad73a021f2aacd25470808e21d34a562a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 27 2025 at 03:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (04ee432c20cf5d81cde4db377ad870b2b82ae761).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 27 2025 at 06:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f55f4ddb29bdfcf56213f642a0b43f781ea874fa).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 27 2025 at 06:58):

Kim Morrison schrieb:

Robin Arnez said:

We have a lot of lost commits in nightly-testing so I'm trying to restore them in nightly#16

What happened?

I'm unsure but from what I can tell these changes have been merged but the conflict resolution just dropped them or something

Robin Arnez (Jul 27 2025 at 06:58):

Maybe we should change our conflict resolution strategy to "prefer mathlib4 files but keep lean-toolchain and lake-manifest.json"

Kim Morrison (Jul 27 2025 at 07:05):

Previously I've thought that it was less confusing if we preserved changes that have been made already on nightly-testing. It seems easier to me to restore things from master than to restore things from the nightly-testing history (precisely because the nightly-testing history is a messed, and unreviewed, whereas anything you take from master is "good").

Robin Arnez (Jul 27 2025 at 07:26):

Hmm well the problem was definitely also the failed merge commits before

Robin Arnez (Jul 27 2025 at 07:27):

It seems like 33579c0836cc407d6952852c274042552084c083 actually "merged" some of the changes that got lost

Robin Arnez (Jul 27 2025 at 07:27):

maybe this is a git quirk? Hmm, not sure

Robin Arnez (Jul 27 2025 at 07:30):

Oh yeah 33579c0836cc407d6952852c274042552084c083 messed up a lot

Robin Arnez (Jul 27 2025 at 07:31):

It was supposed to change 610 files but only changed 28

Robin Arnez (Jul 27 2025 at 07:31):

and there were only 2 conflicts?

github mathlib4 bot (Jul 27 2025 at 07:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (38c4645f88e4dd56395502f75374e86236879fdd).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 27 2025 at 08:09):

Oh no the merge master to nightly only checks out the repository at depth 1

Robin Arnez (Jul 27 2025 at 08:09):

No wonder funny quirks occur

Robin Arnez (Jul 27 2025 at 08:14):

Okay #27533 should fix it for real this time

Robin Arnez (Jul 27 2025 at 08:59):

I just realized that because only that one merge commit was bad I should've just reverted that one and done the merge myself (nightly#18)

Robin Arnez (Jul 27 2025 at 08:59):

But we should probably merge #27533 before another "Merge master to nightly-testing" happens

github mathlib4 bot (Jul 27 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3151d47630dd4f675c9624fe18da6ebc5e557ae1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 27 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d18ab42522e7f5ac7552057f484e5bcc1cebc517).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 27 2025 at 10:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (29dfa79b7e340b8963af06e25f525a8343e501ca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 27 2025 at 11:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d2b26006d0eedded5ce0128e8ad9b992453a710f).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 27 2025 at 11:34):

It's maybe easier if we don't do it both at the same time? nightly#18 seems to work fine by now

Kim Morrison (Jul 27 2025 at 11:39):

@Robin Arnez, I'm hesitant to merge something like nightly#18, because it contains both a huge blob of merged code from master, and your subsequent tweaks to it.

Kim Morrison (Jul 27 2025 at 11:39):

I would much prefer the merge happens first, and the fixes separately.

Robin Arnez (Jul 27 2025 at 11:40):

You can also

git branch nightly-testing-test 15c20f8e14302f8100c32c69e6dedccce114e2ac # one commit before the bad merge
git merge --squash upstream/master
git merge testing/nightly-testing

yourself if you're more comfortable with that

Kim Morrison (Jul 27 2025 at 11:42):

Okay, I've merged... I need to go to bed I guess anyway. :-) Thanks for the help, and sorry for the lack of coordination. We should setup better processes so it's clearer. I didn't see you PR until just now.

Robin Arnez (Jul 27 2025 at 11:43):

Just one more thing: #27533 didn't quite merge correctly, I assume a bors retry or something is necessary?

Kim Morrison (Jul 27 2025 at 11:46):

I think that bors output actually means it is still in progress.

Kim Morrison (Jul 27 2025 at 11:46):

#bors

Kim Morrison (Jul 27 2025 at 11:47):

Maybe not. I'll bors r+ now.

github mathlib4 bot (Jul 27 2025 at 12:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (303b31d2a6aa270ef008be0326d63ec94a9f7998).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Jul 27 2025 at 15:06):

Finally, we have nightly#19 building (except cache, which is still broken). Another nightly-with-mathlib coming soon!

Robin Arnez (Jul 27 2025 at 19:05):

https://github.com/leanprover-community/mathlib4/actions/runs/16551252134/job/46806399939
The "Merge master to nightly" workflow seems to be missing some permissions

Robin Arnez (Jul 27 2025 at 19:08):

Specifically the permission to change the "Merge master to nightly" workflow :-)

Bryan Gin-ge Chen (Jul 27 2025 at 19:27):

I think @Kim Morrison will need to update the token permissions here since the 2FA notifications for leanprover-community-mathlib4-bot go to them. I updated the notes in #passwords, but basically we need to add the "workflow" scope to "mathlib4 NIGHTLY_TESTING".

Bryan Gin-ge Chen (Jul 27 2025 at 19:39):

OK, I just attempted to merge master into nightly manually, hopefully everything went well.

github mathlib4 bot (Jul 27 2025 at 20:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (865f164be02289b17095d9b2107db225b0c667fe).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 27 2025 at 22:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (75f7e70f4c79252b2822990d631822a6ad9363f1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Jul 27 2025 at 23:31):

Okay, I have updated that token, and installed it as a secret, per #passwords.

Kim Morrison (Jul 27 2025 at 23:31):

(And merged nightly#19)

Kim Morrison (Jul 27 2025 at 23:43):

Robin Arnez said:

Okay, managed to reduce the problem it to lean4#9562

This was fixed in lean4#9578.

github mathlib4 bot (Jul 28 2025 at 00:05):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (257ccd813b5753f70ed278e63212cf1d172f7f08)

github mathlib4 bot (Jul 28 2025 at 00:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f7ade977be08078a3e8bfec3a3956a434eadda30).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 28 2025 at 00:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a1f446eb4a9431e8513aa7bbcd30d8d14e1a4f05).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 28 2025 at 01:47):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (257ccd813b5753f70ed278e63212cf1d172f7f08)

github mathlib4 bot (Jul 28 2025 at 08:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (01645a8321aea0e49534a90b86707974caf1e7ad).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 28 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a1877a8cf3bdbe5d99f316831ab88a8320fa6a93).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 28 2025 at 11:42):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (44bab86fc836b21dbf5303db4f107dd8d57a7bf7)

Kim Morrison (Jul 28 2025 at 12:22):

Notice to users of nightly-testing: @Mac Malone is testing some changes to the caching infrastructure, and using the nightly-testing branch to do so. Don't expect the cache to be reliable on nightly-testing in the near future. :-)

Kim Morrison (Jul 28 2025 at 12:50):

@Mac Malone the cache upload in nightly-testing is not working, see https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/16568879407/job/46855597666#step:22:3592

Credential sigv4 header should have at least 5 slash-separated parts, not 1

Mac Malone (Jul 28 2025 at 12:51):

Yep, I noticed that. Seems like we need to back out the change and I need to debug the FRO cache setup.

Kim Morrison (Jul 28 2025 at 12:52):

I think you have write access to the branch, can I leave it to you to revert?

Robin Arnez (Jul 28 2025 at 12:55):

Just a quick reminder that we can also revert the commenting out in Mathlib/Geometry/Euclidean/Congruence.lean now that we're on nightly-2025-07-28

Kim Morrison (Jul 28 2025 at 13:18):

Done.

github mathlib4 bot (Jul 28 2025 at 13:58):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (44bab86fc836b21dbf5303db4f107dd8d57a7bf7)

github mathlib4 bot (Jul 29 2025 at 09:41):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (ee1994d1ce21f0a4df25782e30eb48ab2024291f)

github mathlib4 bot (Jul 29 2025 at 16:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (731ffc9dc33d247924bff4ccb6a63c4ec9bb746a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 29 2025 at 22:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5eb1c137ad262339f0bb67c79bb9503fe1fcabc8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 30 2025 at 01:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (bc680c70ac35673b95d89c734a773e6bdfb8091e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 30 2025 at 04:52):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (ee1994d1ce21f0a4df25782e30eb48ab2024291f)

github mathlib4 bot (Jul 30 2025 at 04:52):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

Kim Morrison (Jul 30 2025 at 07:21):

That URL is missing the master after blob...

github mathlib4 bot (Jul 30 2025 at 09:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c02367d055012fc8c8b5c2eaf2d44b15779faa82).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 30 2025 at 13:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2eebb74a805646ede4f312f8e8a68cafbc1be24c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 30 2025 at 22:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3302efb3f4ae3befa9869b2c099bb14812acf94c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 31 2025 at 00:10):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (4ad95cf1699e4a24612145830975c0adfc27d2ed)

github mathlib4 bot (Jul 31 2025 at 00:10):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Jul 31 2025 at 01:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (30de3e432005e777c9ee809f5c2160dca493fe04).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 31 2025 at 02:45):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (4ad95cf1699e4a24612145830975c0adfc27d2ed)

github mathlib4 bot (Jul 31 2025 at 02:45):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Jul 31 2025 at 04:49):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (4ad95cf1699e4a24612145830975c0adfc27d2ed)

github mathlib4 bot (Jul 31 2025 at 04:50):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Jul 31 2025 at 06:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (16343f7f9e5ae34ffb0065036b5dddde45a582cf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 31 2025 at 08:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e75d688816b826834de24447b5f1161c384d7fed).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 31 2025 at 11:53):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e9b6d7c7bf68aec35feadf75e134c35db2a0170f)

github mathlib4 bot (Jul 31 2025 at 11:53):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Jul 31 2025 at 13:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (101715d4df32f28088d0c1ac393f1a302ac37844).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 31 2025 at 16:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3747b7ba3d8e7b8a4e753752e02852c1b1320e3a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 31 2025 at 19:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (36a043cd21c27a378a3bab774fece49b34bdc053).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Jul 31 2025 at 21:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (983138476716864b69da915de5b787d5d4ca889e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 01 2025 at 00:10):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e9b6d7c7bf68aec35feadf75e134c35db2a0170f)

github mathlib4 bot (Aug 01 2025 at 00:11):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Aug 01 2025 at 01:45):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e9b6d7c7bf68aec35feadf75e134c35db2a0170f)

github mathlib4 bot (Aug 01 2025 at 01:46):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

Kim Morrison (Aug 01 2025 at 01:50):

github mathlib4 bot said:

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

Hopefully resolved by #27793.

github mathlib4 bot (Aug 01 2025 at 05:01):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e9b6d7c7bf68aec35feadf75e134c35db2a0170f)

github mathlib4 bot (Aug 01 2025 at 05:01):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Aug 01 2025 at 07:30):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e9b6d7c7bf68aec35feadf75e134c35db2a0170f)

github mathlib4 bot (Aug 01 2025 at 11:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d1435a4cd5ae6ebcfd0be14d129ee52aaf508fc6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 01 2025 at 16:33):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (8d5ff4faaeba47cc2573d5d61a49b7391a2cb272)

github mathlib4 bot (Aug 02 2025 at 09:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (95260f8bb65a6b6fd87951fe5e4c1cca06be8dcc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 02 2025 at 10:33):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (a12f25fd5923181dd4b9452c5785cacf5a3b9424)

github mathlib4 bot (Aug 03 2025 at 08:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (324922f6f5e664a588465e2ff5274e973ea7abbb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 03 2025 at 10:33):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (79a314b098441b3c3a91abdc6bd42cc49785da5d)

github mathlib4 bot (Aug 03 2025 at 21:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (de754d94feadf983389f00dcb03d21394616542a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 03 2025 at 23:11):

For me, lake exe cache get on nightly-testing is currently failing with

 [2/2] Running proofwidgets:release
error: failed to fetch GitHub release (run with '-v' for details)
Some required targets logged failures:
- proofwidgets:release

(Running with -v doesn't provide any additional information: @Mac Malone, is this something we need to fix?)

Could someone try to reproduce?

Kim Morrison (Aug 03 2025 at 23:17):

Hmm, after a few more attempts the problem has disappeared.

github mathlib4 bot (Aug 04 2025 at 00:36):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (79a314b098441b3c3a91abdc6bd42cc49785da5d)

github mathlib4 bot (Aug 04 2025 at 00:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1da9e28ff8544b902aaf17cd01a3e5eb17d3c2d6).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 04 2025 at 02:15):

Merging batteries-pr-testing-1306 into nightly-testing now.

github mathlib4 bot (Aug 04 2025 at 03:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (75f6391292209c95cea0c2337455ab5ce2d0be6f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 04 2025 at 04:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (948559c90f0a77c86665cd1ce44a2147868ebc50).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 04 2025 at 07:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (63b1cf7b8f259bc082e77b3e3a1514d9f7df1ca3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 04 2025 at 10:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2b58bf82a8da8d6d1ec4bb3dc62d2e50bc6ad8db).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 04 2025 at 13:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7aff3db2ef9522cc0396757ac18455ffbac0769f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 04 2025 at 14:02):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (efb1ad60cc856e8a021ed33c99bdded07cf6a967)

github mathlib4 bot (Aug 05 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (222bed4d037140c84a5796ad0af0eae3f52976ea).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 05 2025 at 10:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fb72f53a7453a639349e5341aefe239d1ba446f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 05 2025 at 13:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (85d25dfca4fd8f526b6bfd94eca840c69660456e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 05 2025 at 16:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (581d554b50c44fa1289033f6040ca85a226dfae8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 05 2025 at 19:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (44f3045a402187693a092391d47b04d1250ee68f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 05 2025 at 23:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (52dadd72ff8514441c1ba6365a3aa0f72a045bb2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 06 2025 at 00:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5cce686f41127236c9685f93816eb4bc929cf3ae).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 06 2025 at 01:39):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (6de9b2a206a6a36bcbc2abf7853a05086342a542)

github mathlib4 bot (Aug 06 2025 at 09:41):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c0f7deeff2ef123138077bc358816adb702cab09)

github mathlib4 bot (Aug 06 2025 at 16:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ad9e4e1c867ad56020a03f761c2ecd4ce328bbcc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 06 2025 at 19:20):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a97f06097c3fa1d6b2efac443a3eacd0d7ff9d00).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 06 2025 at 22:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8587cf664a80bd1dbe4703cb22b7733d1fe15ef4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 07 2025 at 00:35):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c0f7deeff2ef123138077bc358816adb702cab09)

github mathlib4 bot (Aug 07 2025 at 09:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (595b152f77fc4171759de9389b40fcd19e3125c9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 07 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4523a85ae79c3ff4786e8cb955a1997d17a76c51).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 07 2025 at 12:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f319c3d748dcbeb40c2c0f95bdcfcee711eeeef2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 07 2025 at 15:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (244bc0e47c6093e3d3d2f17d2b9c55120e0a2269).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 07 2025 at 18:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b5ea6ed998d3840201ba2f1fdbb294fd98c8efc4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 07 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8aa3037f12d96348eb37e04dd0e921342b3e6584).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6ffc3538e40e28a9b7c379a6870bef82f470bc6f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 03:17):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (53594a5427ee279d5d88eecf589beba63781d533).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 03:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (15b8ed5856b691e8127824294c5571d3de70f9e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 04:15):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d599424ab411e464570ff11b2e6e20359c83188e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 06:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (19fbde5aeeb12a89caa8d7bf2f93be2f3c94711c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 09:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (030a1ee3679099d4707bce3a0f63090b180343f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7ee0a37e03c3e0b2f5df09b80cd5857f9ad65583).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 12:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ef7a10e5edecfce4e390b62c04094270ec68d3bf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 15:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5e881c57a51b881e2acefa3a1ebb6eccd78f0fd7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 18:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ade22f56fff6b166fe87f98efd5f4fa126908c3c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 08 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (80c6f5adef66e9c37ab7316763850a6659bdeb1c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 09 2025 at 00:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (12ba9658cc7c0dc610d6e940eee18265f84d9daa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 09 2025 at 06:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (069327597ab4f911ea0748ccfab5a0d851fa8345).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 09 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0e84a01812f3d094038354d15cb049b6a43704f4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 09 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (81f21dee9e18c85861e80d4fd18132c05853782d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 09 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ac1f250102a3c1c6d129bc8a615f2b9930588c4e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 00:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cec6094d61c9e92c1932dbf91d29dc9ecd10c620).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 03:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (91319379db41d1fa4fc2d83b45cc88885f9677dd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 06:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (723c971a3bf3bd1a706e6d104e2d81264f067a78).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 08:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (13a4683455a988bfdf47e927325b5abacfb0ec78).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (88b82b755e7a1474113ea438476569927f996f8b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 09:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9f95d0fe928d89ab75216f3b17a74024a1b3e096).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 12:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (231422eb2e32001ea63c31547ca2fbf692268d88).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 15:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f5acf40f45a439105d076f2ab591781d53c7934f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 18:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e769cc13c16fad58101b13b7d6fb11ee2f536f3c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 10 2025 at 21:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e0f9f4a18ffd4602b607b255c0d6f77f54205166).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 11 2025 at 00:03):

Finally starting on this again.

github mathlib4 bot (Aug 11 2025 at 00:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a44dc2fe122a64269c2cb2fbf5f7b08bc96a364e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 11 2025 at 00:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3eff1247619b125f963f58b38c8a77e8fd40dd44).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 11 2025 at 02:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (39495562c74300b71e3e98dfc765c7b047584cc2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 11 2025 at 04:13):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b3c5da5aa7c82275bd6afe434ca4a12cca851c5a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 11 2025 at 05:28):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (4391fe7dabfd4bd01c40669ea759cef39d652948)

github mathlib4 bot (Aug 11 2025 at 09:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a89da126f55358ae88b508d47a67eae55098e55f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 11 2025 at 10:29):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c70e7a7dfbef3a1c25a3fa27ed699400ca82df64)

github mathlib4 bot (Aug 11 2025 at 11:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (49e9c0996c37288637914ba7fda536047dcd40bb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 11 2025 at 11:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (980076ee736e2880c0fe28447cc2235308feeb53).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 11 2025 at 13:42):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c70e7a7dfbef3a1c25a3fa27ed699400ca82df64)

github mathlib4 bot (Aug 12 2025 at 00:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (71588a4f9dc01b89fbea0073bbffd02da6397c83).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 01:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b7b2ebff165c60d6d3a12dedf842c4b51f719dbb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 04:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f1bb1583984e3554d81c43dd2c434cfd61ade778).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 07:20):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (17929540e69505ec47f8ac16bc5e49d151a4998b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 09:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5eae025749fc0fe7ad7fd46e4fa429f124e0bec2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 10:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (126d9b5c6ffe8878a0683b7672dc31f405dd2333).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 13:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e6eb83f9e00790ab81b50b7640d112d93b60f9b6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 16:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5e6393311222007801efc43b5c7f25eeec0570a8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 19:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f54ccae0db8664989563bf49756dcb3f2c530e2b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 12 2025 at 22:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (84943f37f4c2a564c72927dc1eea846d813d13fe).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 12 2025 at 23:46):

@Mac Malone, as far as I can see this is "just" cache issues. We are getting very close to the line for a release --- what are next steps here? Shall I revert your changes to use the new cache backend?

Kim Morrison (Aug 12 2025 at 23:47):

Locally I can lake build Mathlib Archive Countexamples && lake test && lake lint, so hopefully we're otherwise good to go for release tomorrow.

github mathlib4 bot (Aug 13 2025 at 01:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3369322d09700e3f21ec4ffc10aa126c522ab3ab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 13 2025 at 03:13):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0365d54a62b46417f32e6cdab5e3a24a48979100).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 13 2025 at 03:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7c6202bf661ffb79a69ac63ac8ceca9189de24f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 13 2025 at 04:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d700790ae7de5caf9ae16dbe689aa3bbcb671ce1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 13 2025 at 05:30):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9e1fd7ccc418c5437ca6a6bd29d10c6924f18299)

github mathlib4 bot (Aug 13 2025 at 10:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7b917fe2fc55921f54786560b4a22ed67dab3307).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 13 2025 at 12:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (203219dda688bbebb9bd62e4064dfb061caec6fc).
You can git fetch; git checkout nightly-testing and push a fix.

Bryan Gin-ge Chen (Aug 13 2025 at 12:05):

@Kim Morrison I just pushed a few commits here fixing some grind warnings. I also added back the grind proofs I removed in #28272 (and checked that they were all indeed deterministic).

Kim Morrison (Aug 13 2025 at 12:35):

Thanks, @Bryan Gin-ge Chen!

Kim Morrison (Aug 13 2025 at 12:35):

I'm hopeful this one can become v4.23.0-rc1 tomorrow, it's looking good.

Kim Morrison (Aug 13 2025 at 12:35):

I just pushed a fix to the tests, so hopefully we get a :check: shortly.

github mathlib4 bot (Aug 13 2025 at 13:50):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (38ae17aa6cd305a4e6c265a1939c67376499066a)

github mathlib4 bot (Aug 14 2025 at 07:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a80352557fc69c487189365c1b3d5bd8e8589dc0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 14 2025 at 09:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b607cb8d7253f20572d493fdb4a1d40606924df5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 14 2025 at 09:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e2bcf7f9d254c8bff41bb90364e7fd1aa32713c3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 14 2025 at 10:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6fae542614a73d493091166cbee8f77ddf29bdc9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 14 2025 at 12:22):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (0954551f84596d579803a24ae8efdd3da8eaa49a)

github mathlib4 bot (Aug 15 2025 at 01:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1802d43d481ee637365f686b79fb75cfbbfd7b80).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 15 2025 at 04:47):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (0954551f84596d579803a24ae8efdd3da8eaa49a)

github mathlib4 bot (Aug 15 2025 at 06:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (bce5646a249d57f396d2be80129b3ba80a1c290b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 15 2025 at 09:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5a7f0092eb63d306553773a79290d32b0b1df773).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 15 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ae35a9be15a5b3292aeeb5fe5c28b11f42cf879a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 15 2025 at 18:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9c2e2755a0608da18785504a4a3d7c7c3d706d0c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 16 2025 at 00:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (21eaaf30472a9e163249e0aa7a0e2faee1b4e5b1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 16 2025 at 03:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (51610399cab6d6339aec0455d9abc325265ec073).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 16 2025 at 06:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2a3c5071d7330bc711898496e18002f4a4719c98).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 16 2025 at 08:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cc1a5df20bb481d3b2f86501315c4c1f9723d33a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 16 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2d1a8f1255bb3552068e87ac9afda15365d79e93).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 16 2025 at 10:42):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9c555129b68629832c422698eb2f326220df1395)

github mathlib4 bot (Aug 16 2025 at 13:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (41c1e3c32c473c1c207585b6791e0659766d67f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 16 2025 at 16:13):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9c555129b68629832c422698eb2f326220df1395)

github mathlib4 bot (Aug 17 2025 at 10:25):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (a777e305e9c1fcb7a3225e3a17ce0fb2ff5d5789)

github mathlib4 bot (Aug 18 2025 at 09:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (839d025f00c4c6a37c9fdf95421a65ab939eeff7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 18 2025 at 10:35):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (16cb4390726f8ec8e7bfa8e9edf73221398a51bc)

github mathlib4 bot (Aug 18 2025 at 16:58):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (c46e3b0c5bc5e724f0f1de6a367c370a553db587).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 18 2025 at 19:24):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (16cb4390726f8ec8e7bfa8e9edf73221398a51bc)

Kim Morrison (Aug 19 2025 at 01:55):

github mathlib4 bot said:

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (c46e3b0c5bc5e724f0f1de6a367c370a553db587).
You can git fetch; git checkout nightly-testing and push a fix.

Ooh, exciting! Who made this happen?

The failed link is broken, and the instructions afterwards probably need tweaking, as these failures are likely problems in doc-gen4 and/or lean, rather than in Mathlib.

github mathlib4 bot (Aug 19 2025 at 02:16):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (3c73a38c40c2acb5295d86bb1240494a384e46e6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 19 2025 at 04:41):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (16cb4390726f8ec8e7bfa8e9edf73221398a51bc)

github mathlib4 bot (Aug 19 2025 at 08:37):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (956f99f90395a67ef4c7aca39e2d679981a9dacc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 19 2025 at 08:49):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (16cb4390726f8ec8e7bfa8e9edf73221398a51bc)

github mathlib4 bot (Aug 19 2025 at 08:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7ad7be828ee6c5210a459b0f792ed53d820721a1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 19 2025 at 09:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3403dce19e9785bffe718d3392da65f063741d8d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 19 2025 at 10:11):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (3403dce19e9785bffe718d3392da65f063741d8d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 19 2025 at 12:12):

Kim Morrison said:

github mathlib4 bot said:

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (c46e3b0c5bc5e724f0f1de6a367c370a553db587).
You can git fetch; git checkout nightly-testing and push a fix.

Ooh, exciting! Who made this happen?

The failed link is broken, and the instructions afterwards probably need tweaking, as these failures are likely problems in doc-gen4 and/or lean, rather than in Mathlib.

Just trying to track this down: @Anne Baanen, did you implement this?

Bryan Gin-ge Chen (Aug 19 2025 at 12:24):

Seems so, here's the workflow file: https://github.com/leanprover-community/mathlib4-nightly-testing/blob/nightly-testing/.github/workflows/nightly-docgen.yml

github mathlib4 bot (Aug 19 2025 at 13:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (63d442dd22d058e4de00de339f34bdb6f905d63d).
You can git fetch; git checkout nightly-testing and push a fix.

Anne Baanen (Aug 19 2025 at 14:30):

Kim Morrison said:

Kim Morrison said:

github mathlib4 bot said:

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (c46e3b0c5bc5e724f0f1de6a367c370a553db587).
You can git fetch; git checkout nightly-testing and push a fix.

Ooh, exciting! Who made this happen?

The failed link is broken, and the instructions afterwards probably need tweaking, as these failures are likely problems in doc-gen4 and/or lean, rather than in Mathlib.

Just trying to track this down: Anne Baanen, did you implement this?

Yes, that's my docgen testing workflow! Still working on getting the action working as expected (since nightly-testing needs a bunch of custom configuration). Will fix the error message before I continue testing.

github mathlib4 bot (Aug 19 2025 at 14:46):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (ed1405f731c8a8c89e6d1317fb383ed23df808bc).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

github mathlib4 bot (Aug 19 2025 at 14:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ed1405f731c8a8c89e6d1317fb383ed23df808bc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 19 2025 at 16:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1df36c362cc51134376cab36d5bda86533bc0b0c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 19 2025 at 18:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (21aef280d1e29dbb2d5d55143951b3be52d4e3e6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 19 2025 at 22:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (11ae10f3a900943f41ad857d10bf89ea9bcd2ce6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 19 2025 at 23:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (89245ba6061a40a3aa36ac0743854ee6169cdb73).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 01:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1bad8a43a00d83b09c033407d9ccd53668840400).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 02:28):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (e373c7e9ef4583d448f9d2a3861dfda1c6701dad).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

github mathlib4 bot (Aug 20 2025 at 02:34):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e373c7e9ef4583d448f9d2a3861dfda1c6701dad)

Kim Morrison (Aug 20 2025 at 02:38):

github mathlib4 bot said:

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (e373c7e9ef4583d448f9d2a3861dfda1c6701dad).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

Oh, interesting, the doc-gen4 build catches:

  error: Mathlib/Algebra/Order/CauSeq/Basic.lean:438:2: Tactic `simp? [not_forall]
     at nk` produced `simp only [gt_iff_lt, ge_iff_le, not_exists, not_and, not_forall, Classical.not_imp, not_le] at nk`,
  but was expecting it to produce `simp only [gt_iff_lt, ge_iff_le, not_exists, not_and, not_forall, not_le] at nk`!

  You can reproduce this error locally using `set_option says.verify true`.
  error: Lean exited with code 1

but the main nightly-testing build doesn't! This check on says statements only runs when CI=true. I guess somehow this is no longer set in our CI run (ah, because of landrun!) but it is when run via lean-action in the doc-gen build.

Kim Morrison (Aug 20 2025 at 02:42):

I've fixed this in nightly-testing, but we should:

  1. tunnel CI=true through landrun
  2. consider just deprecating says as a failed experiment

github mathlib4 bot (Aug 20 2025 at 03:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e7f484e7b12e416f6557483142c81d58ef36ba9b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 03:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c5e64fb301ff728635e2a9101f734c69d2542e23).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 04:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4f3d0aea5253552ddbbedf8edbefc6da109895b0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 06:45):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e373c7e9ef4583d448f9d2a3861dfda1c6701dad)

github mathlib4 bot (Aug 20 2025 at 08:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e28a7091153beedcbe25efa29dee38248ed96d8d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 08:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5b096de4fab972769073aa38cd76c9abc844ab8a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 09:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (354465c05bd223d54ae700b80cbed67a72deb96d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 11:57):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0f8d03d07b8fcdbf21ace65574f7bac6e4f75eca).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 20 2025 at 11:59):

The warning in Mathlib.Data.Seq.Seq.lean is a linter warning arising form #9915. Unfortunately set_option linter.dupNamespace false in breaks the notation, because it makes it too local (i.e. local to the set_option).

For now we can get by with just set_option linter.dupNamespace false (no in). But we need to change something, I think, to avoid generating the name with the duplication, as there's no mechanism to control this at the call site.

@Sebastian Ullrich?

Sebastian Ullrich (Aug 20 2025 at 12:02):

Oh, did it fail to pick up the fixes from lean-pr-testing-9915 because it was merged manually? This is so confusing

Kim Morrison (Aug 20 2025 at 12:03):

Sorry, yes! It doesn't automatically pick up manually merged PRs.

Kim Morrison (Aug 20 2025 at 12:03):

I should have checked ofr that branch, sorry. I'll merge it now.

Sebastian Ullrich (Aug 20 2025 at 12:04):

I can't fault you, it is too easy to miss from either direction, during merge and during bump

Kim Morrison (Aug 20 2025 at 12:05):

I guess the bot that looks for lean-pr-testing-NNNN branches that have been merged could be smarter, and specifically look for rebase-merged PRs.

Sebastian Ullrich (Aug 20 2025 at 12:07):

Does the script currently look at the master history? If it looked at the merged PRs via the API that might work, yeah

Kim Morrison (Aug 20 2025 at 12:08):

Ick:

        # Find all commits to lean4 between the $OLD and $NEW toolchains
        # and extract the github PR numbers
        # (drop anything that doesn't look like a PR number from the final result)
        PRS=$(git log --oneline "$OLD..$NEW" | sed 's/.*(#\([0-9]\+\))$/\1/' | grep -E '^[0-9]+$')

Sebastian Ullrich (Aug 20 2025 at 12:09):

It works, until it doesn't :smile:

Sebastian Ullrich (Aug 20 2025 at 12:10):

Fortunately our needs for manual merging have declined so this might not be too pressing but that also makes it less likely we'll remember the issue the next time around

Kim Morrison (Aug 20 2025 at 12:13):

It's a bit nasty to do this properly. To query for PRs merged in a given time window, I'd first have to actually extract timestampes from the OLD and NEW tags. There's not really an obvious way to go from commits back to their PRs.

Kim Morrison (Aug 20 2025 at 12:14):

I guess I could enumerate all lean-pr-testing-NNNN branches, and for each one check if the PR has been merged. But there'd have to be some amount of filtering there anyway as that would be a lot of queries.

Kim Morrison (Aug 20 2025 at 12:14):

Maybe not worth the trouble this evening...

Bryan Gin-ge Chen (Aug 20 2025 at 12:23):

Kim Morrison said:

There's not really an obvious way to go from commits back to their PRs.

I haven't been following this thread fully so I'm just responding to this sentence, but there is a GitHub API endpoint to list PRs associated to a commit.

It also looks like you can search with gh pr list:

# Find a PR that introduced a given commit
$ gh pr list --search "<SHA>" --state merged

Apologies if I've misinterpreted what you're looking for

Kim Morrison (Aug 20 2025 at 12:37):

Nice, that looks like what we need.

Kim Morrison (Aug 20 2025 at 12:43):

#28692

github mathlib4 bot (Aug 20 2025 at 13:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8efca8d950c32e120c1e38f2671c23b705fca909).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 16:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f913aa5b173dbb3c62f08be0b46432f21fa2493e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 19:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (62983e84d6f67f6d73d9446feeed99571fe98256).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 20 2025 at 23:17):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (d5f898864ce75858d5d5d51057cce15e936c5c66)

github mathlib4 bot (Aug 21 2025 at 02:18):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (1236f501e50c4483de26d1a22b174197097d61b6).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

github mathlib4 bot (Aug 21 2025 at 04:39):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (d5f898864ce75858d5d5d51057cce15e936c5c66)

github mathlib4 bot (Aug 21 2025 at 10:20):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (22de30992624cb78874fb9d3937f1eaf28eef35e)

github mathlib4 bot (Aug 22 2025 at 02:19):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (c2299359f081971ca75e597473ca593b68903a54).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

github mathlib4 bot (Aug 22 2025 at 07:41):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (22de30992624cb78874fb9d3937f1eaf28eef35e)

github mathlib4 bot (Aug 22 2025 at 13:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (46271117fff1c8aa2f8a073f11bf2a4e5109773a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 22 2025 at 16:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b91f1794176ae01a7b9a1f13b351c72f79201295).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 22 2025 at 23:36):

Lean's nightly release process failed last night, so failures will continue here until we get that sorted.

github mathlib4 bot (Aug 23 2025 at 02:16):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (b91f1794176ae01a7b9a1f13b351c72f79201295).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

github mathlib4 bot (Aug 23 2025 at 10:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (53682aa14fd9927beab404717fc0b6896d5e6a0e).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 23 2025 at 12:06):

Unfortunately the nightly release failed again.

Robin Arnez (Aug 23 2025 at 13:13):

Which part? https://github.com/leanprover/lean4-nightly/releases/tag/nightly-2025-08-23 exists

Bryan Gin-ge Chen (Aug 23 2025 at 13:40):

Looks like it's missing darwin_aarch64 and linux_aarch64 in the assets; cf. https://github.com/leanprover/lean4-nightly/releases/tag/nightly-2025-08-21

Robin Arnez (Aug 23 2025 at 13:46):

oh I should look at this? https://github.com/leanprover/lean4/actions/runs/17172609665/job/48726222641

Bryan Gin-ge Chen (Aug 23 2025 at 13:53):

lean4#10076 looks like it might be related.

Robin Arnez (Aug 23 2025 at 14:16):

oh it's a json problem lol

Robin Arnez (Aug 23 2025 at 14:17):

              {
                ...
                "CMAKE_OPTIONS": "-DLEAN_INSTALL_SUFFIX=-darwin_aarch64",
                ...
                "CMAKE_OPTIONS": "-DUSE_LAKE=OFF",
              },

doesn't mean both but it means only the second one and the install suffix is gone

github mathlib4 bot (Aug 24 2025 at 02:26):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (53682aa14fd9927beab404717fc0b6896d5e6a0e).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

github mathlib4 bot (Aug 24 2025 at 08:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (bfd6a054aa5c25e43b11e87cb15bf281f0fb6ba2).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 24 2025 at 09:02):

And we're back to actually failing (i.e. the nightly-2025-08-24 toolchain was produced correctly)

github mathlib4 bot (Aug 24 2025 at 09:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7f4298fff7f1d8d891dfe880f92715152bdeed76).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Aug 24 2025 at 09:14):

nightly#42 should fix everything but I'm running into the problem that build master-branch tools still uses the code from nightly-testing

github mathlib4 bot (Aug 24 2025 at 09:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8e4809bdb14e715d5171981664d32063ff93d294).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 24 2025 at 09:49):

Looks like a few more fixes are needed after nightly#42.

github mathlib4 bot (Aug 24 2025 at 10:05):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9b58a23e03bd71147ece3d810c5f9d3922c12b1f).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Aug 24 2025 at 10:20):

num_intCast and den_intCast should be norm_cast

Robin Arnez (Aug 24 2025 at 10:20):

attribute [norm_cast] num_intCast den_intCast or whatever

github mathlib4 bot (Aug 24 2025 at 11:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e08ccf0188f54be48446870d334af1a648a0a638).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 24 2025 at 11:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (aa4e9536a0b705282174110a3b83a4e86a237180).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 24 2025 at 13:13):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fb7bdf00a2b6e53d2f2edd7df535251a7bcc4a1e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 24 2025 at 15:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (931046fa5c9addaa84cf49ebc8420612ef787945).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Aug 24 2025 at 18:07):

Invalid field notation: Polynomial.eval has a parameter with expected type

Polynomial ?R

but it cannot be used

That problem comes from the constant macro scopes but really what it tells me is:
"I mean like yeah, it looks like this should work but sorry, our implementation is a hack and this case doesn't really work right now"

Robin Arnez (Aug 24 2025 at 18:08):

Could we fix this maybe? I'd expect the parameter to be passed by index or whatever and not by some weird user-specified name

github mathlib4 bot (Aug 24 2025 at 19:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ef785e63a325fd706ea025e76cad1ec28f489fcd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 24 2025 at 21:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cf7fdda47ea9db8bdab1829d1316e21da39f47e1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 24 2025 at 22:53):

Commit b33c9d7aaea comments out two broken proofs about the ShiftLeft Int instance that Mathlib defines. My preferred solution here is simply to deprecate these instances in Mathlib, per #28884, but if we'd like to keep them could someone please put up their hand to:

  • fix the doc-strings to explain what happens for negative shifts
  • revert b33c9d7aaea and fix the proofs on nightly-testing

Robin Arnez (Aug 24 2025 at 23:16):

I fixed it but I agree that those instances are in a bit of a weird position; being in conflict with core instances without there being any proofs correlating them; but one thing that it does well is that <- shiftLeft_sub is nice (compare with Int.shiftLeft_shiftRight_eq which is pretty ugly)

Robin Arnez (Aug 24 2025 at 23:16):

Ideally we would have some proofs though that say that those definitions (with Int vs with Nat) are equivalent

github mathlib4 bot (Aug 24 2025 at 23:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (35fdd5d6f6e459d908215c9ac34bb2432a4c10f2).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 25 2025 at 00:00):

A remaining problem on nightly-testing is:

 [953/7112] Building Mathlib.CategoryTheory.Iso
info: stderr:
libc++abi: terminating due to uncaught exception of type lean::exception: cannot evaluate `[init]` declaration '_private.Mathlib.Tactic.CategoryTheory.Reassoc.0.CategoryTheory.reassocImplRef' in the same module
error: Lean exited with code 134
 [954/7112] Building Mathlib.CategoryTheory.NatTrans
info: stderr:
libc++abi: terminating due to uncaught exception of type lean::exception: cannot evaluate `[init]` declaration '_private.Mathlib.Tactic.CategoryTheory.Reassoc.0.CategoryTheory.reassocImplRef' in the same module

@Sebastian Ullrich, do you have a guess what may have caused this? The error is happening on the files which import Mathlib.Tactic.CategoryTheory.Reassoc, so the error message is slightly off.

Kim Morrison (Aug 25 2025 at 00:06):

(If you don't recognize it I can minimize and bisect against Lean.)

Robin Arnez (Aug 25 2025 at 00:30):

Hmm I think I get where the problem is that we run the initializers in the wrong order so it does registerReassocExpr before initializing reassocImplRef. In InitAttr we seem to assume that ModuleData.constNames is the correct order; but that isn't a guarantee:

          for c in modData.constNames do
            -- make sure to run initializers in declaration order, not extension state order, to respect dependencies
            if let some (decl, initDecl) := modEntries.binSearch (c, default) (Name.quickLt ·.1 ·.1) then
              if initDecl.isAnonymous then
                let initFn  IO.ofExcept <| ctx.env.evalConst (IO Unit) ctx.opts decl
                initFn
              else
                runInit ctx.env ctx.opts decl initDecl

github mathlib4 bot (Aug 25 2025 at 01:16):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (88a2c8412f4c532f223a164de9ba238fcc0d487a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 25 2025 at 01:22):

Robin Arnez said:

Invalid field notation: Polynomial.eval has a parameter with expected type

Polynomial ?R

but it cannot be used

That problem comes from the constant macro scopes but really what it tells me is:
"I mean like yeah, it looks like this should work but sorry, our implementation is a hack and this case doesn't really work right now"

This is fallout from lean#10048. @Sebastian Ullrich, what do you think we should do here?

Polynomial.eval is defined as

def eval : R  R[X]  R :=
  eval₂ (RingHom.id _)

so it is easy to work around this as

def eval (x : R) (p : R[X]) : R :=
  eval₂ (RingHom.id _) x p

(which arguably is an improvement as it enabled named arguments), but it is not a great error message!

(I've made this change for now, so no action necessary, just for consideration.)

Kim Morrison (Aug 25 2025 at 01:29):

Robin Arnez said:

registerReassocExpr

Thanks, @Robin Arnez, for diagnosing this!

What do you think of the workaround in ddc9144a447?

github mathlib4 bot (Aug 25 2025 at 01:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ddc9144a44701b1e8db7ff5b0fa1e7a4e9463759).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 01:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ddc9144a44701b1e8db7ff5b0fa1e7a4e9463759).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 02:22):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (ddc9144a44701b1e8db7ff5b0fa1e7a4e9463759).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

github mathlib4 bot (Aug 25 2025 at 04:15):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c288098e415e0131adc2313b785371044869f962).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 05:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6b527e3d87f79b59e9f9a658ca38cf64cae9f83d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 25 2025 at 06:41):

Oooh, this is not fun: the remaining failure on nightly-testing is the MathlibTest.RewriteSearch.Basic segfaults.

Kim Morrison (Aug 25 2025 at 06:43):

% lake env lldb lean MathlibTest/RewriteSearch/Basic.lean
(lldb) target create "lean"
Current executable set to '/Users/kim/.elan/toolchains/leanprover--lean4-nightly---nightly-2025-08-24/bin/lean' (arm64).
(lldb) settings set -- target.run-args  "MathlibTest/RewriteSearch/Basic.lean"
(lldb) run
Process 4391 launched: '/Users/kim/.elan/toolchains/leanprover--lean4-nightly---nightly-2025-08-24/bin/lean' (arm64)
Process 4391 stopped
* thread #3, stop reason = EXC_BAD_ACCESS (code=1, address=0x10)
    frame #0: 0x000000010eefc7b8 libleanshared.dylib`mi_malloc_small + 48
libleanshared.dylib`mi_malloc_small:
->  0x10eefc7b8 <+48>: ldr    x8, [x9, #0x10]
    0x10eefc7bc <+52>: cbz    x8, 0x10eefc7e0           ; <+88>
    0x10eefc7c0 <+56>: ldr    x10, [x8]
    0x10eefc7c4 <+60>: str    x10, [x9, #0x10]
Target 0: (lean) stopped.
(lldb) bt
* thread #3, stop reason = EXC_BAD_ACCESS (code=1, address=0x10)
  * frame #0: 0x000000010eefc7b8 libleanshared.dylib`mi_malloc_small + 48
    frame #1: 0x000000010eee6a08 libleanshared.dylib`lean::fix_args(lean_object*, unsigned int, lean_object* const*) + 76
    frame #2: 0x000000010eed6248 libleanshared.dylib`lean_apply_1 + 184
    frame #3: 0x000000010ec7b568 libleanshared.dylib`lean::ir::interpreter::eval_expr(lean::object_ref const&, lean::ir::type) + 2524
    frame #4: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #5: 0x000000010ec7c070 libleanshared.dylib`lean::ir::interpreter::call(lean::name const&, lean::array_ref<lean::object_ref> const&) + 1212
    frame #6: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #7: 0x000000010ec7c070 libleanshared.dylib`lean::ir::interpreter::call(lean::name const&, lean::array_ref<lean::object_ref> const&) + 1212
    frame #8: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #9: 0x000000010ec7c070 libleanshared.dylib`lean::ir::interpreter::call(lean::name const&, lean::array_ref<lean::object_ref> const&) + 1212
    frame #10: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #11: 0x000000010ec7c070 libleanshared.dylib`lean::ir::interpreter::call(lean::name const&, lean::array_ref<lean::object_ref> const&) + 1212
    frame #12: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #13: 0x000000010ec7c070 libleanshared.dylib`lean::ir::interpreter::call(lean::name const&, lean::array_ref<lean::object_ref> const&) + 1212
    frame #14: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #15: 0x000000010ec7c070 libleanshared.dylib`lean::ir::interpreter::call(lean::name const&, lean::array_ref<lean::object_ref> const&) + 1212
    frame #16: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #17: 0x000000010ec7dfac libleanshared.dylib`lean::ir::interpreter::stub_m(lean_object**) + 556
    frame #18: 0x000000010ec7dba8 libleanshared.dylib`lean::ir::interpreter::stub_m_aux(lean_object**) + 92
    frame #19: 0x000000010ec7daac libleanshared.dylib`lean::ir::interpreter::stub_15_aux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*) + 76
    frame #20: 0x000000010eedfdf0 libleanshared.dylib`lean_apply_7 + 3036
    frame #21: 0x000000010ec7b568 libleanshared.dylib`lean::ir::interpreter::eval_expr(lean::object_ref const&, lean::ir::type) + 2524

<snip>

    frame #109: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #110: 0x000000010ec7c070 libleanshared.dylib`lean::ir::interpreter::call(lean::name const&, lean::array_ref<lean::object_ref> const&) + 1212
    frame #111: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #112: 0x000000010ec7dfac libleanshared.dylib`lean::ir::interpreter::stub_m(lean_object**) + 556
    frame #113: 0x000000010ec7dba8 libleanshared.dylib`lean::ir::interpreter::stub_m_aux(lean_object**) + 92
    frame #114: 0x000000010eee15b8 libleanshared.dylib`lean_apply_9 + 996
    frame #115: 0x000000010eedcf5c libleanshared.dylib`lean_apply_5 + 1096
    frame #116: 0x000000010af1672c libleanshared.dylib`l_Lean_MVarId_withContext___at___Lean_Elab_Tactic_withMainContext_spec__0___redArg + 152
    frame #117: 0x000000010af16ad4 libleanshared.dylib`l_Lean_Elab_Tactic_withMainContext___redArg + 644
    frame #118: 0x000000010eed60a4 libleanshared.dylib`lean::curry(void*, unsigned int, lean_object**) + 404
    frame #119: 0x000000010ec7bdc8 libleanshared.dylib`lean::ir::interpreter::call(lean::name const&, lean::array_ref<lean::object_ref> const&) + 532
    frame #120: 0x000000010ec7a148 libleanshared.dylib`lean::ir::interpreter::eval_body(lean::object_ref const&) + 3192
    frame #121: 0x000000010ec7dfac libleanshared.dylib`lean::ir::interpreter::stub_m(lean_object**) + 556
    frame #122: 0x000000010ec744b0 libleanshared.dylib`lean_object* lean::ir::interpreter::with_interpreter<lean_object*>(lean::elab_environment const&, lean::options const&, lean::name const&, std::__1::function<lean_object* (lean::ir::interpreter&)> const&) + 320
    frame #123: 0x000000010ec7dba8 libleanshared.dylib`lean::ir::interpreter::stub_m_aux(lean_object**) + 92
    frame #124: 0x000000010ec7d9c8 libleanshared.dylib`lean::ir::interpreter::stub_13_aux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*) + 68
    frame #125: 0x000000010eee170c libleanshared.dylib`lean_apply_9 + 1336
    frame #126: 0x000000010aee59a0 libleanshared.dylib`l_Lean_Elab_withInfoTreeContext___at_____private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTactic_eval_spec__5___redArg + 540
    frame #127: 0x000000010eee16a4 libleanshared.dylib`lean_apply_9 + 1232
    frame #128: 0x000000010aee703c libleanshared.dylib`l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTactic_eval + 820
    frame #129: 0x000000010aef855c libleanshared.dylib`l_Lean_Elab_Tactic_evalTactic___lam__1 + 1396
    frame #130: 0x000000010eee163c libleanshared.dylib`lean_apply_9 + 1128
    frame #131: 0x000000010aef92bc libleanshared.dylib`l_Lean_Elab_Tactic_evalTactic___lam__3 + 1056
    frame #132: 0x000000010eeda050 libleanshared.dylib`lean_apply_3 + 1128
    frame #133: 0x000000010eed64b0 libleanshared.dylib`lean_apply_1 + 800
    frame #134: 0x000000010ead7b58 libleanshared.dylib`l_Lean_profileitIOUnsafe___redArg___lam__0 + 20
    frame #135: 0x000000010eed6378 libleanshared.dylib`lean_apply_1 + 488
    frame #136: 0x0000000108ac0864 libleanshared.dylib`l_unsafeBaseIO___redArg + 20
    frame #137: 0x000000010eed6378 libleanshared.dylib`lean_apply_1 + 488
    frame #138: 0x000000010ec6f428 libleanshared.dylib`lean_profileit + 128
    frame #139: 0x000000010ead7e44 libleanshared.dylib`l_Lean_profileitIOUnsafe___redArg + 168
    frame #140: 0x000000010aef01b0 libleanshared.dylib`l_Lean_Elab_Tactic_evalTactic + 756

Kim Morrison (Aug 25 2025 at 06:45):

@Sebastian Ullrich and/or @Cameron Zwarich, does this ring any bells?

github mathlib4 bot (Aug 25 2025 at 07:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ba9c622e37b391d509a058d8c4878c697fa0da83).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Aug 25 2025 at 07:46):

I expect this to be due to some miscompilation, maybe because of lean4#10080? (specializing bestFirstSearchCore?) I didn't look into it that much though

Robin Arnez (Aug 25 2025 at 08:23):

Hmm actually, adding @[nospecialize, noinline] everywhere doesn't seem to help at all

Sebastian Ullrich (Aug 25 2025 at 08:26):

Hmm, thanks for trying. It might be best to try with a debug builds of Lean next but I don't want to jump ahead of Cameron Zwarich

Sebastian Ullrich (Aug 25 2025 at 08:34):

Kim Morrison said:

which arguably is an improvement as it enabled named arguments

It's not great that implementation details would leak like this but given what you said above, perhaps "consider naming them explicitly" would suffice as a hint? /cc @Kyle Miller

Sebastian Ullrich (Aug 25 2025 at 08:35):

I should mention that I made the constant macro scope change as it was an easy win of -1.5% olean size on core (how much on Mathlib?). It it's not that easy after all... we can also revert

github mathlib4 bot (Aug 25 2025 at 08:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (039362c3565ab3e652725c6fde0eea5acf72c275).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Aug 25 2025 at 09:39):

I tried running it compiled, in hopes of getting a better backtrace but then it didn't segfault anymore!

import Mathlib.Tactic.RewriteSearch

open Qq in
def rwSearchTest : Lean.MetaM Unit := do
  IO.println "Running test..."
  let u : Lean.Level := .param `u
  let goalType := q({α : Type u}  (xs ys : List α)  (xs ++ ys).length = ys.length + xs.length)
  let goal := ( Lean.Meta.mkFreshExprMVar goalType).mvarId!
  let (_vars, goal)  goal.introNP 3
  IO.println "Running rw_search tactic..."
  let stx  `(tactic| rw_search)
  let tactic := Mathlib.Tactic.RewriteSearch._aux_Mathlib_Tactic_RewriteSearch___elabRules_Mathlib_Tactic_RewriteSearch_tacticRw_search__1
  let ((_, _st1), _st2)  (((tactic stx).run { elaborator := decl_name% }).run { goals := [goal] }).run {} { levelNames := [`u] }
  let newGoals := _st1.goals
  if newGoals.isEmpty then
    IO.println "success!"
  IO.println s!"{newGoals.length} goals remaining"
  IO.println ( ( Lean.addMessageContext m!"{newGoals}").format)

def main : IO Unit := do
  Lean.initSearchPath ( Lean.findSysroot)
  let env  Lean.importModules #[{ module := `Init }, { module := `Mathlib.Tactic.RewriteSearch }]
    {} (loadExts := true) (trustLevel := 1024)
  discard <| rwSearchTest.toIO {
    fileName := "<thing>"
    fileMap := .ofString ""
  } { env }
  unsafe env.freeRegions

prints

Running test...
Running rw_search tactic...
1 goals remaining
[α : Type u
 xs ys : List α
  ys.length + xs.length = ys.length + xs.length]

Robin Arnez (Aug 25 2025 at 09:40):

slightly weird that it didn't close the goal though

Sebastian Ullrich (Aug 25 2025 at 09:41):

But it does segfault if you --run the same test file?

Robin Arnez (Aug 25 2025 at 09:42):

Yeah

Sebastian Ullrich (Aug 25 2025 at 09:42):

Huh. Might either be a bad draw in the UB lottery or an interpreter/codegen mismatch

Robin Arnez (Aug 25 2025 at 09:55):

It might still be a compiler issue, e.g. a reference counting issue; I believe one difference between compiled and interpreted is that compiled uses persistent objects more often; maybe that avoided a reference counting problem somewhere?

github mathlib4 bot (Aug 25 2025 at 10:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0a77f02f7536cbae1d8f6c2813346bca553fe37b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 10:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c430e6977dad473443f4d6c8f74f2be752c1340e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 12:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (65f3f36b8efe85830339dff773aa4f4f7b255eb0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 15:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fe8bea84faf94f9e03a1f0fcf35942312a4e45f3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 19:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (19b193ae881a85aa81046dde04a05a22ae08809f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 19:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (53e88d71e373f41aa439ea0ba3557b717b88a08e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 20:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e1279ca36bc5d9294d14c56e9eea72056615d87c).
You can git fetch; git checkout nightly-testing and push a fix.

Cameron Zwarich (Aug 25 2025 at 21:23):

Kim Morrison said:

Sebastian Ullrich and/or Cameron Zwarich, does this ring any bells?

This stack trace looks like a use-after-free stomping on some allocator state. There is no compiler change that looks obviously related (although there were a few big optimizations that changed a lot of things and thus could've exposed a latent bug), so I'll have to revert them one by one and see what's to blame.

There are a few differences in object lifetimes between the interpreter and the C backend (e.g. how closed term decl initialization works, the interpreter using the _boxed versions of decls more often, etc.) but I also don't quite see how they would interact with any of the changes since the last green build.

github mathlib4 bot (Aug 25 2025 at 21:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (14efc83ef191c7ae4f8ba65d7c099532262e2552).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 22:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b9ad933d5ebb527ee50f1767e395034e1687e6bb).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Aug 25 2025 at 22:44):

I temporarily disabled the rw_search tests now (in b118ce2f6d4) so we should hopefully get a build now

github mathlib4 bot (Aug 25 2025 at 23:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b118ce2f6d4af5b60401c2d7de53f2ec9c2a9092).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 25 2025 at 23:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9ca6b7c24f508c9e81b71ed905e114ac0a86dc1b).
You can git fetch; git checkout nightly-testing and push a fix.

Cameron Zwarich (Aug 26 2025 at 01:29):

Cameron Zwarich said:

Kim Morrison said:

Sebastian Ullrich and/or Cameron Zwarich, does this ring any bells?

This stack trace looks like a use-after-free stomping on some allocator state. There is no compiler change that looks obviously related (although there were a few big optimizations that changed a lot of things and thus could've exposed a latent bug), so I'll have to revert them one by one and see what's to blame.

There are a few differences in object lifetimes between the interpreter and the C backend (e.g. how closed term decl initialization works, the interpreter using the _boxed versions of decls more often, etc.) but I also don't quite see how they would interact with any of the changes since the last green build.

This is indeed #10080 as @Robin Arnez expected. Assuming I did the compiler binary juggling correctly, rebuilding every other file with #10080 reverted and only Mathlib/Tactic/RewriteSearch.lean with #10080 in place suffices to trigger the bug.

It looks like RewriteSearch.lean relies heavily on Batteries.Data.MLList, which has a lot of unsafe code. Based on my past experiences with unsafe code being used by Mathlib, it wouldn't surprise me if this unsafe code is subtly incorrect, but the increased specialization is causing the compiler to now perform optimizations that expose this incorrectness.

github mathlib4 bot (Aug 26 2025 at 02:00):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f214e78436f4a4b0f4dfc54e072c37334ce4e04e)

github mathlib4 bot (Aug 26 2025 at 02:21):

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (f214e78436f4a4b0f4dfc54e072c37334ce4e04e).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

Kim Morrison (Aug 26 2025 at 02:50):

As the author of that unsafe code, I would not be surprised if it is incorrect. :-)

Let me see how everyone feels about simply deprecating RewriteSearch. I still like the idea, but I have not had a chance to work on it for a long time, and no one else has taken it up.

Kim Morrison (Aug 26 2025 at 02:56):

github mathlib4 bot said:

:cross_mark: The docgen run for Mathlib's nightly-testing branch has failed (f214e78436f4a4b0f4dfc54e072c37334ce4e04e).
This likely indicates an issue with the nightly Lean build, or a required update in doc-gen4.

@Anne Baanen, I'm leaving this for you to look at for now? Perhaps we could move this to a different thread as it is a bit distracting here.

github mathlib4 bot (Aug 26 2025 at 04:15):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f214e78436f4a4b0f4dfc54e072c37334ce4e04e)

Cameron Zwarich (Aug 26 2025 at 06:13):

Cameron Zwarich said:

This is indeed #10080 as Robin Arnez expected. Assuming I did the compiler binary juggling correctly, rebuilding every other file with #10080 reverted and only Mathlib/Tactic/RewriteSearch.lean with #10080 in place suffices to trigger the bug.

If I add

diff --git a/Mathlib/Data/MLList/BestFirst.lean b/Mathlib/Data/MLList/BestFirst.lean
index 254dcdfde25..c6d1414af89 100644
--- a/Mathlib/Data/MLList/BestFirst.lean
+++ b/Mathlib/Data/MLList/BestFirst.lean
@@ -250,6 +250,7 @@ where
 /--
 Wrapper for `impl` implementing the `maxDepth` option.
 -/
+@[nospecialize]
 def implMaxDepth (maxSize : Option Nat) (maxDepth : Option Nat) (f : α → MLList m α) (a : α) :
     MLList m α :=
   match maxDepth with

on nightly-testing-2025-08-21 (the last green build before this string of failures), then I get similar memory corruption crashes. If this is a compiler issue rather than a bug in unsafe code, then I don't think it's a recent one.

Cameron Zwarich (Aug 26 2025 at 06:16):

The same failure occurs with master and stable.

github mathlib4 bot (Aug 26 2025 at 08:32):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f214e78436f4a4b0f4dfc54e072c37334ce4e04e)

Kim Morrison (Aug 26 2025 at 13:16):

I'm discussing with maintainers just ripping out this code (all MLList and rw_search material in Mathlib). As much as I love it (it was my first project in Lean back in ????), no one is using it.

github mathlib4 bot (Aug 26 2025 at 13:44):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f214e78436f4a4b0f4dfc54e072c37334ce4e04e)

github mathlib4 bot (Aug 26 2025 at 18:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9e8e11b3f439fb2f9b27ee07993bb62c9bddbe7c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 26 2025 at 21:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (eadb897205c7c7c75319e5bb00d1aac5a286e678).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 27 2025 at 00:47):

In commit 348f72ec963 I have commented out the "Try this" suggestion that replaces @[to_additive] string style comments with doc-string style comments. lean#9966 redesigned the interface here, and removed a private function. Unfortunately, @Thomas Murrills when installing this suggestion had used open private. (I think it's a good idea if any PR to Mathlib using open private involves during review an explicit discussion of that use of open private.)

Would anyone like to adopt this problem?

Note that a warning is still logged, my commenting out only removes the Try this. I would recommend that we choose not to work on this, as it is clearly not worth the effort for the payoff. :-)

github mathlib4 bot (Aug 27 2025 at 00:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d55a0757fac143156ac878cc289a7ff989126b2e).
You can git fetch; git checkout nightly-testing and push a fix.

Thomas Murrills (Aug 27 2025 at 01:00):

I can fix this; the corresponding declaration I would need in place of addSuggestionCore after lean4#9966 is no longer private, if I recall correctly. :)

Thomas Murrills (Aug 27 2025 at 01:03):

(I will do so in about half an hour; the fix should be straightforward.)

Thomas Murrills (Aug 27 2025 at 01:46):

mathlib4-nightly-testing#45

Thomas Murrills (Aug 27 2025 at 01:52):

There's another lean4#9966 adaptation necessary: we lost suggestion styling :( What should we do for successful tactics in the hint tactic? Emoji? Separate lists (which is easier to have in a single message now)?

Kim Morrison (Aug 27 2025 at 02:14):

Emoji sounds good to me.

Thomas Murrills (Aug 27 2025 at 02:15):

I thought so too! :) mathlib4-nightly-testing#46

Thomas Murrills (Aug 27 2025 at 02:15):

However, I can't test that yet, and the tests will need to be updated due to new indentation; imports seem to be stuck on Lean.Grind.PartialOrder missing?

Kim Morrison (Aug 27 2025 at 02:16):

Yes, I'm about to work on that.

Kim Morrison (Aug 27 2025 at 02:16):

Are we treating the styling as just gone for good? If so, no need for the adaptation note.

Thomas Murrills (Aug 27 2025 at 02:19):

Honestly, I'm not sure. The reasoning in the PR is that the hint infrastructure uses diff colors so styling is not needed, but, of course, try this suggestions typically do not use a diff. I'm not sure there was ever any discussion on it.

Thomas Murrills (Aug 27 2025 at 02:24):

I've asked in #lean4 > Try This suggestion styling .

Kim Morrison (Aug 27 2025 at 02:29):

Okay, nightly-testing should be available for testing this now, most of the other issues are fixed.

Kim Morrison (Aug 27 2025 at 02:32):

In f23f2657a53 I've commented out Mathlib.Data.UInt, as these are broken by lean#10095. @Eric Wieser, might you be able to look at this file again?

Thomas Murrills (Aug 27 2025 at 02:46):

(note: there's a weird whitespace issue. I'm currently chasing it down.)

github mathlib4 bot (Aug 27 2025 at 03:16):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f23f2657a53c55dc28026f75fcb0f7d4b4404241).
You can git fetch; git checkout nightly-testing and push a fix.

Thomas Murrills (Aug 27 2025 at 03:34):

Ok, hint should be fixed in mathlib4-nightly-testing#46!

However, because the suggestions are just embedded in MessageData now, I had to rework how it extracts Try This messages from the message logs. Without the change, it e.g. resulted in the entire text of "The ring tactic failed to close the goal. Use ring_nf to obtain a normal form. Note that ring works primarily in commutative rings. ..." etc. becoming part of the clickable link for ring_nf!

Also, apparently unrelated to my changes, the "remaining subgoals" info is now inline. (I'm not sure why that didn't appear before, to be honest...)

github mathlib4 bot (Aug 27 2025 at 04:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (faa8f51e9f0a626466b8e2be4af3aa50fadf7a1e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 27 2025 at 07:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (dd9d2df1a66f8a0294085cff0e59bf4757d2a95b).
You can git fetch; git checkout nightly-testing and push a fix.

Eric Wieser (Aug 27 2025 at 09:28):

Kim Morrison said:

In f23f2657a53 I've commented out Mathlib.Data.UInt, as these are broken by lean#10095. Eric Wieser, might you be able to look at this file again?

Could you try to upstream these API lemmas? This file is fragile in mathlib because the API is missing in core.

github mathlib4 bot (Aug 27 2025 at 10:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (268156f1afd235b90b268f12830593dec03728a8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 27 2025 at 14:17):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (46bc1d577efe31c33665a8f514f516b7f226485d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 27 2025 at 16:03):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (aaa84839f37fe188d883c3484c976f4b2d8c18e3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 27 2025 at 19:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1a87afd394e950ecfa6689376e1b7f023c755458).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 27 2025 at 22:11):

@Mario Carneiro, TMToPartrec was failing on nightly-testing. I have patched it with a

@[simp] theorem default_Γ' : (default : Γ') = .consₗ := rfl

in 7403ebf52c8. If you'd like to investigate and see if there is a better fix than relying on the default value picked by deriving Inhabited, please do!

Mario Carneiro (Aug 27 2025 at 22:14):

the definitions in that file generally care about what the Inhabited instance value is

Mario Carneiro (Aug 27 2025 at 22:16):

IIRC there used to be arbitrary and default which differed in opacity

Mario Carneiro (Aug 27 2025 at 22:17):

in the absence of additional info on this situation I think I will say that your fix is good and working as intended

github mathlib4 bot (Aug 27 2025 at 23:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (19143a453b8ced0b8bfdae7456279c6d9da38ee0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 28 2025 at 00:06):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (1d38490977bf42f87ba86618f8513cdb33e3b66e)

Eric Wieser (Aug 28 2025 at 00:17):

Kim Morrison said:

In f23f2657a53 I've commented out Mathlib.Data.UInt, as these are broken by lean#10095. Eric Wieser, might you be able to look at this file again?

The fix was just to delete the failing change tactic, this probably didn't need my input!

github mathlib4 bot (Aug 28 2025 at 00:36):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (1d38490977bf42f87ba86618f8513cdb33e3b66e)

Kim Morrison (Aug 28 2025 at 01:18):

Eric Wieser said:

Kim Morrison said:

In f23f2657a53 I've commented out Mathlib.Data.UInt, as these are broken by lean#10095. Eric Wieser, might you be able to look at this file again?

The fix was just to delete the failing change tactic, this probably didn't need my input!

I wish it didn't need my input either. :-)

github mathlib4 bot (Aug 28 2025 at 01:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7ac4458414b1b1f9a3727a7ff811d78c57a5b2db).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 28 2025 at 03:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f46954a961506e2db50438c46be04bbf06d40a23).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 28 2025 at 05:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9e3aa70b7224ccb0bf53b353debfa000f9b473d4).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Aug 28 2025 at 05:26):

@Heather Macbeth, this failure on nightly-testing come from the new field_simp implementation, which seem to be depending on the HMul Nat Int Int instance that Lean briefly provided, until it was removed again in lean#10095.

Might you be able to take a look, as it it hopefully fresh in mind? :-)

github mathlib4 bot (Aug 28 2025 at 10:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9919010ab300194e909b03cbe4f739c3ab374f53).
You can git fetch; git checkout nightly-testing and push a fix.

Heather Macbeth (Aug 28 2025 at 11:14):

Kim Morrison said:

Heather Macbeth, this failure on nightly-testing come from the new field_simp implementation, which seem to be depending on the HMul Nat Int Int instance that Lean briefly provided, until it was removed again in lean#10095.

Might you be able to take a look, as it it hopefully fresh in mind? :-)

I can look tonight (UK), if that's not too late?

Kim Morrison (Aug 28 2025 at 13:01):

No problem!

github mathlib4 bot (Aug 28 2025 at 13:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1228e72d8b68683e2db2883126866edb51a61030).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 28 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0d49ab1eff9d96b07e33502baca1ee0f1eea7357).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 28 2025 at 18:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5974f8a2bbe61cda614fdc0fc7aa8bdf425f57c4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 28 2025 at 21:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (973a7c56604d0c22589c540766c903e430672cb4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 00:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (abaa12bd2107ae2bb14783df3f180df597863422).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 01:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d68f1d1f0a92f871b00c20ca469dcd683f7d4998).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 04:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5ed0251e34d48b8456d9804cf32cbb1b18ab62a6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 07:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7022ab8bcfa901eeb8e3a43aae284ecc7fac529c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 07:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e570c810a89d1dbb9161cabfd850a91da6c13217).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 08:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0c04996ed5cb31e282827c2a290c2291266aad34).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 09:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (065ecc7b79c2337cd366470f483a531cef675e2f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 10:45):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (afe72e68283d0c004c4edb52dcda9b07a814e967)

github mathlib4 bot (Aug 29 2025 at 22:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a3d4ccd7739565ab64ae40535fb0f2adca08f787).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 29 2025 at 22:39):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (afe72e68283d0c004c4edb52dcda9b07a814e967)

github mathlib4 bot (Aug 30 2025 at 09:47):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (2e6efbfc49121caf1cd26ab0369e3bd669224793)

github mathlib4 bot (Aug 30 2025 at 15:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f13cef247bc878836a4e88669e5f44b0631914dc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 30 2025 at 18:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b6ea1437c3b877db0a2109ad669ba409dd75e5f4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 30 2025 at 21:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4fe4bc874db0fb7bb50f042285e0afb3fa4988b9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 31 2025 at 00:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (59688f30ccd8be604a6058bb0734c2aca99dc464).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 31 2025 at 03:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (23d4593d4575c82c287252f9002456804e5b0f93).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 31 2025 at 06:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9470bafc734f508c715e723a1d3f522a16a7e342).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 31 2025 at 09:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d57156e908c5d36101e4487f90410089d8a17db2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 31 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (107af67327b1d88ee6529529ca0384fa2cda22c8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 31 2025 at 11:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d751ecbf2c22521bd0950c6c6ceaed08fb455420).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Aug 31 2025 at 13:22):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (2fc09c9e3531633ca62167e46418d9b374878be8)

github mathlib4 bot (Sep 01 2025 at 23:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c3b90ae8ac2cc99fd8f4d2e62cf14c53fd526850).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 02:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d055e8423fcfe976c3cac4c024cb82a3f9073d48).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 03:16):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (2fc09c9e3531633ca62167e46418d9b374878be8)

github mathlib4 bot (Sep 02 2025 at 04:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f0421f4cf5127fba0f640c9f83aef0905cce9cab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 07:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (16575b154651ef009f3ef5fe28b5c0f01a5f2c92).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 10:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a0c93326d2ab0bfb05c3b937bd58cb1aff6c8b9b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 11:03):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b437a03eab185fc2323153812b21a76ecfce01c7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 13:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a1a3872cdb8e829dd636a572a7147e32122fdf18).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 14:20):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c0a856404dee9deb13c105e0132addd8447e8897).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 15:05):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b0b16e210ec91ba36e62da3ec71103d95e86697d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 15:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ed40e1fa33cb6928ad145697a401f0201cc50026).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 16:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (29f22042b3abe588dfbb76893a627bccad0c64c9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 18:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9f00ccffeff080df8783ceebb65618dacb42426d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 18:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f3c2c804d16088e6f44b9b71bc9a4cb8fe3108df).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (453d7bc24cd2044fe61d763baa9c0a510557c0e2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 23:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6661b3e08f7f00fe25835ad06d0362c36b066417).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 02 2025 at 23:23):

@Frédéric Dupuis, we've enabled some experimental linters on nightly-testing, and your lemma docs#AkraBazziRecurrence.smoothingFn_mul_asympBound_isBigO_T is timing out. It's not a big deal: we can disable the linter on that particular theorem.

But the proof of that theorem is pretty epic... Would you be able to take a look at refactoring it into some smaller pieces?

(Just a PR to master will suffice for our purposes.)

github mathlib4 bot (Sep 02 2025 at 23:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ac788fd6288294f5f30308228e7f25a392059113).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 02 2025 at 23:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (df9b40f3019f8dab7f37bbd56fd488f6afce6ddf).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 03 2025 at 00:55):

@Anne Baanen, this is failing now because the linters are turned on, but we still run with --iofail, so the new linter warnings fail the build.

Kim Morrison (Sep 03 2025 at 00:57):

I have commented out linter.nightlyRegressionSet in the lakefile, so we can get to green.

Frédéric Dupuis (Sep 03 2025 at 01:18):

Kim Morrison said:

Frédéric Dupuis, we've enabled some experimental linters on nightly-testing, and your lemma docs#AkraBazziRecurrence.smoothingFn_mul_asympBound_isBigO_T is timing out. It's not a big deal: we can disable the linter on that particular theorem.

But the proof of that theorem is pretty epic... Would you be able to take a look at refactoring it into some smaller pieces?

(Just a PR to master will suffice for our purposes.)

Sure, I can have a look.

BTW, is there a good way to just count the number of heartbeats in a proof? I can't seem to find this particular option anywhere, and sometimes it's hard to figure out if I'm making things worse or better performance-wise.

github mathlib4 bot (Sep 03 2025 at 02:30):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f21162f1c74a5fca6c307b107ed4509d01211db4)

Kim Morrison (Sep 03 2025 at 05:08):

#count_heartbeats in

github mathlib4 bot (Sep 03 2025 at 07:37):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f21162f1c74a5fca6c307b107ed4509d01211db4)

Anne Baanen (Sep 03 2025 at 09:13):

Kim Morrison said:

I have commented out linter.nightlyRegressionSet in the lakefile, so we can get to green.

Sorry about that. I'll move the debugging to another branch so it's not in your way!

github mathlib4 bot (Sep 03 2025 at 10:16):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (19646373efebfe279efe5f2e081a451c8077dbb7)

Frédéric Dupuis (Sep 03 2025 at 13:29):

Kim Morrison said:

#count_heartbeats in

Hmm... when I try to use it, I get an absurdly low number (108 for the proof in question), and then in the proof I get warnings on every tactic used saying that they're not being executed.

Ruben Van de Velde (Sep 03 2025 at 13:34):

Frédéric Dupuis said:

Kim Morrison said:

#count_heartbeats in

Hmm... when I try to use it, I get an absurdly low number (108 for the proof in question), and then in the proof I get warnings on every tactic used saying that they're not being executed.

See #mathlib4 > Is count_heartbeats broken

Frédéric Dupuis (Sep 03 2025 at 13:38):

Ah, I see...

github mathlib4 bot (Sep 03 2025 at 13:57):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (19646373efebfe279efe5f2e081a451c8077dbb7)

github mathlib4 bot (Sep 04 2025 at 10:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (059d67009720902a541bbf8caaa0b2b1d963b555).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 04 2025 at 11:17):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (d06300bafa0768331d81d5d0578b7f80cd22d947)

github mathlib4 bot (Sep 05 2025 at 10:53):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (3e9027c0d42944b12f9e1f5889e6635fb8afd822)

github mathlib4 bot (Sep 06 2025 at 10:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (45a653e4e768209e80192b08562d72f4efb7c562).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 06 2025 at 13:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e84eb70f32a07878fc13d12b3290792776a68e83).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 06 2025 at 15:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (af5ceb540466569085f33f79f0f6e3ae56e7a589).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 06 2025 at 21:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d709f77c9b318e243a4d60bbf31e589ced4aceee).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 07 2025 at 01:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a3c6a5a14d8b2491fe4f2af8af226a3f1ae2f19a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 07 2025 at 04:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cd080dec63f0e5a0d53d46af8443890c39b35ca7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 07 2025 at 07:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8a7e8b2e556a006da5864bd028c680be83ad9a72).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Sep 07 2025 at 08:39):

The test that's failing seems to uncover a performance regression in grind:

import Mathlib

variable {K : Type*} [Field K] {x : K}

-- about half a second / more than twice as long as before
set_option maxHeartbeats 13692 in -- uses about 4000 as of 2025-08-06
example : x ^ 3 * x ^ 42 = x ^ 45 := by grind

The problem seems to be that the HSMul instances take much longer to find:

import Mathlib

set_option maxHeartbeats 2900 in
#synth HSMul  (Lean.Grind.IntModule.OfNatModule.Q K) (Lean.Grind.IntModule.OfNatModule.Q K)

set_option maxHeartbeats 2700 in
#synth HSMul  (Lean.Grind.IntModule.OfNatModule.Q K) (Lean.Grind.IntModule.OfNatModule.Q K)

-- previously

set_option maxHeartbeats 160 in
#synth HMul  (Lean.Grind.IntModule.OfNatModule.Q K) (Lean.Grind.IntModule.OfNatModule.Q K)

set_option maxHeartbeats 990 in
#synth HMul  (Lean.Grind.IntModule.OfNatModule.Q K) (Lean.Grind.IntModule.OfNatModule.Q K)

github mathlib4 bot (Sep 07 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b9279110bd82fcfae085b22f44f2e7a0174a7e9b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 07 2025 at 10:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c6a0dadeed5e42ce66c578a6a64f645431584417).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 07 2025 at 13:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c243dd2051513066d79315d01780eb5b10bea7b4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 07 2025 at 22:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fe5f6cf66400f67ea8d1679fba244b4a42500647).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 08 2025 at 00:52):

@Joachim Breitner, we are seeing linter failures on nightly-testing which are presumably due to your recent changes to deriving DecidableEq, e.g.

% lake exe runLinter Mathlib.CategoryTheory.Limits.Shapes.WidePullbacks
Running linter on specified module: Mathlib.CategoryTheory.Limits.Shapes.WidePullbacks
-- Found 3 errors in 13126 declarations (plus 9014 automatically generated ones) in Mathlib.CategoryTheory.Limits.Shapes.WidePullbacks with 15 linters

/- The `unusedArguments` linter reports:
UNUSED ARGUMENTS. -/
-- Mathlib.CategoryTheory.Limits.Shapes.WidePullbacks
/Users/kim/projects/lean/mathlib4/Mathlib/CategoryTheory/Limits/Shapes/WidePullbacks.lean:57:12: error: @CategoryTheory.Limits.WidePullbackShape.instDecidableEqHom.decEq argument 4 inst : DecidableEq
  J
/Users/kim/projects/lean/mathlib4/Mathlib/CategoryTheory/Limits/Shapes/WidePullbacks.lean:159:12: error: @CategoryTheory.Limits.WidePushoutShape.instDecidableEqHom.decEq argument 4 inst : DecidableEq
  J

-- Mathlib.Tactic.ToAdditive.Frontend
/Users/kim/projects/lean/mathlib4/Mathlib/Tactic/ToAdditive/Frontend.lean:495:12: error: ToAdditive.instReprConfig.repr argument 2 prec : 

I see in this example we previously had

-- This is relying on an automatically generated instance name, generated in a `deriving` handler.
-- See https://github.com/leanprover/lean4/issues/2343
attribute [nolint unusedArguments] instDecidableEqHom

and adding .decEq here resolves the linter warning. But do we want to fix this more fundamentally?

Kim Morrison (Sep 08 2025 at 00:53):

The linter error in ToAdditive.Frontend did not previously require a @[nolint] attribute, but now does.

Kim Morrison (Sep 08 2025 at 00:56):

I created https://github.com/leanprover/lean4/issues/10295 to track this, and will add a link to this issue at each place I need to write or update a @[nolints] attribute.

Kim Morrison (Sep 08 2025 at 01:00):

These are all in 9fd69a855164, in case we're able to revert later.

github mathlib4 bot (Sep 08 2025 at 02:07):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5c98deb5fa1eb4f539c1e70d0bc875815dadb820).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 08 2025 at 07:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f5e6060d2ae950e483dc06221265b196ab944a5d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 08 2025 at 11:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d9df815917a3e6e32b9d4aeebbc7ad1bf6587275).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 08 2025 at 12:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (300aa9a66e8de177acb32a2ec0df170ba59cccfb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 08 2025 at 16:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3dfd8802d9c07a41e079d4bbaa9e436066dadb96).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 08 2025 at 19:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ff7f68366dfdbef6c7885992470d8883a151c848).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 08 2025 at 21:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a4dd12474903d8ddea1d13a02ba50c91c5935195).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 02:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1e0a22c4b304a2ae239466f03d6a9e5144b4acd9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 04:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (bac6a71fa83116a8c2ae39bbe323ff77982f8559).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 06:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (84bd3e991a2ef2163784901f76cd1229a8b73687).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 09:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (38938eb33835cc5c507306537ece9bfdfd92ff56).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 09:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1c54a07e9521261483aed57816c2169290626b9f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 13:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a1b5ed2427e9829b5270a33f27aef6c8a90e2e21).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 14:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ca7a22ba8f3fe6a761f7c8703e7bcbcda11e7069).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 16:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6382c1cee7fcfffda2ebe1738b977238ddac0294).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 18:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4593f6b663ee740802aba6405c85d5aa7d6ec00d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 09 2025 at 21:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b89ef87a41e16424e5111529de6ddc62711fb1e9).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 10 2025 at 00:13):

I have temporarily commented out the slow typeclass search test that has been failing for the last couple of days, hoping to get a green build again.

But we need to sort this out still. :-(

github mathlib4 bot (Sep 10 2025 at 00:15):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8bbff1856c14e96c1220c3805cbc9ab28cda343a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 10 2025 at 00:41):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (03abcf53054fb3e5138e0407f758919b4a0d8d01)

github mathlib4 bot (Sep 10 2025 at 03:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f0322dc5a8bdc3e97a815f4a055733488117c8da).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 10 2025 at 05:18):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (03abcf53054fb3e5138e0407f758919b4a0d8d01)

github mathlib4 bot (Sep 10 2025 at 10:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (82a044e0f6d552bd40084a43b3e91a0dc346ac1b).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Sep 10 2025 at 10:34):

Hmm getting hit by lean4#10317 again

github mathlib4 bot (Sep 10 2025 at 13:29):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0ab5d6dc754b1d07188cdd8072be2415bf88f410).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 10 2025 at 14:04):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f81ff0cf5025143c506c98ad3675c5db470f506e)

github mathlib4 bot (Sep 10 2025 at 16:15):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a585cf4b0b6d33dfd9aad8c8ac22c186627af1d6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 10 2025 at 19:41):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f81ff0cf5025143c506c98ad3675c5db470f506e)

github mathlib4 bot (Sep 11 2025 at 03:36):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (03abcf53054fb3e5138e0407f758919b4a0d8d01)

Kim Morrison (Sep 11 2025 at 10:08):

Kim Morrison said:

I have temporarily commented out the slow typeclass search test that has been failing for the last couple of days, hoping to get a green build again.

But we need to sort this out still. :-(

I've just restored this test. :-)

github mathlib4 bot (Sep 11 2025 at 10:35):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f81ff0cf5025143c506c98ad3675c5db470f506e)

github mathlib4 bot (Sep 11 2025 at 13:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6a13077c5bfbdabaa69f590e55207d8703129f02).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 11 2025 at 15:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5658f4e868d947da1d131524e7bcc1bf86f41a32).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 11 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (48ab2a0944ec17e2f56b24b0d3a17347010b5b92).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 11 2025 at 21:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0c4a789ffe6c0139467b91265cb8dc6e9a54f9e0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 11 2025 at 22:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (080113a9fb1294c38c8d464d49240b15d87f3176).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 11 2025 at 22:37):

@David Thrane Christiansen, similarly, could you please review bba7bb8f54d9 on Mathlib's nightly-testing, also regarding changes from lean#10307.

github mathlib4 bot (Sep 11 2025 at 22:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e0b8b8badcb9830b4a340e22f0ec2ac52bffdf8f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 11 2025 at 22:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e0b8b8badcb9830b4a340e22f0ec2ac52bffdf8f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 11 2025 at 22:42):

@Thomas Murrills, @David Thrane Christiansen, could I get one of you to review e0b8b8badcb on Mathlib's nightly-testing? Here validateDocComment has changed from CoreM to TermElabM, so is relatively hard to call from this position. However the surrounding comments, which I haven't taken the time to understand, suggest that it is perhaps no longer necessary. (I'm very happy to drop full support of string mode comments for to_additive, if that helps!) So my commit for now just removes the call to validateDocComment! :woman_shrugging:

Robin Arnez (Sep 11 2025 at 23:02):

Kim Morrison schrieb:

David Thrane Christiansen, similarly, could you please review bba7bb8f54d9 on Mathlib's nightly-testing, also regarding changes from lean#10307.

The bool flag is isVerso, again. I'm not quite sure when toModifiers gets used but doc.verso.get (← getOptions) might be a reasonable value. Also again, mkNullNode #[] would probably be a better default for binders.

github mathlib4 bot (Sep 11 2025 at 23:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0460eb84ed78102f683cefa4b36cdc298f582d32).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 12 2025 at 00:31):

Robin Arnez said:

Kim Morrison schrieb:

David Thrane Christiansen, similarly, could you please review bba7bb8f54d9 on Mathlib's nightly-testing, also regarding changes from lean#10307.

The bool flag is isVerso, again. I'm not quite sure when toModifiers gets used but doc.verso.get (← getOptions) might be a reasonable value. Also again, mkNullNode #[] would probably be a better default for binders.

Thanks, I've adopted both these suggestions. @David Thrane Christiansen, is you could take another look at this one that would be great.

Kim Morrison (Sep 12 2025 at 00:37):

The DeriveTraversable handler is broken on nightly-testing. It is not used in Mathlib, so for now I have just commented it out. I'm not sure if anyone is interested in rescuing it. It was last touched by Simon Hudon back in 2018. Please ping me here if you are interested in working on it. Otherwise I will prepare a deprecation PR for master shortly.

Kim Morrison (Sep 12 2025 at 00:42):

chore: deprecate Traversable deriving handler #29573

github mathlib4 bot (Sep 12 2025 at 01:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9a65e648970e99ee73c55b1cd5026c3d34d8a7d7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 12 2025 at 02:20):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1ee14ece202bee14a3cb8a48285b843095df8c70).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 12 2025 at 02:22):

Having trouble with shake here. This will still need a shake --update after the next build.

github mathlib4 bot (Sep 12 2025 at 03:41):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c9135c5fc71ebb63d4c7c80bee1c0071329ad9d5)

Thomas Murrills (Sep 12 2025 at 04:45):

Kim Morrison said:

Thomas Murrills, David Thrane Christiansen, could I get one of you to review e0b8b8badcb on Mathlib's nightly-testing? Here validateDocComment has changed from CoreM to TermElabM, so is relatively hard to call from this position.

Nothing will break immediately by commenting out vaidateDocComment, but we probably should not leave it like that!

(I'm very happy to drop full support of string mode comments for to_additive, if that helps!)

Unfortunately, since addDocstring has ascended to TermElabM too, such a change would no longer help us out (since attributes work down in abbrev AttrM := CoreM). (In fact, the TODO comment there should probably simply be removed now in favor of an adaptation note stating that more care needs to be taken.)

I'll start a separate zulip discussion (though it's possible @David Thrane Christiansen already has plans for what to do in this sort of situation).

Thomas Murrills (Sep 12 2025 at 05:39):

#lean4 > Adding docstrings from within attributes after lean4#10307

David Thrane Christiansen (Sep 12 2025 at 06:33):

The only problem that skipping validateDocComment might cause is that ill-formed links to the Lean reference manual will be caught at docstring-rendering time rather than docstring-adding time. Which is to say, you'd get a hover with an error message in it instead of red squigglies. This is not great, but I'll work on getting you the feature you need to eliminate that.

David Thrane Christiansen (Sep 12 2025 at 06:51):

https://github.com/leanprover/lean4/pull/10357 makes validateDocComment monad-polymorphic.

David Thrane Christiansen (Sep 12 2025 at 06:57):

And as @Robin Arnez worked out, doc.verso.get (← getOptions) is the right value for the Bool; failing that, it should be false rather than true (which would mean that said docstring is only ever in Markdown, which is an OK assumption for now).

github mathlib4 bot (Sep 12 2025 at 07:35):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c9135c5fc71ebb63d4c7c80bee1c0071329ad9d5)

github mathlib4 bot (Sep 12 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (dea79f03108f14a22fd9a7a3cd9cfd9092d70f2d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 12 2025 at 09:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (015925bde7216fd2b3dcb5d8738fac8492c9c40c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 12 2025 at 13:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (adffc256abd40495f29256a0fe9411b19dfb99a7).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Sep 12 2025 at 15:25):

Kim Morrison schrieb:

The DeriveTraversable handler is broken on nightly-testing. It is not used in Mathlib, so for now I have just commented it out. [...] Otherwise I will prepare a deprecation PR for master shortly.

I don't think it's fair to deprecate things just because they aren't used in mathlib; I believe the e.g. Functor deriving handler defined in the same file might be useful for some people. Anyways, I think I fixed it, I'll see how the build goes.

github mathlib4 bot (Sep 12 2025 at 16:38):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c1aa8dc90067cf84f56cfb9b452437223cc51936)

Kevin Buzzard (Sep 12 2025 at 22:07):

I guess the argument for pruning unused stuff from mathlib is that Kim has to keep the nightly-testing show on the road and this is a daily challenge for them.

github mathlib4 bot (Sep 13 2025 at 01:34):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c1aa8dc90067cf84f56cfb9b452437223cc51936)

github mathlib4 bot (Sep 13 2025 at 09:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5e75367745f224b0e928f2166bdd2d0665cfbe19).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 13 2025 at 09:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f3ab6aa3a8cf2e174d0bf4b7f8de0a6b4c545d91).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 13 2025 at 13:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a89e375dd84ea790bb45293955d6a9e13376d8e1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 13 2025 at 16:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d54657561441e89139d3305a594b449e220e5dca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 13 2025 at 19:29):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ca1004d5372a3fea99efaf06f3b23533753bfbbe).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 13 2025 at 22:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (324c8c1452559bd9f7d45c3a4098a7b0d1cf8776).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 14 2025 at 01:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (16094030a086b1a28a32408a3aaa84ab99baffec).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 14 2025 at 04:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c94be3e807280906ee53d49202f4985c82e5f345).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 14 2025 at 07:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3883da6eec1eb6ec117fa3daf20cc90861ca5d9e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 14 2025 at 08:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7748c712805e80d2f8bd2f513887ab6277466216).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 14 2025 at 12:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d3c1c7fb3eee4a07f485f1887fdaf31fac7b815d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 14 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b0d923ba5e2a6661da587aeaf33f35aa934e41fb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 14 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (18262b20769f2339759765c56c16acd05576f0b5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 15 2025 at 00:16):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (8a984e169a6584136d074abd730d95e52503d176)

github mathlib4 bot (Sep 15 2025 at 10:21):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (86840272ee346e3b58ad6d96b156696881fe7848)

Kim Morrison (Sep 15 2025 at 13:35):

Robin Arnez said:

Kim Morrison schrieb:

The DeriveTraversable handler is broken on nightly-testing. It is not used in Mathlib, so for now I have just commented it out. [...] Otherwise I will prepare a deprecation PR for master shortly.

I don't think it's fair to deprecate things just because they aren't used in mathlib; I believe the e.g. Functor deriving handler defined in the same file might be useful for some people. Anyways, I think I fixed it, I'll see how the build goes.

I think the criteria should be:

  • if it is used in Mathlib, or if it a leaf file but nevertheless "in scope" for Mathlib, then we should certainly be bringing it up to date as upstream dependencies change (or organising for fixes upstream to make this happen)
  • if it is a leaf file and arguably "out of scope" for Mathlib, but there are identifiable users, then we should attempt to keep it alive during updates, but we have the escape clause of asking those users to take responsibility for fixing it (either inside or outside Mathlib)
  • if it is a leaf file, out of scope, and there are no identified downstream users, then it's a good opportunity to clean up (e.g. comment out on nightly-testing, and deprecate on master)

github mathlib4 bot (Sep 15 2025 at 13:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a4e4a50dd491e3db03cfd498f234c8f17f4c327f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 15 2025 at 16:40):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (86840272ee346e3b58ad6d96b156696881fe7848)

github mathlib4 bot (Sep 16 2025 at 10:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e055bf02405f5b5773e7b915de6bf5783972f6d9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 16 2025 at 13:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (10051602bed8527d7bf2babc32f9b05a05ee13d0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 16 2025 at 16:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (45e487b3ee8f98b014a3f803fba3bc5e590b1252).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 16 2025 at 19:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fe04e9b1f01c3170e838b609c500da21ad44be74).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 16 2025 at 21:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (10051e8244ed7f8c66493b06c1db905acc2ccb6f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 17 2025 at 01:29):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (37737dd1cd6277bf9681be15531cd2d11159dc41)

github mathlib4 bot (Sep 17 2025 at 08:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4d6a0256252d25dac4608c9567ec77ed508fd4b6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 17 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a4b37b2423b87e1c289072f7279a75d29d536657).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 17 2025 at 10:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (526190d5eaa76b20872adf8331e9ab9725e35750).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 17 2025 at 10:59):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (90a85422a20137251a9edc48739a18fbeea15d6a)

github mathlib4 bot (Sep 18 2025 at 08:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (889210388069fc1940dddec996416cc897ecd50b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 18 2025 at 09:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3ef9899579f6babeabc2b3773d68a241e26a14ce).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 18 2025 at 11:53):

Kim Morrison said:

We need to build with

-- Compare old and new
set_option backward.grind.checkInferPatternDiscrepancy true
-- Use old
set_option backward.grind.inferPattern true

to identify files where the behaviour has changed, then in those files set

set_option backward.grind.inferPattern false

and change the grind attribute to plain @[grind], which will now give a list of suggestions.

I've now set these options in the Mathlib nightly-testing lakefile, so we can get CI to help.

Sebastian Ullrich (Sep 18 2025 at 12:04):

It looks like #10437 will be necessary to unbreak proofwidgets

Kim Morrison (Sep 18 2025 at 12:13):

lean#10437

Kim Morrison (Sep 18 2025 at 13:29):

Okay, I think I've fixed up the grind annotations. We may change the behaviour so ! remains the default for local theorems, in which case we can remove a few that I've just added.

Robin Arnez (Sep 18 2025 at 13:46):

We seem to have two conflicting fixes! @Kim Morrison, we should probably revert https://github.com/leanprover-community/ProofWidgets4/commit/524d83dedae24aad3660fd7bf28c1a6b431ee7bd

github mathlib4 bot (Sep 18 2025 at 14:26):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f1456087fae76f4362fa3107824c3f95522f71b9)

Kim Morrison (Sep 18 2025 at 22:37):

Robin Arnez said:

We seem to have two conflicting fixes! Kim Morrison, we should probably revert https://github.com/leanprover-community/ProofWidgets4/commit/524d83dedae24aad3660fd7bf28c1a6b431ee7bd

Yes, we can do it tonight once the nightly lands.

github mathlib4 bot (Sep 19 2025 at 07:08):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f1456087fae76f4362fa3107824c3f95522f71b9)

github mathlib4 bot (Sep 19 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5823fefe477a67e746cb05ab34756a849cf6ea27).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 19 2025 at 10:16):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (160e8ad2bd088f05994ef8964c96bac3b03e598a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 19 2025 at 13:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (572e219401d7aa06a47742227e70de230991c3f1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 19 2025 at 15:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0e0ad1cbc8227396cfbc05ecdfc8dd85f8c90491).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 19 2025 at 19:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e841a1387805b74b2da659043d69b02427ce4387).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 19 2025 at 21:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (298066b8c7fe42fa35dfe6389d6c95f48e961cbf).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 20 2025 at 01:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c8e4e42213c636079e09e7ca0f883386d239fd34).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 20 2025 at 09:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (37972575d233a0200b8b0477bc3ed3f30a38d365).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 20 2025 at 13:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b18e5d361cb36111822f91959a5be40338ca1258).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 20 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4efa14cbf1f9450dd68a3cccc7fc837dfcd828b3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 20 2025 at 18:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1e728803fbb687efcd5b3b4c34e67e4644b54034).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 20 2025 at 22:05):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ae800f6d21821d6101eae28687f37905a19b643e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 21 2025 at 00:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0ab22dd232a7ba67285ba69e6b31cb621469ae46).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 21 2025 at 13:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4f59a4dd4366c7f2dabd6453814eb9018007272c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 21 2025 at 15:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (68f672cba160d193cef36337016cb098ceb7f042).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 21 2025 at 19:17):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (349f6202acd4b325eb89db631ec779fc4a7911de).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 21 2025 at 21:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4ed318cd95e8b2d84b0c36f0fd9255be881a1aeb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 22 2025 at 00:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (46f697f11d3e75f8b317a8817dcb322c91ce73dd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 22 2025 at 01:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ec8929eec0d6a9cd506813fe028209fbf5fd43d2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 22 2025 at 02:13):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (8416b90e756b4bdf56b0de9c0d735986255d56d2)

github mathlib4 bot (Sep 22 2025 at 07:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b689b0d634b43605592337670185413c665856d7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 22 2025 at 08:53):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (8416b90e756b4bdf56b0de9c0d735986255d56d2)

github mathlib4 bot (Sep 22 2025 at 10:04):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c5605312dd4cbef30187192fdbaf3d0730fcb92d)

github mathlib4 bot (Sep 23 2025 at 09:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d5ea3b7f3019f49b5bbe7bfe31b93648b6aadf22).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 23 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7c6ee4d1cf67df1245090cb42548fa99d140c33e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 23 2025 at 11:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e606cfd77b2a4887d1ce852f06504d88ad9039e8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 23 2025 at 11:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (666f3426a9d5ee88913dcf6d257f84bbee9fba6f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 23 2025 at 13:56):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (815adf2464144efaabbba281977d6581609ba222)

github mathlib4 bot (Sep 23 2025 at 15:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (333e3d639db89867d9476114311810a94089c70c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 23 2025 at 18:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (bad876b689375495a77627abda7236ff9ea095fd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 23 2025 at 21:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8326cdde318a88c96cfa9002ba7905cf3dc9d55d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 03:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c530e201598ab08a1dfe57c7ee2a894b6258da91).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 06:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (41f69a4018f164c9be11e8c065271aa15b1943d3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 09:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fd030f4f168b52a4244ffa89037360673c853ab5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 09:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cbb146e7ac4cc5880f9e1ce747ce3e25371bb6fe).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 12:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (aabf6748849c12535c7eb9136f516a17d25b8f31).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e230e16ba033e114e7713b067dfeaef7633f9c45).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 18:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f1218c36a7cfc1644d2835a07bd0c2c3f685c5c5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 19:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (13e6aad6f761d148800e0c2060a1d6c7de7313ba).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 19:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (13e6aad6f761d148800e0c2060a1d6c7de7313ba).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 24 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0cbdd9890de3ec44b04e4f17868691724e8ae04e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 25 2025 at 00:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (96ab6a52dfca09b041f9fbe28f25d37e809672da).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 25 2025 at 02:23):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c1437285a5e1f7f19daf852142702ffbeaa1279d)

Kim Morrison (Sep 25 2025 at 05:17):

Just a heads up that I will be offline from about 24 hours from now until ~October 12, and so unavailable to fix problems on nightly-testing. Any attention to this from others very much appreciated. :-)

Ruben Van de Velde (Sep 25 2025 at 05:18):

Have fun!

github mathlib4 bot (Sep 25 2025 at 05:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4f48035147cc197b8f17c21cdee678bf19756668).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Sep 25 2025 at 07:01):

Oh hmm, looks like I didn't get access to nightly-testing after the move to forks

github mathlib4 bot (Sep 25 2025 at 07:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b63b8797effc3c8b17749945c2190b6f95b31e11).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 25 2025 at 10:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6e7ecde8145c50f2532fc67dd0809bfd30103080).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 25 2025 at 10:31):

Ruben Van de Velde said:

Oh hmm, looks like I didn't get access to nightly-testing after the move to forks

@Ruben Van de Velde, I've sent you an invitation to join the leanprover-community nightly-testing team, which should give you the necessary permissions.

github mathlib4 bot (Sep 25 2025 at 12:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0535eef8719b8d911c143530ce7228be4948f21b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 25 2025 at 13:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (658ea9bcb380a390b978757c1508ae2d09b26942).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 25 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e5af8a0473dbdbafe1753e27a939ea46a5448cd9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 25 2025 at 18:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c479358b3c7772e79fbe48445a5db3d88e67bb4d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 25 2025 at 21:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9c3512d04e785e6e468f092b132bef512d2a8b13).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 26 2025 at 00:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5afb2e8371acdf09593080cfa85dcc7cbd04be4b).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 26 2025 at 03:59):

Oooh, this is exciting. quote4's nightly-testing branch is the first Mathlib dependency to have moved to the module system, and lake exe cache is unhappy.

Kim Morrison (Sep 26 2025 at 03:59):

I think we need to add some file extensions to the list cache handles.

Kim Morrison (Sep 26 2025 at 04:00):

I think:

    (packageDir / LIBDIR  / path.withExtension "olean.private", false),
    (packageDir / LIBDIR  / path.withExtension "olean.private.hash", false),
    (packageDir / LIBDIR  / path.withExtension "olean.server", false),
    (packageDir / LIBDIR  / path.withExtension "olean.server.hash", false),

Kim Morrison (Sep 26 2025 at 04:04):

I added these in 6ad0b9e77b3bbe677c4898dfeb475ad7a64f33a5. Let me ping @Sebastian Ullrich, @Mario Carneiro, and @Mac Malone, as I'm running out of time before PTO and may not get this over the line.

Kim Morrison (Sep 26 2025 at 04:05):

Hmm, still failing, as we've got cached files available, that don't contain these files.

github mathlib4 bot (Sep 26 2025 at 04:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6ad0b9e77b3bbe677c4898dfeb475ad7a64f33a5).
You can git fetch; git checkout nightly-testing and push a fix.

Mac Malone (Sep 26 2025 at 04:08):

@Kim Morrison Is leantar even compatible yet with the OLean format used by the module system? I would presume that module parts are formatted somewhat differently than a full module. I guess that is a question for @Sebastian Ullrich and @Mario Carneiro ?

Kim Morrison (Sep 26 2025 at 04:46):

Indeed! If that's the case we'll need to revert https://github.com/leanprover-community/quote4/pull/103 against the nightly-testing branch (alternatively, temporarily pin the Mathlib nightly-testing lakefile's require statement to an particular SHA).

Kim Morrison (Sep 26 2025 at 04:51):

It would nevertheless be nice to get to the point of actually seeing an error message for leantar rejecting the new format.

github mathlib4 bot (Sep 26 2025 at 05:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (19120fefc79dcb7149b8de1df0bdd8e55e906622).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Sep 26 2025 at 06:11):

Okay, after touching the lakefile to invalidate the cache, it now fails while compressing to the cache ready for upload, but without any error message.

https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/18028218364/job/51299383767#step:24:24

Kim Morrison (Sep 26 2025 at 06:12):

Without any error message it's hard to know what's going on, but this would be consistent with leantar encountering a module-system-olean from Qq and exploding.

Kim Morrison (Sep 26 2025 at 06:13):

I propose we revert quote4#103 for now, and then on a branch off Mathlib's nightly-testing we can investigate further?

Johan Commelin (Sep 26 2025 at 06:47):

I think that makes sense, yes.

github mathlib4 bot (Sep 26 2025 at 07:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8fac228605412cdda5db6f5e3ead9b3ea2e9c254).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 26 2025 at 10:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0ef1b4d9d396e0d50e6dd155a49e0a2436141663).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Sep 26 2025 at 11:05):

I'll note that if leantar compressed .olean.server/.olean.private as a generic file, it should just work and be good enough until we get to porting Mathlib itself. But apparently leantar already tries to decode those files and then fails because it doesn't expect pointers across files. Note that the error message is a few pages up because of parallelism:

uncaught exception: failure in /home/lean/.cache/mathlib/leantar-0.1.16-pre2 #[/home/lean/.cache/mathlib/c34d47807362b7eb.ltar, .lake/packages/Qq/.lake/build/lib/lean/Qq.trace, -c, git=mathlib4@0ef1b4d9d396e0d50e6dd155a49e0a2436141663, .lake/packages/Qq/.lake/build/lib/lean/Qq.olean, .lake/packages/Qq/.lake/build/lib/lean/Qq.olean.hash, .lake/packages/Qq/.lake/build/lib/lean/Qq.ilean, .lake/packages/Qq/.lake/build/lib/lean/Qq.ilean.hash, .lake/packages/Qq/.lake/build/ir/Qq.c, .lake/packages/Qq/.lake/build/ir/Qq.c.hash, .lake/packages/Qq/.lake/build/lib/lean/Qq.olean.private, .lake/packages/Qq/.lake/build/lib/lean/Qq.olean.private.hash, .lake/packages/Qq/.lake/build/lib/lean/Qq.olean.server, .lake/packages/Qq/.lake/build/lib/lean/Qq.olean.server.hash]:

thread 'main' panicked at /project/src/lgz.rs:836:47:
index out of bounds: the len is 0 but the index is 2305843009213680257
note: run with `RUST_BACKTRACE=1` environment variable to display a backtrace

Sebastian Ullrich (Sep 26 2025 at 11:20):

The general idea is that .olean/.olean.server/.olean.private each have their own olean header with its own base address but pointers may point into the address space of files prior in that list /cc @Mario Carneiro

github mathlib4 bot (Sep 26 2025 at 11:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (dee33e95a79cc1316e54635016b51e6908c096fb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 26 2025 at 13:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9cdfe19d722653d82245284853df302912358b71).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 26 2025 at 16:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (276dd6b5a72db24fbb8665d93693910731d83220).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 26 2025 at 22:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7d00b7f51de230e6fcb0159f413ed4241d9cc8d3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 27 2025 at 10:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (58ae08fb1ed483486a3039a818e5be8c5e18efb2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 27 2025 at 13:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (020049f13a69cdcd81834d39f14247179661fb1c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 27 2025 at 16:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (06dc6545071306c2c90e52669432b9cb0b598ff1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 27 2025 at 19:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c4e3eb3deaf376a5fcbb1ddca646780316c94a37).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 27 2025 at 22:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3b7368e348780c0f0600c1197c34273c6dae507d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 28 2025 at 01:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6da53fa708b7196a725cefb032de88c4c47b4afd).
You can git fetch; git checkout nightly-testing and push a fix.

Mario Carneiro (Sep 28 2025 at 05:36):

Sebastian Ullrich said:

The general idea is that .olean/.olean.server/.olean.private each have their own olean header with its own base address but pointers may point into the address space of files prior in that list /cc Mario Carneiro

Note that module system oleans are supposed to be supported in the upcoming version of leantar that I've been preparing with Mac. The plan is to enable it at the same time as the local cache support

github mathlib4 bot (Sep 28 2025 at 10:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2120cf6d1f009ef4225ac5a353d0123dd16ead2b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 28 2025 at 13:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (144a6f544aa8de2b74777195f00c1d226bc079b2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 28 2025 at 16:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ad67ca8abe456bf507e3f3c04f46f17f1bc3c3f0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 28 2025 at 19:06):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (adba7c4862466eb8689edd2eea4bdb00fe28af3c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 28 2025 at 20:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (adba7c4862466eb8689edd2eea4bdb00fe28af3c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 28 2025 at 22:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c50a5525f69ad58ad9034b16d53f9395567c0a1f).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Sep 28 2025 at 22:14):

For some reason it seems like it's failing to upload the cache

github mathlib4 bot (Sep 29 2025 at 01:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b20b7ed23f231f211900ad0c59c294b073b5dfd8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 29 2025 at 07:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5d850d3c5ec0474f454aef4359bf5c512a667cf8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 29 2025 at 10:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (764ae2bb4a8020ffd8660f760bbdeaea9dcfd0ac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 29 2025 at 13:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (dcbbfc4d7be309a1ea56b77dcbbe2a3a82798ac6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 29 2025 at 16:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (278376142a70d5006587767a5f4e72f14fb73211).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 29 2025 at 19:13):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (73ed2839b81d466ba8777b533da0acea06577d6d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 29 2025 at 22:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (07dcec0ba6435e8c7a58571484a3573a16e52e0a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 30 2025 at 04:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (597bf947c26681388ad5ed3f4d958fd97deacada).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 30 2025 at 07:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9c3bb427fa8f3d8daca22183a4bdb68eb6b2b2c7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 30 2025 at 08:16):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (791bc4685b99033d3d2336c8caa27145f8a84f5b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 30 2025 at 10:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5db1fd1fa3854746dcedcf292599cc83d3d23e70).
You can git fetch; git checkout nightly-testing and push a fix.

Markus Himmel (Sep 30 2025 at 11:18):

Mario Carneiro said:

Note that module system oleans are supposed to be supported in the upcoming version of leantar that I've been preparing with Mac. The plan is to enable it at the same time as the local cache support

@Mario Carneiro is this already part of 0.1.16-pre2?

Mario Carneiro (Sep 30 2025 at 11:22):

seems not, I thought I had added it

Mario Carneiro (Sep 30 2025 at 11:22):

the trace file parsing for multiple-olean tarfiles is supported but not the actual olean parsing

Mario Carneiro (Sep 30 2025 at 11:23):

I think this will need to be fixed before mathlib's dependencies can be modulified

Sebastian Ullrich (Sep 30 2025 at 11:25):

Would not special-compressing these olean variations be a significantly simpler first step?

Mario Carneiro (Sep 30 2025 at 11:26):

I think this happens because they have a header that looks like an olean file

Sebastian Ullrich (Sep 30 2025 at 11:27):

Yes they do. But likely the file extension would be available to check there as well?

Mario Carneiro (Sep 30 2025 at 11:31):

done

Mario Carneiro (Sep 30 2025 at 11:33):

but I would like to release a proper parser soonish

Sebastian Ullrich (Sep 30 2025 at 11:34):

Thanks, that would be great! Let me know if any info is missing.

Mario Carneiro (Sep 30 2025 at 11:34):

what do you mean?

Mario Carneiro (Sep 30 2025 at 11:35):

let me know if you can't wait anymore for me to release a new version because your modulization PRs are blocked

Mario Carneiro (Sep 30 2025 at 11:36):

otherwise I will try to release a proper parser

Markus Himmel (Sep 30 2025 at 11:38):

The modularization PR for quote4 is already merged (to nightly-testing, not master), so we'll have to revert this until a new version of leantar is available.

Mario Carneiro (Sep 30 2025 at 11:41):

Note I'm at ITP right now so I don't have too much free time

Markus Himmel (Sep 30 2025 at 11:43):

That's fine. I'll just revert the Qq PR and you can take your time.

github mathlib4 bot (Sep 30 2025 at 12:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c5b4287e9750db1c1c9192af833bb3d0aa5997fd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 30 2025 at 13:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (91d85231c19572e2eb052210ef0042998541be1f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Sep 30 2025 at 14:47):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (7ec524ff29ebcf2708770ddf4d8d37f84a27e149)

github mathlib4 bot (Oct 01 2025 at 10:58):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e7ff8fecd7cbe4bbf06794c6baa154f6269980aa)

github mathlib4 bot (Oct 02 2025 at 09:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (67bf7c11fef2e81af67b36fa268010ac67d8aabb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 02 2025 at 11:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (472669a74f78b53aa2abf407435c6406d8d595d0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 02 2025 at 13:34):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f01e2ea4f5b8fdd61a5e1441d2343560a1c9b6d1)

github mathlib4 bot (Oct 03 2025 at 18:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (05acb6c3af9535ade2374304bab36a6d663d4ce5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 03 2025 at 18:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (61865c072e0e48678697113c9bd822263b469f35).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 03 2025 at 21:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cc3de921b27e75124186c406f4c469baa5d8d4f6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 04 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8e9a8409142b13a4dd0c531d49158057afc693d9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 04 2025 at 03:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f76e609368a08552752c8cfadfd47933128f2ce5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 04 2025 at 06:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7dce98c584239760884e81881f8397ab6907fbdb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 04 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0b7f245bc3b49ac1cd3f94eca338639f6fa1f98b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 04 2025 at 12:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9722f7e2237c572e31b43c72d034af886dbfabab).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 04 2025 at 15:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (624e914a3ee120139e21aba0072b3f8ab7302be7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 04 2025 at 21:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (153004c946eb30180b50c062c13ddc488f3ea2c0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 05 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f799cf4289c7122fab96d61c9d63725c92e2c2a3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 05 2025 at 12:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7df377d90dda14cca9ec96046db7d76657b998ef).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 05 2025 at 14:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (176ebb691065fa0386f9d41ae63f20e960389989).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 05 2025 at 14:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6683f5ddc87d7508320fa08ca604ab9769ea04df).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 05 2025 at 15:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ab78a68fc61117693334df054340a52a34f7c0d3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 05 2025 at 19:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ac8a764b52b88ac588443dbd5adc5c7a4dd5b623).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 06 2025 at 06:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c870f76ad56ecde0826479ba3909949169264e42).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 06 2025 at 09:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7d6d06d5006e3e86c11df71d2a298612d0b754ed).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 06 2025 at 09:22):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (904d9aa32a55625ea137f6f7d952270e8a9e1a64)

github mathlib4 bot (Oct 06 2025 at 11:43):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (7bb1cf18dad0e818b2dacb14fe1625b7e45f85fe)

github mathlib4 bot (Oct 07 2025 at 11:07):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (873e009aedeb816734ce388ad830cac6ff9e68c1)

github mathlib4 bot (Oct 07 2025 at 13:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (94fef1a4e88b73f261bd3fb897a1bca493f91bdf).
You can git fetch; git checkout nightly-testing and push a fix.

Markus Himmel (Oct 07 2025 at 14:30):

This seems to be a regression from leanprover-community/aesop#255, causing an aesop_cat in docs#CommAlgCat.instMonoidalCategory to run out of heartbeats. This also affects mathlib master, see #30298 (CI is still busy, but it fails on my machine).

@Jannis Limperg, do you have any opinions here? Do you think there is a way to change aesop to avoid this regression, or should mathlib try to work around this issue?

Jannis Limperg (Oct 07 2025 at 14:31):

Thanks for the ping, I'll try to figure out who needs to adapt.

github mathlib4 bot (Oct 07 2025 at 16:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (29a622dc36955c27b94f9565ba3b841de4b0bca9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 07 2025 at 19:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (19b2d2ece012026472980d1c17ffbadb98d1060f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 07 2025 at 21:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ed369c34ec0c08d69538ab1d250b636ebda4c972).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2025 at 00:57):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (344943d97ed094c2eb259341ebdcdedc243cf1b4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2025 at 03:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (104fa779cd9a131c1ba2fa86c9523be5fd5f9ab3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2025 at 06:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (41049a14be3e1882e838d16df92f58a8bdc425c9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2025 at 09:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f052386d3666d6e65a626d62b5b104f706e9e569).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2025 at 12:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d856b9b7d4b1a472c70198de23ce8ae4e1a07dd1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2025 at 15:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ab0b3a78efa0c1e032fa55bb63d18cf91ba8c709).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 08 2025 at 16:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (bceba31f4b6c715a4e6a83fb4493a136dd44acc1).
You can git fetch; git checkout nightly-testing and push a fix.

Joachim Breitner (Oct 08 2025 at 16:50):

Jannis Limperg schrieb:

Thanks for the ping, I'll try to figure out who needs to adapt.

Any news on this front?

github mathlib4 bot (Oct 08 2025 at 19:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (58cb65cfc0343e65d659f3aea855c66e966cbc67).
You can git fetch; git checkout nightly-testing and push a fix.

Jannis Limperg (Oct 08 2025 at 21:15):

See this PR for the Aesop breakage: https://github.com/leanprover-community/mathlib4/pull/30347

Fixing it requires only one heartbeat bump, but Aesop becomes 35% slower overall, which is a bit much. I'll revert this change in Aesop for now.

Jannis Limperg (Oct 08 2025 at 21:32):

aesop#256

github mathlib4 bot (Oct 08 2025 at 22:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6e9273f5e12a79cfdc0b2ce4536030c65d807413).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 09 2025 at 02:07):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (0bf50add06fd53f0e1df02728797cf1627a1b5f7)

github mathlib4 bot (Oct 09 2025 at 11:03):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c1e2e72e6a759e7cd35595bcb01e1dadda64273f)

github mathlib4 bot (Oct 09 2025 at 13:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (58101158d66f73821b7ce54dbb67e04497b9ae31).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 09 2025 at 16:55):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c1e2e72e6a759e7cd35595bcb01e1dadda64273f)

github mathlib4 bot (Oct 10 2025 at 09:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (039b56acae9c0aab7342d8b0d929a210935e1286).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 10 2025 at 11:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (df20867a9835bf94fef2af6864d129951f8da683).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 10 2025 at 13:59):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (106f523ecc75b845cf1509f717e2ae748639c4bc)

github mathlib4 bot (Oct 11 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a21c8bbb13ecd92dc0c838c4ffd2dc48a57390a8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 11 2025 at 13:49):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (759a866d90cdf45873827430bfa7e56312836f25)

github mathlib4 bot (Oct 11 2025 at 22:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (256708f422adb514710d09864670ad6ec5d5f181).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2025 at 01:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (556169194d932e268c0c157139eb62dcb4065b34).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2025 at 04:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (824f91d5ed71e3f08b69fd50ba788a0b628c8505).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2025 at 06:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9d611b790c52acf210d2e858dcfa9578aa3c50c8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2025 at 07:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f06bb3439ba08f5daf83e3953412c2f5b8fba018).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2025 at 11:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2fd965ad0351ddcc7be19f0725df76a17df56e9f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 12 2025 at 14:04):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (0a180fbdaef46603c83c310ae40dca54728d4a7f)

Kim Morrison (Oct 13 2025 at 01:55):

Lovely to see a green checkmark here on the day I'm arriving back from holidays!

@Mac Malone / @Mario Carneiro would either of you be able to give me an update on the status of leantar and/or lake cache? I'd like to cut the next release of Lean soon if possible, and would like to be able to start modulizing everything after that is out.

(Apologies if this is already discussed elsewhere -- I'm just starting to catch up on zulip on my phone while traversing airports.)

Mac Malone (Oct 13 2025 at 02:01):

@Kim Morrison lake cache is beginning use in core, so use in Mathlib will come significantly later. @Mario Carneiro will have to speak on leantar support for the module system. I have not been involved in that process. For the release, the one hurdle on my end I can think of is that there is a new leantar release for lake cache which is currently in use on nightly-testing. It currently uses v0.1.16-pre2, but I imagine we would one want to bump that up to v0.1.16 as part of the release process.

github mathlib4 bot (Oct 13 2025 at 04:06):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (0a180fbdaef46603c83c310ae40dca54728d4a7f)

Mario Carneiro (Oct 13 2025 at 08:14):

Is there a place I can test module olean packing with leangz? Is there a nightly branch which incorporates a modulization PR which fails currently?

Sebastian Ullrich (Oct 13 2025 at 08:17):

As far as we could tell, https://github.com/leanprover-community/mathlib4-nightly-testing/commit/19120fefc79dcb7149b8de1df0bdd8e55e906622 failed because of leangz/module system incompatibilities. Let's start a branch there?

Mario Carneiro (Oct 13 2025 at 08:25):

great, reproducing locally

Mario Carneiro (Oct 13 2025 at 08:26):

and FYI the file extension fix does work

Mario Carneiro (Oct 13 2025 at 08:28):

I see one cache issue I want to send upstream to mathlib: I would like the three olean arguments to be passed in a group and in order [olean, server, private]; what is currently being done is

cargo run --bin=leantar -- test.ltar \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.trace \
  -c git=mathlib4@19120fefc79dcb7149b8de1df0bdd8e55e906622 \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.olean \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.olean.hash \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.ilean \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.ilean.hash \
  ../mathlib4/.lake/packages/Qq/.lake/build/ir/Qq.c \
  ../mathlib4/.lake/packages/Qq/.lake/build/ir/Qq.c.hash \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.olean.private \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.olean.private.hash \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.olean.server \
  ../mathlib4/.lake/packages/Qq/.lake/build/lib/lean/Qq.olean.server.hash

Sebastian Ullrich (Oct 13 2025 at 08:29):

Makes sense.

github mathlib4 bot (Oct 13 2025 at 11:27):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (81b2656df338a656f46701b8114baac30739c671)

Mario Carneiro (Oct 13 2025 at 13:43):

Actually I take it back, I think it will be better not to have them as separate inputs at all. If it's okay I'm going to set it up so that it checks for the existence of .server and .private files regardless and packs all 3; you then only pass the main olean file and it figures out the rest.

Sebastian Ullrich (Oct 13 2025 at 13:46):

That's basically analogous to what lean -o does now so SGTM. I can't speak for lake cache but it I assume there will be a way to ensure that.

Mario Carneiro (Oct 13 2025 at 15:52):

Finished the compressor, I'll work on the decompressor tomorrow. For the moment I'm using a -m flag for module files so you can specify if you expect the file to exist, rather than silently ignoring the file if something fails

Sebastian Ullrich (Oct 13 2025 at 16:32):

Is that still easier than having leangz check for every .olean input whether paths for additional parts have been passed as well and if so process them together?

github mathlib4 bot (Oct 13 2025 at 16:46):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (81b2656df338a656f46701b8114baac30739c671)

Kim Morrison (Oct 14 2025 at 05:32):

Given that @Mario Carneiro is actively working on this, I'm happy to delay cutting v4.25.0-rc1 so we can test this, and hopefully beginning deploying the module system this cycle.

github mathlib4 bot (Oct 14 2025 at 07:50):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (81b2656df338a656f46701b8114baac30739c671)

Mario Carneiro (Oct 14 2025 at 08:13):

Sebastian Ullrich said:

Is that still easier than having leangz check for every .olean input whether paths for additional parts have been passed as well and if so process them together?

It would be possible to do this but there isn't much connecting the files other than being adjacent to one another on the filesystem. I prefer having the archive format just pack things as described in the command line in order, especially since we're assuming the inputs are generated by another program anyway

Mario Carneiro (Oct 14 2025 at 08:14):

For decompression you don't need to be so picky, you just say unpack this file and it does it

Mario Carneiro (Oct 14 2025 at 08:33):

ah, this doesn't work either, when combined with lake cache:

 "outputs":
 {"r": "566a8d63d6b18c9f.ir",
  "o":
  ["d818c56013bb70c4.olean",
   "a8b2e45898215027.olean.server",
   "c596252d9c20803c.olean.private"],
  "i": "3c8925ca84a04080.ilean",
  "c": "c126825f4f4250bf.c"},

the olean parts are all over the place, so you have to specify them separately

github mathlib4 bot (Oct 14 2025 at 10:48):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (81b2656df338a656f46701b8114baac30739c671)

Mario Carneiro (Oct 14 2025 at 12:00):

decompressor is working on completely trivial examples such as in the Qq test. In the end, I removed the -m and went back to the old CLI, the only constraint is that the three olean parts have to come in a group and in order

Mario Carneiro (Oct 14 2025 at 12:01):

pushed as leantar v0.1.16-pre3

Mario Carneiro (Oct 14 2025 at 12:02):

is there a mathlib branch for the cache changes?

Mario Carneiro (Oct 14 2025 at 12:28):

(I'm setting this work down for now, it needs testing now and perhaps @Mac Malone or @Kim Morrison can help on this front)

github mathlib4 bot (Oct 14 2025 at 16:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c7d70abd52ac916fb32813ed8c010307681c7fb2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 14 2025 at 19:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (46487c231f44b36440c4c440dc4ccffc86ba91ba).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 14 2025 at 21:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c6e65985e7e0f7f53f880b450ec34131c603d4f5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 14 2025 at 23:43):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (81b2656df338a656f46701b8114baac30739c671)

Kim Morrison (Oct 15 2025 at 00:20):

I've pushed 00dd146765e6e23ed993a25d9d6e9a131dd1e834, which bumps leangz, and deb7e14ce002e53d08891a3e99eefd2717da81c1, which attempts to use the modulized quote4 again.

github mathlib4 bot (Oct 15 2025 at 01:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5ffe548bd1d363427fca34b4d02b0b6da38dfb04).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2025 at 02:08):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a87897fc37568b533d7f0319002d13e8701f9c34).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2025 at 02:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (20129c2f94ac03aca2e00f0c8c06098a5fd61d8e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2025 at 04:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cda8e891afb8be29c1abd6fc2ab6ffb6ce83ff09).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 15 2025 at 04:41):

Argh, I'm so confused. It failed with lots of errors about things not having been found in the cache, but none of it is about quote4!

https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/18517049327/job/52772009720#step:8:7589

Kim Morrison (Oct 15 2025 at 04:44):

What is the distinguishing feature of

olean not found

Kim Morrison (Oct 15 2025 at 04:46):

I guess unfortunately I have tested two things at once here: moving to leantar 0.1.16-pre3, and switching the quote4 dependency to a modulized version, and I really should have done those one at a time.

Kim Morrison (Oct 15 2025 at 04:48):

I've reverted both, to make sure we get back to green. Then I'll do leantar first.

github mathlib4 bot (Oct 15 2025 at 04:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2a0f1ee28b67ad06de91c8c0eb4e2a2a31b53b47).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2025 at 05:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9c16fb7dc3ce6b175a1fd3b99ef396b0ce2d1cc6).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Oct 15 2025 at 06:41):

Should we do these experiments on a separate branch?

Kim Morrison (Oct 15 2025 at 06:50):

Unfortunately the failure in nightly-testing is not actually due to these experiments! It's failing even after reverting both.

Kim Morrison (Oct 15 2025 at 06:51):

But I'm feeling pretty stumped as to what is causing the failure. :-(

Sebastian Ullrich (Oct 15 2025 at 06:52):

Hmm, could it have anything to do with files uploaded from the experiments? Not sure how that could manifest as a miss though...

Robin Arnez (Oct 15 2025 at 06:56):

Aren't these just those files that don't have other dependencies?

Robin Arnez (Oct 15 2025 at 06:56):

It doesn't seem like it got any cache

Robin Arnez (Oct 15 2025 at 07:04):

Wait...

Uploading cache to Azure...
Compressing cache
No files to upload

Sebastian Ullrich (Oct 15 2025 at 07:09):

Let's try resetting/bumping rootHashGen once more?

Robin Arnez (Oct 15 2025 at 07:29):

Do we always emit .ir files, even with module system disabled? Because if not then

-    (packageDir / LIBDIR / path.withExtension "ir", true),
-    (packageDir / LIBDIR / path.withExtension "ir.hash", true),
+    (packageDir / LIBDIR / path.withExtension "ir", false),
+    (packageDir / LIBDIR / path.withExtension "ir.hash", false),

Sebastian Ullrich (Oct 15 2025 at 07:38):

It looks like Kim reverted that and the root hash, let's see if the next build passes

Robin Arnez (Oct 15 2025 at 07:39):

Yeah I guess if that one works then the next one I'd try would be the one with ir not required though

Sebastian Ullrich (Oct 15 2025 at 07:40):

Ah yes, you're right for the next module system run

github mathlib4 bot (Oct 15 2025 at 08:08):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (81b2656df338a656f46701b8114baac30739c671)

github mathlib4 bot (Oct 15 2025 at 10:07):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (789d7da56fa9f7fc78443b259673b0bfcab73402).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 15 2025 at 11:59):

As there at lots of new interesting failures on nightly-testing (and also Batteries/Qq/Aesop), when I get back to this tomorrow I'll investigate getting cache to work on the modulized Qq on a branch (starting from the green commit above), to avoid having to interact with the main nightly-testing work.

github mathlib4 bot (Oct 15 2025 at 12:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8fb3ae873be593e80a76daf6b0c88b0c54e7f014).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2025 at 15:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0a9f66d2a556a287885703bb8ba668e7d971a956).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 15 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6b832de385b24773084bf5e0afc077ef3818e85b).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 15 2025 at 22:53):

(This will stay broken until this evening, waiting on lean#10799.)

Kim Morrison (Oct 16 2025 at 02:27):

Kim Morrison said:

As there at lots of new interesting failures on nightly-testing (and also Batteries/Qq/Aesop), when I get back to this tomorrow I'll investigate getting cache to work on the modulized Qq on a branch (starting from the green commit above), to avoid having to interact with the main nightly-testing work.

I've started doing this in nightly#90.

Bumping leangz causes no problems, but as soon as we add

    (packageDir / LIBDIR / path.withExtension "ir", false),
    (packageDir / LIBDIR / path.withExtension "ir.hash", false),
    (packageDir / LIBDIR / path.withExtension "olean.private", false),
    (packageDir / LIBDIR / path.withExtension "olean.private.hash", false),
    (packageDir / LIBDIR / path.withExtension "olean.server", false),
    (packageDir / LIBDIR / path.withExtension "olean.server.hash", false),

(note that .ir and .ir.hash are optional here, unlike my previous attempt) then the cache check fails in the same way it did previously:

https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/18547466841/job/52868736303?pr=90#step:8:7594

Kim Morrison (Oct 16 2025 at 02:34):

Ideas very welcome. :-)

Thomas Murrills (Oct 16 2025 at 02:55):

Just in case it helps minimize anything (or provides a hint that the file content is not actually relevant?), I noticed the failing Batteries.Lean.Meta.Expr is a very small file, containing only a namespaced instance:

Batteries.Lean.Meta.Expr

(I'll also note, just to fact-find, that some of these failing files have no imports.)

github mathlib4 bot (Oct 16 2025 at 03:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (09c801ea5c5fd16373f8dfbd49b0d1cebe16c88d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2025 at 06:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0b36ca667a886519e167614f17cc46d14fe9ad24).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2025 at 09:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6c45e02c308972007ece49916cc1aedd227913bc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2025 at 14:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ee63490e8db33a2802ac4f1c33351e66cb5fef64).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Oct 16 2025 at 15:01):

New nightly has arrived but looks like there's still loads of inaccessible names (edit: ah, the previous fix may have focused on Batteries)? /cc @Joachim Breitner

github mathlib4 bot (Oct 16 2025 at 15:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ff99d94ff1cac8ed23019d2e7f79192c24016e77).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2025 at 18:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b4b94e10eff629a21d1fe94c9d446e2c2337e2c9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2025 at 21:33):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3aa31a7994adb7e167601f557893f52873920ab4).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 16 2025 at 21:47):

Fixed in lean#10809 and lean#10810. I'm intending to re-release nightly-2025-10-16 after those are in, otherwise I won't be able to get this green until Monday.

github mathlib4 bot (Oct 16 2025 at 23:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ab1cf50a3b334a5385c7e127157167cdf4380fb2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 16 2025 at 23:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fd11747f8806e54ebef10d92ea8e73938c49be0a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 17 2025 at 00:29):

I've just re-released nightly-2025-10-16.

github mathlib4 bot (Oct 17 2025 at 00:29):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1240e30a9efc3426ca095b4477b7055fc4e3c5ff).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 17 2025 at 01:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9da4d23e6d9f46c3cb9ebc3f81efa75c83e987b1).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 17 2025 at 02:16):

Ah, my efforts on nightly#90 (trying to use modulize'd quote4) are in vain: because of our new security measures, CI only uses the cache executable from the master branch, or nightly-testing branch for PRs to the mathlib4-nightly-testing fork. So the step I'm trying to test has to be done on nightly-testing itself.

I'm hopeful still (despite the failure above), that nightly-testing will get to green again shortly.

github mathlib4 bot (Oct 17 2025 at 03:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ea509a6cf819b09c735eb4cfd5843ece4390bf38).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 17 2025 at 05:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2f924cb79c413ce5cf158cf653bb8fe287622b1e).
You can git fetch; git checkout nightly-testing and push a fix.

Markus Himmel (Oct 17 2025 at 05:56):

During the Upload cache to Azure step here, we get a lot of HTTP 409 conflict "The specified blob already exists" error messages.

Then during the Verify cache step here it looks like we're fetching the wrong files for (some of?) mathlib's dependencies.

github mathlib4 bot (Oct 17 2025 at 06:03):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ebecc07d6165d213c650fb51d9a5adb48d711a0f).
You can git fetch; git checkout nightly-testing and push a fix.

Markus Himmel (Oct 17 2025 at 06:14):

It looks like this run now used the old nightly-2025-10-16 again, not the re-released one?

Kim Morrison (Oct 17 2025 at 06:15):

Hm, I deleted the toolchains from all the Hoskinson machines.

Kim Morrison (Oct 17 2025 at 06:15):

but yes

Markus Himmel (Oct 17 2025 at 06:15):

That job ran on hoskinson7

Sebastian Ullrich (Oct 17 2025 at 06:16):

Will the cache have to be invalidated as well? Maybe easier to use the PR toolchain after all if one of them is in the correct state?

Markus Himmel (Oct 17 2025 at 06:17):

In the last commit I force-invalidated the cache by incrementing rootCacheGeneration in Cache/IO.lean

Kim Morrison (Oct 17 2025 at 06:17):

We should get nightly-2025-10-17 shortly in any case.

Kim Morrison (Oct 17 2025 at 06:17):

I'm unfortunately about to go offline for the weekend. :-(

Kim Morrison (Oct 17 2025 at 06:20):

I see now that nightly-testing-2025-10-13 (when we last succeeded) actually had:

    (packageDir / LIBDIR / path.withExtension "olean.private", false),
    (packageDir / LIBDIR / path.withExtension "olean.private.hash", false),
    (packageDir / LIBDIR / path.withExtension "olean.server", false),
    (packageDir / LIBDIR / path.withExtension "olean.server.hash", false),

but these have been commented out on current nightly-testing. As far as I can tell, this shouldn't make any difference, because none of the upstream nightly-testing branches we're using are on the module system, so there shouldn't be any olean.private or olean.server files anywhere.

Sebastian Ullrich (Oct 17 2025 at 06:22):

If I succeeded in speeding up release CI, we should get a nightly in about two hours. Here's hoping I, or anyone else, didn't break it :smiling_face_with_tear:

Sebastian Ullrich (Oct 17 2025 at 06:22):

But if it's okay to fall back to PR toolchains on nightly-testing, I'm sure we'll find a working setup

Sebastian Ullrich (Oct 17 2025 at 06:47):

Sebastian Ullrich said:

If I succeeded in speeding up release CI, we should get a nightly in about two hours. Here's hoping I, or anyone else, didn't break it :smiling_face_with_tear:

Pre-testing at #10813

Kim Morrison (Oct 17 2025 at 07:00):

lean#10813

Sebastian Ullrich (Oct 17 2025 at 08:03):

It's green! https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/18585359830/job/52988031064

Sebastian Ullrich (Oct 17 2025 at 08:36):

Oops, it failed in the post-build step... https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/18585359830/job/52991839284 /cc @Marc Huisinga - looks like we can just update the test output there?

Marc Huisinga (Oct 17 2025 at 09:54):

aesop#259

I don't have merge rights for Aesop.

Sebastian Ullrich (Oct 17 2025 at 09:55):

Thanks! I think it's okay to point nightly-testing at your branch until it is merged

Sebastian Ullrich (Oct 17 2025 at 09:55):

That is, Mathlib nightly-testing

github mathlib4 bot (Oct 17 2025 at 11:26):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c84ee75fe89338a5ca15ea04ad57789461a5cc7a)

github mathlib4 bot (Oct 17 2025 at 16:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a349d1aa691cd597a8e5970325d9cb51310a7cea).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 17 2025 at 19:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (42fb65f75c09dba4b7a2c4bd1d0c9e9e7c4cb10f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 17 2025 at 21:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1b8918e9f7d6591414d0354289cec29fa1bab47d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2025 at 13:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ea4441a212713dc97ba09851574759d2e4caa710).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2025 at 16:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3284690d85f1592779d0e79083aff6ebc6cc67c3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2025 at 19:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5099a32a08c42f9b03cffc2182c118175fe6222c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 18 2025 at 22:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (125e5b4d14ef8e6b0c53c90ca39a9f7d62744bfd).
You can git fetch; git checkout nightly-testing and push a fix.

Mario Carneiro (Oct 18 2025 at 22:04):

Kim Morrison said:

I see now that nightly-testing-2025-10-13 (when we last succeeded) actually had:

    (packageDir / LIBDIR / path.withExtension "olean.private", false),
    (packageDir / LIBDIR / path.withExtension "olean.private.hash", false),
    (packageDir / LIBDIR / path.withExtension "olean.server", false),
    (packageDir / LIBDIR / path.withExtension "olean.server.hash", false),

but these have been commented out on current nightly-testing. As far as I can tell, this shouldn't make any difference, because none of the upstream nightly-testing branches we're using are on the module system, so there shouldn't be any olean.private or olean.server files anywhere.

reminder that in the last leangz revision, you need to pass the three files [olean, olean.server, olean.private] together in that order and with no intervening files (the hash files can come after in any order)

Mario Carneiro (Oct 18 2025 at 22:05):

Also, just to double check: in a non-module file, we only have .olean, and in a module we have .olean, .olean.server, .olean.private, even if the latter two are empty, right?

Mario Carneiro (Oct 18 2025 at 22:07):

empty module files compress very well btw, it's only about 2 extra bytes of content, so the majority of the space is in the extra paths themselves (which are left uncompressed in the archive)

github mathlib4 bot (Oct 19 2025 at 00:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3a09765e211bee40f7eebb7529a4b7dd90ba202a).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Oct 19 2025 at 10:20):

Kim Morrison said:

Ah, my efforts on nightly#90 (trying to use modulize'd quote4) are in vain: because of our new security measures, CI only uses the cache executable from the master branch, or nightly-testing branch for PRs to the mathlib4-nightly-testing fork. So the step I'm trying to test has to be done on nightly-testing itself.

If there already is a special case for nightly-testing, wouldn't temporarily adding another one for this branch be the simplest solution?

github mathlib4 bot (Oct 19 2025 at 10:29):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6f1b9cb04c16d61644c3fcecbd5b097f76ae1ec9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2025 at 13:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2ae9d73776a02cf003e7c3270edf2447948cdeec).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2025 at 16:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c2b96d5754b133e957736e3fa35c26a016a5a2b0).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 19 2025 at 18:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8ed5356eeb868bf878ced71b674c68b83efeefed).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 19 2025 at 22:31):

Marc Huisinga said:

aesop#259

I don't have merge rights for Aesop.

merged. (I merged master into nightly-testing, and then nightly-testing into this branch first, to get Github to show the desired diff.)

github mathlib4 bot (Oct 20 2025 at 00:16):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (3aad5efa232cac1b73faa6501e2e3056f23a261b)

Kim Morrison (Oct 20 2025 at 06:12):

Mario Carneiro said:

reminder that in the last leangz revision, you need to pass the three files [olean, olean.server, olean.private] together in that order and with no intervening files (the hash files can come after in any order)

Fixed now, thanks!

github mathlib4 bot (Oct 20 2025 at 06:34):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (3aad5efa232cac1b73faa6501e2e3056f23a261b)

Kim Morrison (Oct 20 2025 at 08:07):

Okay, nightly#92 is the new attempt to switch nightly-testing to using the modulized version of quote4.

Sebastian Ullrich (Oct 20 2025 at 08:20):

The suspense, having to wait for all of Mathlib to build first :) ... but I understand that adjusting the CI script to build less may not be easier than just waiting

Kim Morrison (Oct 20 2025 at 08:21):

I don't trust testing the cache in any way but exactly as CI does it...

Kim Morrison (Oct 20 2025 at 09:35):

Lots of errors during uploading the cache: https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/18646243547/job/53154174437?pr=92#step:24:7434

Sebastian Ullrich (Oct 20 2025 at 09:38):

"The specified blob already exists", is this unexpected? Does this not happen on other branches?

github mathlib4 bot (Oct 20 2025 at 10:57):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f23e0ba9024f6f842294066395815de292210482)

Sebastian Ullrich (Oct 20 2025 at 11:23):

2025-10-20T10:54:12.3153137Z packing ./Mathlib/Algebra/AddConstMap/Basic.lean as 84aa7d2e56c1e9f1.ltar

This is not the hash I get locally on the same branch

packing ./Mathlib/Algebra/AddConstMap/Basic.lean as ccb579e368ee0270.ltar

Mario Carneiro (Oct 20 2025 at 11:26):

Are there any nonempty module files in this test run? I want to make sure leangz is tested on module files that actually do something before the next release

Mario Carneiro (Oct 20 2025 at 11:27):

(The error sounds unrelated to leangz though, this hash is computed by lean exe cache)

Sebastian Ullrich (Oct 20 2025 at 11:27):

Yes, the PR should include quote4 fully ported

Mario Carneiro (Oct 20 2025 at 11:28):

by nonempty I mean the .server file is not the minimum possible size

Sebastian Ullrich (Oct 20 2025 at 11:29):

A single docstring is sufficient for that

Mario Carneiro (Oct 20 2025 at 11:30):

ah, I guess I was testing Qq.olean which would explain it

github mathlib4 bot (Oct 20 2025 at 12:22):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f23e0ba9024f6f842294066395815de292210482)

Sebastian Ullrich (Oct 20 2025 at 20:50):

@Kim Morrison As I couldn't push to your PR, I created a new branch right in the repo at https://github.com/leanprover-community/mathlib4-nightly-testing/pull/94 (and also I accidentally closed yours). A first test using only import Qq worked now, I think the only mistake before was that the cache changes were not active for the executable taken from master. I started a full run now, if that one works (Build (push), ignore Build (fork) for now) I think we can merge this minus the changes to build.in.yml.

github mathlib4 bot (Oct 20 2025 at 23:48):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f23e0ba9024f6f842294066395815de292210482)

Kim Morrison (Oct 21 2025 at 00:06):

Welcome to the module system! :-) Mathlib's nightly-testing is now using a modulized version of the quote4 library, and the cache system is working with it! Congratulations to everyone involved. :-)

I'm now starting the release of v4.25.0-rc1 as nightly-2025-10-20. We'll progressively move more of Mathlib's dependencies over to the module system during this cycle.

Kim Morrison (Oct 21 2025 at 00:25):

oh --- maybe not ... I now see that lean#10819 has not been merged yet, but is essential for module-izing Batteries.

We may end up cutting an rc2 with that.

github mathlib4 bot (Oct 21 2025 at 01:59):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f23e0ba9024f6f842294066395815de292210482)

github mathlib4 bot (Oct 21 2025 at 04:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9ffe5fd0791f1d271211fd961704b8f0a8d7f2af).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Oct 21 2025 at 05:48):

Ah my bad, I didn't remember I was using the same branch for batteries and now newer Mathlib fixes

github mathlib4 bot (Oct 21 2025 at 06:58):

:warning: Warning: The lean-toolchain file in bump branch `` does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: **File URL:** https://github.com/leanprover-community/mathlib4-nightly-testing/blob//lean-toolchain **Current content:**

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Oct 21 2025 at 11:22):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (afe13f6e909d350381903828473a7fe31be315cd)

github mathlib4 bot (Oct 21 2025 at 11:23):

:warning: Warning: The lean-toolchain file in bump branch bump/v4.25.0 does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: bump/v4.25.0
File URL: https://github.com/leanprover-community/mathlib4-nightly-testing/blob/9f149a1f6459fc0c00884abbab0db5006d0a1115/lean-toolchain
Current content: leanprover/lean4:v4.25.0-rc1

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Oct 21 2025 at 12:06):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (afe13f6e909d350381903828473a7fe31be315cd)

github mathlib4 bot (Oct 21 2025 at 12:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (83497509a86713ec3aa7c5895505520319afb997).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 21 2025 at 13:14):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (afe13f6e909d350381903828473a7fe31be315cd)

github mathlib4 bot (Oct 22 2025 at 03:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b14b433fa7c95050360991bc93ea63d0ad664968).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 22 2025 at 06:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d1609034e1b7a04689362d720b5d177ed0d8bc73).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 22 2025 at 09:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6c18cb8b60907b1c9398da5f7489e50c4f5608c7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 22 2025 at 12:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1e88c15c34c7527f472a52329fcddb849bce7974).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 22 2025 at 12:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f251ae5ed4014e18ea642e0b4b867fabea7dcd5b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 22 2025 at 15:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6e593a5a7b83f7c3f6e15e8ddba2f22af608eb1b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 22 2025 at 18:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b5bcd50aa92302a4e3a1367aab4a768107000037).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 22 2025 at 21:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cc0c98e71639d5239ac7c1b3e532f666fa3de0cb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 23 2025 at 00:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cd6ddfd1969a31b2958625e8110b1c26e2c0b835).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 23 2025 at 03:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5c3dd696b785d509ceafbc15ef3e36835b98e51f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 23 2025 at 09:07):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (df5d6b68a9a59dde331426d02d4d6c22c1c2cbe2).
You can git fetch; git checkout nightly-testing and push a fix.

Sebastian Ullrich (Oct 23 2025 at 20:27):

@Mario Carneiro I only just realized, is it correct that all the .olean variants of a module are stored in a single .ltar? That wouldn't allow us to skip downloading the .private data, which is not necessary for most uses. I assume the compressed .private data is/could be made a suffix of the archive data so that it could be saved in a separate .ltar.private, with only the main .ltar being necessary to decompress all other files

Sebastian Ullrich (Oct 23 2025 at 20:40):

As a simpler solution, we could also have cache upload separate .ltar.all and .ltar.all-but-private bundles, which should be <50% space overhead, so might be okay. I guess I could even use current leantar by passing a faux empty .private file for the latter archive, might give that a try tomorrow. Let me know if we should move this discussion somewhere else.

Kim Morrison (Oct 24 2025 at 00:25):

@Henrik Böving, Aesop's nightly-testing branch is failing as a consequence of lean#10625, could you please take a look? (Pinging @Jannis Limperg as well.)

Kim Morrison (Oct 24 2025 at 00:27):

(I think lean#10625 probably shouldn't have been merged until we knew how to fix Batteries/Aesop/Mathlib, as now we're preventing the testing of other PRs.)

Henrik Böving (Oct 24 2025 at 06:58):

I'm somewhat confused that this breaks, the instance from ST to MetaM still exists and works at the moment. If its written as a liftM (n := MetaM) instead it goes through.

Henrik Böving (Oct 24 2025 at 06:59):

I'll try to take a deeper look once I'm at the office

Henrik Böving (Oct 24 2025 at 08:41):

fix #10940

Henrik Böving (Oct 24 2025 at 14:25):

While building mathlib with this PR I noticed another funny new failure, the sleep heartbeats tactic: https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Util/SleepHeartbeats.lean has a test:

example : 1 = 1 := by
  sleep_heartbeats 1000
  rfl

this test basically runs

def sleepAtLeastHeartbeats (n : Nat) : IO Unit := do
  let i  IO.getNumHeartbeats
  while ( IO.getNumHeartbeats) < i + n do
    continue

and hopes that something bumps the heartbeats, but thanks to my optimizations this loop is now completely allocation free so this test just hangs, I would suggest to delete it^^

Henrik Böving (Oct 24 2025 at 14:29):

In any case I pushed an update using a PR toolchain from #10940 to nightly-testing of mathlib now so people can keep experimenting I guess

Sebastian Ullrich (Oct 24 2025 at 14:44):

Pushed a quick fix using new API

Mario Carneiro (Oct 24 2025 at 15:14):

@Sebastian Ullrich I think separate ltar.private is not a high priority. The files are not that big to begin with, file overhead is significant. I think more important than that is improving cache so that it doesn't have to download all 7000 or so cache files and unpack everything regardless of what part of mathlib you are using

Mario Carneiro (Oct 24 2025 at 15:16):

You can indeed make an all-but-private file easily, just don't include the .server and .private files in the archive

Mario Carneiro (Oct 24 2025 at 15:17):

if you want server but not private, that's not currently supported (I feel like I asked about that and was told it can't happen but here we are I guess) but it would not be hard to support

Sebastian Ullrich (Oct 24 2025 at 15:20):

I may have interpreted your previous question too specifically then: lake will never produce .server without .private but it still makes sense for cache to only produce the former. .olean.private is more than 50% of .lake, I would say that's a pretty great start!

Sebastian Ullrich (Oct 24 2025 at 15:21):

While we're at it, not sure I mentioned before that .ir can also be compressed as a (stand-alone) .olean file

Sebastian Ullrich (Oct 24 2025 at 15:22):

Agreed that in the future, we should save even more

Mario Carneiro (Oct 24 2025 at 15:22):

I want to not do this in the current dev cycle, it should be done as part of a clear user facing tool which needs it

Mario Carneiro (Oct 24 2025 at 15:23):

ltar use is a tiny fraction of olean use, you can just not unpack some parts of the archive

Sebastian Ullrich (Oct 24 2025 at 15:24):

True. Is that possible right now or would need a patch?

Mario Carneiro (Oct 24 2025 at 15:25):

that would need a patch, or you can delete files after the fact

Sebastian Ullrich (Oct 24 2025 at 15:25):

(but also I believe for some users downloading the ltars is still a significant bottleneck)

Mario Carneiro (Oct 24 2025 at 15:25):

downloading the ltars is significant but that is because they download all of mathlib, this is the main problem

Sebastian Ullrich (Oct 24 2025 at 15:27):

I would say these two optimizations are orthogonal so we should do both, in their own time

Mario Carneiro (Oct 24 2025 at 15:28):

but keep in mind what I mentioned about file overhead: we are already downloading a lot of files and file overhead is significant when it comes to curl. Splitting into 2 or 3 pieces will make that component worse and may cancel the benefits of downloading less

Mario Carneiro (Oct 24 2025 at 15:30):

another possible parlor trick is to take a ltar with a private section and truncate it off

Sebastian Ullrich (Oct 24 2025 at 15:30):

Yes but I would expect in 95% of cases you will only need the main file

Mario Carneiro (Oct 24 2025 at 15:30):

i.e. you don't need to repack to remove the private section

Sebastian Ullrich (Oct 24 2025 at 15:31):

We can experiment with this when we get there

Mario Carneiro (Oct 24 2025 at 15:33):

@Kim Morrison I released a non prerelease version of ltar, v0.1.16, which is the same as pre4. I think I missed the avenue to avoid having prereleases on master but could you add this to the PR? Is there a PR? I can't follow these processes very well anymore

github mathlib4 bot (Oct 24 2025 at 16:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cbe003a74d122d89e4614d515f37cf96fe37814b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 24 2025 at 18:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (21bbf68c1bf4a90e2060ca0922ca6087a867f0fb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 24 2025 at 21:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2dfc304d6bf71e4281b148e36f7f6f943a2b28c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 25 2025 at 00:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7db953b1c5d3fdef287052f1cc71200abdb32fb3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 25 2025 at 05:28):

Mario Carneiro said:

Kim Morrison I released a non prerelease version of ltar, v0.1.16, which is the same as pre4. I think I missed the avenue to avoid having prereleases on master but could you add this to the PR? Is there a PR? I can't follow these processes very well anymore

I will make a PR to Mathlib master moving to v0.1.16.

Kim Morrison (Oct 25 2025 at 05:30):

#30874

github mathlib4 bot (Oct 25 2025 at 06:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (64cd5c6eff27f7d865d4e12ea5b0cd9c6cfc8cbd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 25 2025 at 10:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (201b0f136af351277af1ff1ed19263bb8c0ce846).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 25 2025 at 12:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1ab508e0740e3dfa8bafe1a060b300193f17140f).
You can git fetch; git checkout nightly-testing and push a fix.

Markus Himmel (Oct 25 2025 at 12:13):

Lots of aesop tests failing with aesop.check.tree: search tree contains a cycle.

Sebastian Ullrich (Oct 25 2025 at 12:22):

Now that sounds like an especially strange failure. /cc @Jannis Limperg

github mathlib4 bot (Oct 25 2025 at 13:08):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (94c44aac99a307dcaf6258aad01c1fade4ffaf93).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 25 2025 at 19:27):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d0bc5692ff0733547faccd064fb5f63d9fc8d64a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 25 2025 at 22:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d76573adf01e5d26e0b4b0bbee9d32ebea7c298a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 25 2025 at 22:48):

I've temporarily removed the AesopTest build from nightly-testing CI, so we hopefully get to green again...

github mathlib4 bot (Oct 25 2025 at 23:07):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (b1e9ded89f681a414f4fe43319a9a0372fe4e750)

github mathlib4 bot (Oct 26 2025 at 10:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (94930ab4a8c644cb0a19819f98ac8276a5016d55).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 26 2025 at 11:13):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (7d2e53aea6e90d6ff50f8081615c53963d000623)

github mathlib4 bot (Oct 27 2025 at 10:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0c52b458f6e0640e57b7c5c4334a7e85177385f9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2025 at 11:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (260dcb323a629242b0188e471f1f538e5bc7734d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 27 2025 at 14:04):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (daa21570b791337ce33135a2d2acceab9c451734)

github mathlib4 bot (Oct 29 2025 at 02:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (965e3c7a87024728ff1f41a7670a0a3c3b09a6dc).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 29 2025 at 02:19):

lean#10934 broke two proofs in Mathlib, @Henrik Böving and @Robin Arnez.

Kim Morrison (Oct 29 2025 at 02:25):

I've pushed horrific temporary fixes in f512a44ba0.

I'm tempted to suggest that we revert #10934 and then proceed more gradually, to find out which annotation change caused this problem. Other ideas?

Kim Morrison (Oct 29 2025 at 02:27):

(There are some other failures from the same cause, but at least grind happily handles these. These changes are in 84c2cec795.)

github mathlib4 bot (Oct 29 2025 at 03:30):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (84c2cec795e7d2aa67cbdccfe8178412d3aead85)

Henrik Böving (Oct 29 2025 at 07:18):

I'd assume it was not any of the annotations but the fact that rob also changed the implication instance on the fly?

Henrik Böving (Oct 29 2025 at 07:19):

I'll revert that part and see if it breaks

github mathlib4 bot (Oct 29 2025 at 07:38):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (84c2cec795e7d2aa67cbdccfe8178412d3aead85)

Robin Arnez (Oct 29 2025 at 07:47):

Right, see also what happened at https://github.com/leanprover/lean4/pull/10934/files#diff-37a274b16b6fff0fa57265829a44c1e9556ea3cadff1f4297b2f3bbe7a4d89aa, the fix should be to add synthInstance.maxSize somewhere (athough it feels like this is a bug)

Robin Arnez (Oct 29 2025 at 07:52):

To be precise, the maxSize calculation somehow decided to be exponential in regard to depth rather than linear.

github mathlib4 bot (Oct 29 2025 at 09:03):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (84c2cec795e7d2aa67cbdccfe8178412d3aead85)

Henrik Böving (Oct 29 2025 at 09:28):

Okay I have a reverter open here #11007 and the more tame version here #11008 based on top of nightly-with-mathlib, it doesn't trigger the instance size explosion in the grind test and I also tested it against mathlib precisely without @Kim Morrison fixes applied and tested against the PR toolchain here https://github.com/leanprover-community/mathlib4-nightly-testing/pull/101/files, I'll merge the more tame Decidable fix to master once that is finished.

github mathlib4 bot (Oct 29 2025 at 10:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (62bbeed300d9533ecafc02e0717f7134852f7d07).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2025 at 11:49):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e3d159a14fe17c79b953b7d56f38ebdde8248062)

github mathlib4 bot (Oct 29 2025 at 16:03):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (836def65b0448631b143fa6586647d88a72edee8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2025 at 19:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1e3d8d42502d0f1029ff24d659034001d98a8634).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2025 at 22:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a75fd12d1fe66eeab66f90c82070973827d1c3ce).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2025 at 22:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (285dee2607c094561df0237856babda8e60e1458).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 29 2025 at 23:10):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e3d159a14fe17c79b953b7d56f38ebdde8248062)

github mathlib4 bot (Oct 30 2025 at 09:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c64b47e6f3fb73f3e7789ccf6e2e417a79f7e4af).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2025 at 10:15):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (97af697c999f402cbe99e6a9dc288c8ec11e8b5a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2025 at 12:05):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (cb0e79929e2a5a2d642721c39b4eb7f89556842e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2025 at 13:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7e956ac8ce15d16a18c391826db47692d643ea2c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2025 at 15:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ee2618e9bf79552fd00ad341e51daa8fe2293e29).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2025 at 19:17):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5856e8689004ed6e3bf1dfaa734a9bab1f621b37).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 30 2025 at 20:29):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (985e8a879b3b159f02f4531edc11f5d3be60d65b)

github mathlib4 bot (Oct 31 2025 at 10:17):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (710a14e42521cda96239ddf119c275cfbf7490dd).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Oct 31 2025 at 10:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (63a6a335a75f64bb4070ad61c5be013008c38a51).
You can git fetch; git checkout nightly-testing and push a fix.

Markus Himmel (Oct 31 2025 at 10:46):

@Kim Morrison I have temporarily commented out the premise selection test that you added recently because I really need this nightly-with-mathlib. I don't understand what the problem is; it fails because it doesn't recognize the set_premise_selector command.

github mathlib4 bot (Oct 31 2025 at 10:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fbc746105b79879635ee31215ede6dca1a613e0e).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Oct 31 2025 at 10:56):

Markus Himmel said:

Kim Morrison I have temporarily commented out the premise selection test that you added recently because I really need this nightly-with-mathlib. I don't understand what the problem is; it fails because it doesn't recognize the set_premise_selector command.

No problem, I'll fix it later.

Kim Morrison (Oct 31 2025 at 11:00):

There are several failing tests. Easy to fix, I'll do it now.

Markus Himmel (Oct 31 2025 at 11:00):

Already done :)

Kim Morrison (Oct 31 2025 at 11:01):

Did you push? I still see symbolFrequency.lean and TacticAnalysis.lean tests with failures.

Markus Himmel (Oct 31 2025 at 11:01):

No, I got a conflict with your commit

Markus Himmel (Oct 31 2025 at 11:02):

So I'll let you do the s/PremiseSelection/LibrarySuggestions

Kim Morrison (Oct 31 2025 at 11:02):

Pushed.

github mathlib4 bot (Oct 31 2025 at 11:24):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (5acb7976977f197185d79a16e6a4a12beb6e96f8)

github mathlib4 bot (Nov 01 2025 at 13:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (606d1ed9e20b323ede055394ef5d18367fdaff2f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 01 2025 at 16:24):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c4ff0c86bc3e0995b2e9e572445cd71faa52e7a2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 01 2025 at 19:08):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2357a5579f4ceecda62bdae3a82384f1e5a55335).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 01 2025 at 22:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3dc2d5a585a56df108592274b9b5bcf5748fcb08).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2025 at 01:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (318efa2722d9da2d9de6dfae77c32d4e2531c83a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2025 at 09:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f7b5c8b4c7d082b00f822b5404fcd03e1295c87e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2025 at 13:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (accdc1e677b3a6b58cc8566ce410b98d6faa0c55).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2025 at 19:16):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (07e675e5870e5312fc892146ecf44ae1d29d9719).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 02 2025 at 22:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fc62d02c25c970cdb807d6d3e08095405c4e383f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 03 2025 at 01:28):

I'm having a bit of trouble with a grind proof in FiveWheelLike by @John Talbot. (Pinging, as maybe they can help me out. :-)

We have a proof that used to be by grind, which by grind => finish? tells us was just running

by
  cases hw
  grind => lia

which is succeeding on nightly-testing-green but now fails on nightly-testing. Leo made quite a few changes to the order and offset modules over the weekend, so something in there has caused this to break. However I'm having trouble sorting it out and would like to be able to move on to other things.

Would anyone be interested in trying to get this proof to work again on nightly-testing?

The lia call now fails with:

[cutsat] Assignment satisfying linear constraints 
  [assign] r := 0
  [assign] k := 0
  [assign] #{x |  y : α⦄, y  s  t  G.Adj x y} := 0
  [assign] #{x |  y : α⦄, y  s  t  G.Adj x y} := 0
  [assign] #(s  t) := 0
  [assign] #({v}  ({w₁}  ({w₂}  (s  t)))) := 3
  [assign]  w  s  t, G.degree w := 1
  [assign]  w  {v}  ({w₁}  ({w₂}  (s  t))), G.degree w := 0

which is easy to contradict, but I haven't explored further.

github mathlib4 bot (Nov 03 2025 at 02:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (768853f0f3097af2b2d5594fbfbd804d98eaa9cf).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 03 2025 at 04:26):

I've now commented out the broken proofs in FiveWheelLike in 34e039175fd7f4eaa7635f9e0df6dc3299ea0b73. This commit can be reverted by anyone interested in fixing this.

github mathlib4 bot (Nov 03 2025 at 04:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (34e039175fd7f4eaa7635f9e0df6dc3299ea0b73).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 03 2025 at 05:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (34e039175fd7f4eaa7635f9e0df6dc3299ea0b73).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 03 2025 at 05:29):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (33840e37a495d9b79526a589490bf83284e930e6)

John Talbot (Nov 03 2025 at 08:27):

@Kim Morrison I'll take a look at this and try to fix it

John Talbot (Nov 03 2025 at 08:50):

I've fixed that proof but I'm afraid I wasn't sure how to push this to the correct branch so it is currently just on my fork here:
https://github.com/jt496/mathlib4/blob/nightly-testing/Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean

github mathlib4 bot (Nov 03 2025 at 09:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (72845e7ce6d2d742c4d9df77ea1ad1204ac75bb4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 03 2025 at 09:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (bca39ae6a868cbfe21fd893309d1f5a25fefd448).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Nov 03 2025 at 11:02):

John Talbot schrieb:

I've fixed that proof but I'm afraid I wasn't sure how to push this to the correct branch so it is currently just on my fork here:
https://github.com/jt496/mathlib4/blob/nightly-testing/Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean

No problem, I merged it

github mathlib4 bot (Nov 03 2025 at 11:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (add50e23d91d066a323fc4cae583b4a9ed4f13e3).
You can git fetch; git checkout nightly-testing and push a fix.

Kevin Buzzard (Nov 03 2025 at 11:27):

John Talbot said:

I've fixed that proof but I'm afraid I wasn't sure how to push this to the correct branch so it is currently just on my fork here:
https://github.com/jt496/mathlib4/blob/nightly-testing/Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean

Thanks John!

github mathlib4 bot (Nov 03 2025 at 11:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (34c91bbb55ab93afdedadee3cec375a5015784d3).
You can git fetch; git checkout nightly-testing and push a fix.

Robin Arnez (Nov 03 2025 at 13:25):

Uhh why did we revert back to nightly-2025-11-02?

github mathlib4 bot (Nov 03 2025 at 13:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a47fa22bd8a189d18f2f911918970d794c8b6317).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 03 2025 at 13:47):

Ah, my mistake. I was get nightly#102 back up to date to merge, and since Kevin made review suggestions there, I then merged it back into nightly-testing, accidentally reverting the toolchain.

github mathlib4 bot (Nov 03 2025 at 16:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5e92d2192edda6a4404e971f67119ab96213406d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 03 2025 at 19:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c3f4d1884d690b3d2b7355153d6bd7f5877e44ed).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 03 2025 at 22:29):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (acf34bc18983fb91e327df30cfa40ad5b2d01cab).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 03 2025 at 22:46):

I've hit merge on

chore: adaptations for batteries#1441 #30138

and separately merged it directly into nightly-testing.

github mathlib4 bot (Nov 03 2025 at 23:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f34c9529d58844e81e1af789557c7c470a2a3767).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 03 2025 at 23:37):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (d6788bb1834fce9d0e2e8ef5dc8e0205bb834190)

github mathlib4 bot (Nov 04 2025 at 10:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a818e5c09a1890d982b8955d543b7be869fa6cca).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 04 2025 at 12:32):

Oops, I pushed a commit removed Std.TreeSet.union, as this now exists upstream. However it seems the behaviour of that union is different, as the linarith test that depends on it now fails.

Kim Morrison (Nov 04 2025 at 12:33):

I need to go to sleep, but in the morning I will probably just restore this function under a different name to preserve this functionality in linarith (oracle := .fourierMotzkin).

github mathlib4 bot (Nov 04 2025 at 12:40):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9fc6a3e4e1107a30c92b1048be0e6e438c5a93ba).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2025 at 13:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (dcb488fd18ecce58f31c10fddbb46bfff82e9285).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2025 at 16:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7fda47fdf555e21e7a99c959fb1c460ccd8e95ba).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 04 2025 at 19:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (465be79baafa77804aa4298981812722f757755c).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 04 2025 at 21:25):

I've pushed a fix, renaming the FourierMotzkin implementation of union to union', and making it private. 92404470b1

@Wojciech Różowski, you may want to sanity check this, or at least be aware that there are downstream implementations of union which differ from yours in lean#10896!

Robin Arnez (Nov 04 2025 at 21:25):

I wonder how the two implementations could be much different. Is it order of arguments or something?

Kim Morrison (Nov 04 2025 at 21:27):

The new implementation adds the items from the smaller map to the bigger one. That presumably affects not-distinguished-by-the-order-but-unequal keys.

Robin Arnez (Nov 04 2025 at 21:29):

I'm not sure how this could be the case, see e.g.

theorem getKey?_union [TransCmp cmp] {k : α} : (t₁  t₂).getKey? k = (t₂.getKey? k).or (t₁.getKey? k)

Robin Arnez (Nov 04 2025 at 21:30):

Actually, I get it, TreeSet.insert uses insertIfNew, right? Then it feels like we should just simply need to swap the order.

Robin Arnez (Nov 04 2025 at 21:31):

The previous implementation favoring the key in the first map and the new implementation favoring the key in the second map

Kim Morrison (Nov 04 2025 at 21:32):

(I'm disinclined to touch this, as the Fourier-Motzkin oracle is unused outside of tests, and moreover grind, but I won't oppose cleaning it up!)

github mathlib4 bot (Nov 04 2025 at 22:48):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c0d7bf79ec8f3779573bc645e3850830f82a9cf4)

Wojciech Różowski (Nov 05 2025 at 10:55):

Thanks @Kim Morrison for flagging this. Yes precisely, in the case of HashSet insert is implemented in terms of insertEntryIfNew, which results in a swapped order of prioritising elements. In the union I implemented that relies on insertEntry (modulo swapping the order in order to iterate through the smaller collection, but behaving the same way as if we would just keep folding using insertEntry).

github mathlib4 bot (Nov 05 2025 at 10:56):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (30907b8b266fae6fbb6806989d03c56bd145a07b)

github mathlib4 bot (Nov 06 2025 at 09:07):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (939eb24b6ae71f6c9b48213fda9524bcd721d5c2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 06 2025 at 09:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d8bae1c8cbf664c31071c533791bb71657cfaf9e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 06 2025 at 10:52):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (ffe067087265bbba429df3ccf633e3ae7c77f82c)

github mathlib4 bot (Nov 07 2025 at 01:07):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0c28cbcc470eba3105750fa4bb7e6330bb6e81ee).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 07 2025 at 09:52):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9c3a040c0ecfaa83dd2bc1079ff4801c52efdc55).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 08 2025 at 02:08):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9ad89e3cafc256baf3475ae573e04be4f4a6dd15)

github mathlib4 bot (Nov 08 2025 at 10:55):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c68d05605c852bffb5dd07fb4a0fa4e7c91b7e2b)

github mathlib4 bot (Nov 10 2025 at 03:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3366f6ffda0db07663a96a587701ecccd801ff66).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 10 2025 at 04:08):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (c68d05605c852bffb5dd07fb4a0fa4e7c91b7e2b)

github mathlib4 bot (Nov 10 2025 at 10:42):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (41b823e92c33dc95da631526f176a2bae82580c6)

github mathlib4 bot (Nov 11 2025 at 09:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (813a62d001314d3d98cd8f23efc48c420388563b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 11 2025 at 11:08):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (2eeab6fa823e239db2f59f20195db3f6e5c49fb6)

github mathlib4 bot (Nov 12 2025 at 09:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9bff135922fcb5025f16fc7e5f184af4368b8ca3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 12 2025 at 11:17):

FromLRAT is failing, after changes to the String API. I've commented it out in 6f868c676a6. @Mario Carneiro, pinging in case you want to restore it. Given that we now have bv_decide, and FromLRAT has apparently been unused for some time, an alternative might be to simply remove this file?

github mathlib4 bot (Nov 12 2025 at 11:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6f868c676a6eb7e082e68d2308b88ed50a80d8d5).
You can git fetch; git checkout nightly-testing and push a fix.

Markus Himmel (Nov 12 2025 at 12:14):

Kim Morrison said:

FromLRAT is failing, after changes to the String API.

I fixed the issue and restored the file. The issue wasn't with the string API, it was due to the fact that the file uses Std.Internal.Parsec, which, being an internal module, changed its API without notice.

github mathlib4 bot (Nov 12 2025 at 12:35):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (e1d1dcb6e3708c37cf66910bc2171eafd187b128)

github mathlib4 bot (Nov 13 2025 at 09:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (882e24b0fe45e171c98fd0494d4a6ebbefb5824d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 13 2025 at 11:21):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (97d6356132c827bf339c05d8ea55f7a5dc7fdeb9)

github mathlib4 bot (Nov 14 2025 at 10:29):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f4335cd9c56b7706c69fe88c29ca6a0fe48ca51e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2025 at 11:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c18e6a6c17ad92c238a19d340a77ade2d2a6592a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2025 at 12:24):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (97d6356132c827bf339c05d8ea55f7a5dc7fdeb9)

github mathlib4 bot (Nov 14 2025 at 14:05):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fa1afaf589fea9433b1fd1a6d8fa623727cc9b0e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 14 2025 at 15:35):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (164dd5447ea6d466353ad9a3c08e0c7d7ff04544)

github mathlib4 bot (Nov 15 2025 at 10:23):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (a1f446e15624935672950bad32dcbf83ab856e34)

github mathlib4 bot (Nov 16 2025 at 00:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (22f65ecb8d8277c06aa54e12efa281e803ed1ac4).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 16 2025 at 09:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (97873b88a8bff66172aec9670197fa51994a710a).
You can git fetch; git checkout nightly-testing and push a fix.

Bryan Gin-ge Chen (Nov 16 2025 at 12:09):

Is fixed by #31182

Kim Morrison (Nov 16 2025 at 22:20):

I had to do the merge of master into nightly-testing manually, because of the conflict in lake-manifest. Hopefully going green soon.

github mathlib4 bot (Nov 16 2025 at 23:30):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (7678c2762c87b7b7262e0800ee1732b41da1912e)

github mathlib4 bot (Nov 17 2025 at 09:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (da2bffe0acdf6fd3470fbeb518c0d249556323c6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2025 at 11:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (de24f50673bcc7bd24050a804d0b0f09c2b71030).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 17 2025 at 12:07):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (eda6b9680a758291aa990e6c7dfa0634f00a8f6b)

github mathlib4 bot (Nov 18 2025 at 01:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (780cbe2da5302ccce8e15061c51f458e969c92dc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2025 at 08:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7f17921568ced599a72d89f4e1998d8c550f85bb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2025 at 09:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b6524e53ac184e081455ec5a7fe9b1b628f73929).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 18 2025 at 11:23):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9e00cef02259376402a852f54693de74e8f84d7a)

github mathlib4 bot (Nov 18 2025 at 11:23):

:warning: Warning: The lean-toolchain file in bump branch bump/v4.26.0 does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: bump/v4.26.0
File URL: https://github.com/leanprover-community/mathlib4-nightly-testing/blob/ec1e4cdcb8cb71da49a21995de8814795ea7b07f/lean-toolchain
Current content: leanprover/lean4:v4.26.0-rc1

This needs to be fixed for the nightly testing process to work correctly.

github mathlib4 bot (Nov 19 2025 at 01:56):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9e00cef02259376402a852f54693de74e8f84d7a)

github mathlib4 bot (Nov 19 2025 at 01:57):

:warning: Warning: The lean-toolchain file in bump branch bump/v4.26.0 does not match the expected pattern 'leanprover/lean4:nightly-YYYY-MM-DD'.

Branch: bump/v4.26.0
File URL: https://github.com/leanprover-community/mathlib4-nightly-testing/blob/ec1e4cdcb8cb71da49a21995de8814795ea7b07f/lean-toolchain
Current content: leanprover/lean4:v4.26.0-rc1

This needs to be fixed for the nightly testing process to work correctly.

Kim Morrison (Nov 19 2025 at 03:16):

I've just created bump/v4.27.0 from master, and set the lean-toolchain there to nightly-2025-11-17. Hopefully that will resolve these warnings.

github mathlib4 bot (Nov 19 2025 at 04:02):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9e00cef02259376402a852f54693de74e8f84d7a)

github mathlib4 bot (Nov 19 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c1eeffd21f26d256dabde384640f860dfef1bc55).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 19 2025 at 11:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (57450663f40fe18b64e4a7cca730c70436d6bc6d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2025 at 01:16):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (8068277c3ab280502aecf3c5100d7dd55806c53a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2025 at 09:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d98fdec7586dc0a2a1ac9f838eaa472b1969c977).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2025 at 11:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (37c4d0a97624eee2dd14930a2bbe32f8bdcc9f7d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 20 2025 at 12:29):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (3dc572b55ec47e50cd184d2b8053cab9e91d4450)

github mathlib4 bot (Nov 21 2025 at 10:39):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (48386d45430f2f135ba092501a6af735d13249ee)

github mathlib4 bot (Nov 22 2025 at 09:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3b0d2ce5da2950d08a21a3592ac9bbc9ff321fa5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 23 2025 at 01:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7dafbfd9df6544ec16d3b4b89d83d7b407277dd1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 23 2025 at 05:15):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fea3bb9371118ada7a5d092cff313b759967270d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 23 2025 at 08:46):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (3c22fdd69e9e3071876087356b1c02ef33536666)

github mathlib4 bot (Nov 23 2025 at 11:40):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9de1959db45bf8c6fb680e10bd787adb30aaafc4)

github mathlib4 bot (Nov 24 2025 at 01:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b02313854c5766832e4a4f822f9dddd9d5c96717).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 24 2025 at 04:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (544a5bad21a682c17de0b86fbab5b0a1707c0a71).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 24 2025 at 06:07):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (9de1959db45bf8c6fb680e10bd787adb30aaafc4)

github mathlib4 bot (Nov 24 2025 at 09:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2d938306fbd862792926dd7e6568624c15c4c917).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 24 2025 at 12:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (931804c828b10e45310413ca668de3c50e8ac566).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 24 2025 at 13:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (84ff9d89f3cd7cf6f0ae864a6f44657de94a75fa).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 24 2025 at 14:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f9640c952ebd3a4681e6614b4d7075be6b8979a6).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 24 2025 at 14:18):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f9640c952ebd3a4681e6614b4d7075be6b8979a6)

github mathlib4 bot (Nov 25 2025 at 00:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (93c47f1843e4cabe08e69dbb110b90dcf2cbf6f8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2025 at 04:53):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f9640c952ebd3a4681e6614b4d7075be6b8979a6)

github mathlib4 bot (Nov 25 2025 at 09:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (edae2b4a62f1efe2a65681f1ac1e4c8e7d247a2b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2025 at 10:15):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c6fed8e84516054b1750f5f450a60cf8513e0357).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2025 at 11:37):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d853bf186426b8e7812a8e06a820727257037516).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 25 2025 at 13:20):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (a911b002d50c434ca1a97696822583ba95da6317)

github mathlib4 bot (Nov 26 2025 at 01:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (69f7ed6b55c6bcb154e63991c8b0131b6baf2c99).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 26 2025 at 02:23):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (a911b002d50c434ca1a97696822583ba95da6317)

github mathlib4 bot (Nov 26 2025 at 12:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1ea88e465819146a21bef2d5b75b9f1b1b82ac21).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 27 2025 at 00:49):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9ce81b10927d4c9c4126c6b5c985064f147a6e30).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 27 2025 at 04:14):

@Henrik Böving nightly-testing is failing with "PANIC at Lean.Compiler.LCNF.UnreachableBranches.Value.addChoice" when compiling Cache/Requests.lean.

Kim Morrison (Nov 27 2025 at 04:14):

Presumably this is lean#11362.

Kim Morrison (Nov 27 2025 at 04:46):

minimization at lean#11393

Kim Morrison (Nov 27 2025 at 04:55):

fix, according to Claude, in lean#11394

github mathlib4 bot (Nov 27 2025 at 09:09):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (90249a695a1d6c2f4ff8cde64f5b59f375500d20).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 27 2025 at 10:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a33d629159519ae71dcd3ae2de858d3fb9732def).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 27 2025 at 10:26):

I just merged lean-pr-testing-10204 into aesop's nightly testing, and ran a lake update. There are still String related issues.

github mathlib4 bot (Nov 27 2025 at 10:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d6e7ecf1621aa073a8e3fdc69133961c1a9b1db2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 27 2025 at 10:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ff76558b4c367ef141c92b4d12a8ee18ed563b33).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 27 2025 at 10:40):

Kim Morrison said:

There are still String related issues.

These were from #25945; fixed using .copy.

github mathlib4 bot (Nov 27 2025 at 11:30):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b0a6d9133033e62eb00603b1c4394c181a17a93f).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 27 2025 at 11:33):

The remaining error on nightly-testing is from a genuine grind bug, hopefully fixed soon.

github mathlib4 bot (Nov 27 2025 at 11:34):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e142c62e0208c576a491c84eaefbb353ae3b476e).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 28 2025 at 01:29):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a9faeaabfed78e92b3e47f6c2f2b3995c3a0b0f2).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 28 2025 at 02:59):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4481ab69015a370e3b2f8da6fceb36e47017fd09).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Nov 28 2025 at 03:21):

I've replaced the two places affected by this grind bug with older proofs and adaptation notes, in case the fix isn't merged immediately.

github mathlib4 bot (Nov 28 2025 at 03:45):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (42c6ec6c6d7049b7b774bad2ee7b91c789e01fa8)

github mathlib4 bot (Nov 28 2025 at 18:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (66b533bc65e58d85d4b4d092a4f59c7aa6b4d21b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 29 2025 at 01:51):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b3687cde5b3ccbaf04e5c3b772a97465ff3949b3).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 29 2025 at 09:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9d1030d34c5b7ba7f8bd4c840ed562aa6a07a680).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2025 at 01:43):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ae8e7b63aea6f3181e3a76e98a859aaf27843c3f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2025 at 09:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7d99553a5773d5c6c1775e02033fedb5302a10b1).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2025 at 22:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2f5a01d8dc80c83834d6dfe88a9142a12d3fc638).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Nov 30 2025 at 23:25):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (3fdd607ea6ff78249b607b72aaea2f92c1152f22)

github mathlib4 bot (Dec 01 2025 at 10:38):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (2100ee662d0d4b3233534f70716a04f15f74c300)

github mathlib4 bot (Dec 01 2025 at 23:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (25e595925d652b22eb0343d8ef0a417e4f58a5c5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 02 2025 at 00:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fb74640173cdca998957d776ed55ad3ab7e4fbfb).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 02 2025 at 01:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (871f8b1529fd5062d298a8265545464f2257ca20).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 02 2025 at 04:08):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (2100ee662d0d4b3233534f70716a04f15f74c300)

github mathlib4 bot (Dec 02 2025 at 09:54):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ff1b41e0d1ce681e5abe01e23431a15af5438f44).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Dec 02 2025 at 10:06):

Could we add a liacutsat alias in mathlib master already so we can see what other changes are left on nightly-testing?

github mathlib4 bot (Dec 02 2025 at 23:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (56b89728291f11b1aefc409b501bfdddeb6ed45c).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 02 2025 at 23:56):

PR for the lia alias: https://github.com/leanprover-community/mathlib4/pull/32376

github mathlib4 bot (Dec 03 2025 at 01:38):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (4c7a6b2ec6b6cfebf6521848b0ee53796a2b66dc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 03 2025 at 04:16):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5bfa1623542d7f245e45ac880c26cfe8f9ecc5ea).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 03 2025 at 10:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e8eda6e4e891ac595a125e06f7c8b5f9ad3ec4aa).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Dec 03 2025 at 14:00):

Ruben Van de Velde said:

Could we add a liacutsat alias in mathlib master already so we can see what other changes are left on nightly-testing?

@Kim Morrison thanks - I tried to fix the linter on #32376 but failed

Kim Morrison (Dec 04 2025 at 01:41):

@Ruben Van de Velde, fixed.

github mathlib4 bot (Dec 04 2025 at 01:53):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (453cce856d41bd2715d9055ecdc877015033095f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 04 2025 at 03:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (5d3913854dd814ae3cf295853b4a10ce74116670).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 04 2025 at 04:55):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (47232c86ec8a757736df7a7e225fff8044ec0913)

github mathlib4 bot (Dec 04 2025 at 10:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (42f7d9c707cc83f542a69d046f73c15975ed20ce).
You can git fetch; git checkout nightly-testing and push a fix.

Joachim Breitner (Dec 04 2025 at 13:54):

discover-lean-pr-testing fails in a way I don't quite understand:

=== PRS =========================
11482 11492 11493
=== prs.txt =====================
11482
11492
11493
Error: Process completed with exit code 1.

Joachim Breitner (Dec 04 2025 at 13:55):

Ah, maybe this line fails if there are no adaption branches (and it’s normal for this job to fail if there are none)?

  MATCHING_BRANCHES=$(git branch -r | grep -f prs.txt | grep "lean-pr-testing")

github mathlib4 bot (Dec 04 2025 at 14:00):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (42f7d9c707cc83f542a69d046f73c15975ed20ce)

Joachim Breitner (Dec 04 2025 at 14:09):

Also linting failed, restarting helped. Got a new nightly green.

Snir Broshi (Dec 04 2025 at 16:39):

Now that #32376 was merged, #32431 fixes some remaining cutsats from PRs that were merged at the same time

github mathlib4 bot (Dec 05 2025 at 01:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (96d98dd8f37a7723fdb3f43a766a7fea4580b92b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 05 2025 at 06:00):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (42f7d9c707cc83f542a69d046f73c15975ed20ce)

github mathlib4 bot (Dec 05 2025 at 10:22):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (d8fd1ebe820a2953f0092a2b117aa51d41485b40).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 05 2025 at 12:32):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a3f0e4ffc7efee40e9e57d1386546fe18e35875d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 05 2025 at 14:17):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (ce00192bf8058fc20bcc4188abf983d16be18ff7)

github mathlib4 bot (Dec 06 2025 at 01:35):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (beb1a1dc8899a9b31359eb461c1562bbced8ec2a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 06 2025 at 10:20):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ed79179ced7b9a869b525cf25376327dca0be1c5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 07 2025 at 01:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f7826d333e7f78a0636e6353ac61dd003abeb484).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 07 2025 at 05:55):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ab1ad83e8ee1e858dca5e2c1e1cffb36d92aa040).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 07 2025 at 08:28):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (c1ec86eaa7fbd85b4e11dd5c5b5816d5546260ca).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 07 2025 at 09:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (dce50d07797e5ed4369a947398963ad807da23c9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 07 2025 at 12:07):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (f83e6b62b6c1afa0e93948e950888d1b7ebdbfc0)

github mathlib4 bot (Dec 08 2025 at 09:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (875db3289c0d5bce55398f7c43f22a6019acf4ae).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 08 2025 at 12:13):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (64d8fd34de4621adbe3924fd081a8f6a92d55872)

github mathlib4 bot (Dec 09 2025 at 02:01):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7ce3f2693854a9dfacf1633fbc1ab62fc2b9a5cc).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 09 2025 at 02:47):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0ba3b8828a1255591cea7a27953334c213ccd029).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 09 2025 at 03:24):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (64d8fd34de4621adbe3924fd081a8f6a92d55872)

github mathlib4 bot (Dec 09 2025 at 10:24):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (bbf1f53abe6a2fbb5d33d72a5ef0bec27e493ec5)

github mathlib4 bot (Dec 10 2025 at 10:10):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (25918fa625b53957490426f591c8f7efe477fe0d)

github mathlib4 bot (Dec 11 2025 at 00:18):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (db12a4c2bbab3230732b747eea73e8c013808a1c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 11 2025 at 02:28):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (25918fa625b53957490426f591c8f7efe477fe0d)

github mathlib4 bot (Dec 11 2025 at 09:39):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (fbd0d7cf2576c1ff2c5adccc870274c407a1d25d).
You can git fetch; git checkout nightly-testing and push a fix.

Joachim Breitner (Dec 11 2025 at 10:14):

I’m a bit confused by the github display here:
foo.png
This looks as if Ci tested chore: bump to nightly-2025-12-11, but not the latest commit (merge lean-pr-testing-11581), but the Zulip bot above reports that the latter has built.

I would guess that because the merge commits are pushed by github-actions and not the bot, i.e. with the wrong token, Github’s annoying “actions by default don't trigger actions” that the github view is correct, that the zulib bot above is confused by the branch being more advanced than the latest CI, and that we are missing out on automatic ✓ when the adaption branches indeed fix the build.

Also note that the link to the log above shows that indeed 35fa128 was checked.

I’ll push an empty commit to confirm.

But I suggest someone changes the action that merges the commits to use the leanprover-community-mathlib4-bot token.

github mathlib4 bot (Dec 11 2025 at 10:19):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ee135c102280f715868fadc59c1b69b81bcf3f4a).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 11 2025 at 10:30):

Joachim Breitner said:

But I suggest someone changes the action that merges the commits to use the leanprover-community-mathlib4-bot token.

fix(ci): use bot token for discover-lean-pr-testing merges #32722

github mathlib4 bot (Dec 11 2025 at 10:36):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9aedaa26604a3d4fa47d81b99674a3bbece38e63).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 11 2025 at 11:06):

Uh oh:

error: Mathlib/Data/Prod/PProd.lean:24:4: code generator failed, unsupported occurrence of `Prod.noConfusion`
error: Mathlib/Data/Prod/Basic.lean:28:4: code generator failed, unsupported occurrence of `Prod.noConfusion`

@Henrik Böving? @Joachim Breitner?

Joachim Breitner (Dec 11 2025 at 11:06):

:raised_hand:

Kim Morrison (Dec 11 2025 at 11:07):

I guess it is easy to replace these with other proofs.

Kim Morrison (Dec 11 2025 at 11:07):

I've pushed other proofs and will let you clean up whenever you like. :-)

github mathlib4 bot (Dec 11 2025 at 11:07):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (517d0ec2ffc055c5391888176a23862ec3e3acd5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 11 2025 at 11:16):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (517d0ec2ffc055c5391888176a23862ec3e3acd5).
You can git fetch; git checkout nightly-testing and push a fix.

Joachim Breitner (Dec 11 2025 at 11:30):

Fix incoming https://github.com/leanprover/lean4/pull/11611. Sorry for that.

Kim Morrison (Dec 11 2025 at 11:47):

The next failures are some genuine grind failures. We pushed a lot of changes today...

Kim Morrison (Dec 11 2025 at 12:21):

I got it down to:

module

public import Mathlib.Data.Int.Order.Basic
public import Mathlib.Order.Max
public import Mathlib.Order.Defs.LinearOrder

section Mathlib.Order.Lattice

variable {α : Type}

class Max' (α : Type) where
  max' : α  α  α

instance Max'.toMax [Max' α] : Max α where max a b := Max'.max' a b

instance LinearOrder.toMax' {α : Type} [LinearOrder α] : Max' α where
  max' := max

end Mathlib.Order.Lattice

section Mathlib.Algebra.Order.Group.Unbundled.Abs

variable {α : Type} [Max' α] [Neg α] {a b : α}

@[grind]
def abs (a : α) : α := a  (-a)

end Mathlib.Algebra.Order.Group.Unbundled.Abs

theorem abs_lt_one_iff {a : Int} : abs a < 1  a = 0 := by
  grind

(succeeding on nightly-2025-12-10, failing on nightly-2025-12-11) but will stop for the day.

Kim Morrison (Dec 11 2025 at 21:17):

Reduced to

section Mathlib.Order.Defs.LinearOrder

class LinearOrder (α : Type) extends Max α where

end Mathlib.Order.Defs.LinearOrder
section Mathlib.Data.Int.Order.Basic

instance instLinearOrder : LinearOrder Int where

end Mathlib.Data.Int.Order.Basic
section Mathlib.Order.Lattice

variable {α : Type}

class SemilatticeSup (α : Type) where
  sup : α  α  α

instance SemilatticeSup.toMax [SemilatticeSup α] : Max α where max a b := SemilatticeSup.sup a b

instance LinearOrder.toSemilatticeSup {α : Type} [LinearOrder α] : SemilatticeSup α where
  sup := max

end Mathlib.Order.Lattice

section Mathlib.Algebra.Order.Group.Unbundled.Abs

variable {α : Type} [SemilatticeSup α] [Neg α] {a b : α}

@[grind]
def abs (a : α) : α := max a (-a)

end Mathlib.Algebra.Order.Group.Unbundled.Abs

theorem abs_lt_one_iff {a : Int} : abs a < 1  a = 0 := by
  grind

and bisected to lean#11589.

github mathlib4 bot (Dec 12 2025 at 01:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0e01e942cf77712b3c312afb0bace9fd6fc540a9).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 12 2025 at 09:25):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (862da6f4ec8569f61d65279d000ab78ca31f1ac8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 12 2025 at 11:41):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b9d27c2d42295ec61e4be7802b374f87753b7cac).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 12 2025 at 12:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (3dc6a531c3723314cda883d11f4afdf60bc58572).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 12 2025 at 12:27):

Haven't fixed the grind regression yet (we fixed one bug, which turned out to be the wrong one), so this will stay broken until (at least) tomorrow.

github mathlib4 bot (Dec 12 2025 at 23:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a43628d6c273c8ef36a2fbc507a41ddbec24c66d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 12 2025 at 23:21):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (af72668a6e4c1fe0541fe2fc40255351d574ca05).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2025 at 00:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (b62a16dd533561fd54375ccb4570e56df88a2063).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2025 at 02:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (65965e968a552e0397c473fc397ac985d5fcc611).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2025 at 02:48):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (653a7b8342044641e50988e16e6e3c7e52c5af8c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2025 at 03:04):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (9b2a09389fcaff1701eed8b6196c9f1402729281).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2025 at 08:58):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2cb7523e305189ee487633caf9ce641f4d1a41ce).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 13 2025 at 10:11):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (f2e157ed3776e5bead67b2769748376f7d60ec1d).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 13 2025 at 10:49):

Hopefully coming good shortly.

github mathlib4 bot (Dec 13 2025 at 11:31):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (a3185bbe22a659e2146e3dc2eab9012f017f4296).
You can git fetch; git checkout nightly-testing and push a fix.

Ruben Van de Velde (Dec 13 2025 at 11:52):

inductive WalkingParallelFamily (J : Type w) : Type w
  | zero : WalkingParallelFamily J
  | one : WalkingParallelFamily J
deriving DecidableEq, Inhabited

fails linting with

/- The `unusedArguments` linter reports:
UNUSED ARGUMENTS. -/
#check @instDecidableEqWalkingParallelFamily.decEq /- argument 2 inst✝ : DecidableEq J✝ -/

Not sure how to deal with that

Joachim Breitner (Dec 13 2025 at 12:02):

See https://github.com/leanprover/lean4/issues/10295. I think these linter errors are allowlisted somewhere in mathlib?

But in this case maybe it was a mistake of mine to use a derived instance, and it’s better to undo
https://github.com/leanprover-community/mathlib4-nightly-testing/commit/f7f11d8000777cacc0ab6c3fdf537dbf5d092bff
and fix the manual instance, and leave a comment that we do not derive DecidableEq becaues it creates instances with too strong assumptions.

github mathlib4 bot (Dec 13 2025 at 12:02):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (72824e46f06f07252964971a2833a0a7e299a29b).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2025 at 01:44):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (e0e4b3764f55ff95f4c6fb9dc2178cb528baafa3).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 14 2025 at 04:55):

Joachim Breitner said:

fix the manual instance, and leave a comment

Done.

github mathlib4 bot (Dec 14 2025 at 05:12):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (ed6eb20497a07651453c0c122f58489107d3bb59).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2025 at 06:31):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (1daec5fd00842e0d97350dd435e75d6da14b68ed)

github mathlib4 bot (Dec 14 2025 at 06:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (95c333015a7ad1963482857ec4c50ec75076705a).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2025 at 09:10):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (92fe33c6853e83627488dc3feaaf98c7317f2183).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2025 at 11:17):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (376a0299823863afc2717dec66e0bf567acdae92)

github mathlib4 bot (Dec 14 2025 at 11:26):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (81be7f1d1cbcc4cd2fd714acc75d5a633556a73f).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 14 2025 at 13:03):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (376a0299823863afc2717dec66e0bf567acdae92)

github mathlib4 bot (Dec 15 2025 at 10:16):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (4d6a1d528583db055842b31879e9432fd9abb02e)

github mathlib4 bot (Dec 16 2025 at 09:00):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (7e787c6da65569af6d091fa09541d317a67b9de7).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 16 2025 at 14:14):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (85312f95a468765a9463fd6596eb6db473496cc8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 16 2025 at 15:23):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (70f9a3a36a25259d0a21a8f6d307b74ed58505e7).
You can git fetch; git checkout nightly-testing and push a fix.

Joachim Breitner (Dec 16 2025 at 16:22):

It seems that the cache doesn’t work reliably on nightly-testing? Locally I got a cache before pushing, and the push only affects tests, but then
https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/20274023177/job/58217429000
rebuilds all of mathlib. Not sure why.

github mathlib4 bot (Dec 16 2025 at 17:11):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (6aa41bc08a8e0425cdced8d1a00189842e517f12)

Bryan Gin-ge Chen (Dec 16 2025 at 17:45):

Joachim Breitner said:

It seems that the cache doesn’t work reliably on nightly-testing? Locally I got a cache before pushing, and the push only affects tests, but then
https://github.com/leanprover-community/mathlib4-nightly-testing/actions/runs/20274023177/job/58217429000
rebuilds all of mathlib. Not sure why.

This is just free association on my part, but is this something that the suggestion at #mathlib4 > Mathlib has moved to the new module system @ 💬 would help with?

Joachim Breitner (Dec 16 2025 at 21:29):

It happend today again that I fixed nightly-testing of mathlib (incuding fixing the batteries build), and nightly-with-mathlib on lean4 advanced, but because I didn’t fix the batteries test suite, which I don’t see when fixing mathlib, there is no batteries nightly tag, and so my PR was still not tested against mathlib, saying

  • :exclamation: Batteries CI can not be attempted yet, as the nightly-testing-2025-12-16 tag does not exist there yet. We will retry when you push more commits. If you rebase your branch onto nightly-with-mathlib, Batteries CI should run now. You can force Mathlib CI using the force-mathlib-ci label. (2025-12-16 10:51:40)

which is not correct (rebasing on nightly-with-mathlib won’ help).

Maybe we should just remove the check whether the batteries tag exists, and run mathlib CI when mathlib is ready?

github mathlib4 bot (Dec 16 2025 at 22:46):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (62e8a6b26b8a6cc309e59e1d9e0d6e25ff121764).
You can git fetch; git checkout nightly-testing and push a fix.

Kim Morrison (Dec 17 2025 at 00:04):

lean#11707 removes the batteries tag check.

github mathlib4 bot (Dec 17 2025 at 01:42):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (1d00b4d59cb464d6d4bcb213b54f4328b743a32d).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 17 2025 at 05:38):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (6aa41bc08a8e0425cdced8d1a00189842e517f12)

github mathlib4 bot (Dec 17 2025 at 10:11):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (178f5fddb4143ecaf7f73e9ec8ef61518323f4a1)

github mathlib4 bot (Dec 18 2025 at 09:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (59c8a61b74fdf8a22a2793cd0a2b719d4d1c20c8).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 18 2025 at 11:17):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (6099272a2a2c4b64c95bf4a53381bd669657b3c5).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 19 2025 at 02:04):

:check: The latest CI for Mathlib's nightly-testing branch has succeeded! (ce5a8af5c1e7ea16ee814574e46e34800897c180)

github mathlib4 bot (Dec 19 2025 at 08:56):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (0ffec2a1beb309de71139284a573b1a379a1be94).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2025 at 01:50):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (2eb6d9e4a3b89acd9b81c67012c8b4ef27b55d4c).
You can git fetch; git checkout nightly-testing and push a fix.

github mathlib4 bot (Dec 20 2025 at 03:45):

:cross_mark: The latest CI for Mathlib's nightly-testing branch has failed (34f9d35c1e2d6467d3ecc1f42722a762a912fb67).
You can git fetch; git checkout nightly-testing and push a fix.


Last updated: Dec 20 2025 at 21:32 UTC