Zulip Chat Archive
Stream: mathlib4
Topic: request for help with failure in Archive
Scott Morrison (Nov 01 2023 at 03:19):
lean4#2790 changes the way some "internal" errors are handled, and it particular makes it "harder to catch" them, so when they occur they will break whatever is going on.
#8056 is the Mathlib adaptation PR.
There are currently several failures of simp
or norm_num
, all occurring in Archive/
, where previously a "max recursion depth" error was being caught, and then the recovery path successfully finished the proof, but now the max recursion depth error is causing a crash.
If anyone is able to look at these, that would be very helpful! A first step might just be to identify where the error is coming from, and/or who used to catch it!
Eric Wieser (Nov 01 2023 at 08:39):
Does locally increasing the depth help?
Mauricio Collares (Nov 01 2023 at 08:49):
Not super helpful but: similar to the failure Leo fixed in Lean's testsuite as part of lean4#2790, this seems to be related to simp calling decide (in this case, norm_num is calling simp). I haven't actually checked it but I'm saying this because in #7834 I had to change the same line that's failing tests in Imo1960Q2.lean.
Scott Morrison (Nov 01 2023 at 11:08):
Eric Wieser said:
Does locally increasing the depth help?
Ah, should have said this: no, increasing the depth only makes it slower, it still fails.
David Renshaw (Nov 01 2023 at 17:52):
I pushed an ugly workaround for Imo1962Q1: https://github.com/leanprover-community/mathlib4/pull/8056/commits/e2c18145218773d1dd36a85d1ef3c0ccfc8c437a
David Renshaw (Nov 01 2023 at 17:53):
(and opened some related discussion: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/whnf.20blowup.20in.20Nat.2Edigits/near/399757322 )
Patrick Massot (Nov 02 2023 at 01:52):
Note that Archive/Imo/Imo1960Q1
is still failing.
David Renshaw (Nov 02 2023 at 15:00):
"fixed" Imo1960Q1 with the same idea here: https://github.com/leanprover-community/mathlib4/pull/8056/commits/f95d8117507cc9401a046ffd9d49764e2373cd18
David Renshaw (Nov 02 2023 at 15:00):
This actually makes the proof go much faster than it currently does on master
David Renshaw (Nov 02 2023 at 16:16):
workaround for BirthdayProblem: https://github.com/leanprover-community/mathlib4/pull/8056/commits/0010b07b87adb9fa5d065e6c1a2b5898729907bf
Last updated: Dec 20 2023 at 11:08 UTC