Zulip Chat Archive

Stream: mathlib4

Topic: A specific file triggers rpc errors


Joël Riou (Oct 31 2023 at 16:21):

When I open the file Mathlib.CategoryTheory.Abelian.Refinements (current mathlib master branch) in VSCode, it becomes very unstable: when I try to see the details of a proof, the infoview would always show "Error updating: Error fetching goals: Rpc error: InternalError: parenthesize: uncaught backtrack exception. ". Does anyone see the same problem when opening this file? If this is reproducible, would anyone know how to fix the bug?

Matthew Ballard (Oct 31 2023 at 16:26):

Odd behavior on nvim also. I am missing the state on some (most) proof lines. The exception seems to be goals accomplished messages.

Matthew Ballard (Oct 31 2023 at 16:33):

Apparently {S₁ S₂ : ShortComplex C} are not used?

Matthew Ballard (Oct 31 2023 at 16:36):

Here is something I have not seen yet [error when printing message: parenthesize: uncaught backtrack exception]

Matthew Ballard (Oct 31 2023 at 16:57):

Here is a statement with the error:

lemma epi_iff_surjective_up_to_refinements (f : X  Y) (A : C) (y : A   Y):
       (A' : C) (π : A'   A) (h : Epi π) (x : A'   X), True := by --π ≫ y = x ≫ f := by

Matthew Ballard (Oct 31 2023 at 16:57):

It goes away if you remove Mathlib.Algebra.Homology.ShortComplex.Exact from the imports

Joël Riou (Oct 31 2023 at 17:20):

Thanks. A more minimal example is as follows:

import Mathlib.CategoryTheory.EpiMono
import Mathlib.Util.Delaborators

open CategoryTheory

variable {C : Type*} [Category C] {A X Y : C} (f : X  Y) (y : A  Y)

lemma test1 :  (A' : C) (π : A'  A) (x : A'  X), π  y = x  f := by
  sorry

lemma test2 :  (A' : C) (π : A'  A) (_ : Epi π) (x : A'  X), π  y = x  f := by
  sorry /- Error updating: Error fetching goals: Rpc error:
    InternalError: parenthesize: uncaught backtrack exception.-/

Removing the import to Mathlib.Util.Delaborators makes test2 work.

Matthew Ballard (Oct 31 2023 at 17:21):

You beat me :)

Mauricio Collares (Oct 31 2023 at 17:34):

The same issue (I think) is being discussed in https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/doc-gen4.20missing.20declaration

Kyle Miller (Oct 31 2023 at 17:51):

Minimaler example:

import Mathlib.Util.Delaborators

theorem test1 :  (_ : True), True := by
  sorry

theorem test2 :  (_ : True) (x : Nat), True := by
  sorry /- Error updating: Error fetching goals: Rpc error:
    InternalError: parenthesize: uncaught backtrack exception.-/

Kyle Miller (Oct 31 2023 at 18:19):

#8070 fixes Joël's example

Patrick Massot (Oct 31 2023 at 18:25):

Did you also try with exists_ne_mem_inter_of_not_pairwise_disjoint?

Matthew Ballard (Oct 31 2023 at 18:30):

It does.


Last updated: Dec 20 2023 at 11:08 UTC