Zulip Chat Archive

Stream: mathlib4

Topic: recall doesn't work in namespaces


Mario Carneiro (Apr 02 2024 at 21:29):

MWE:

import Mathlib.Tactic.Recall

namespace Foo
noncomputable def foo := 0
recall Foo.foo : String := ""

Mario Carneiro (Apr 02 2024 at 21:30):

this is doubly weird:

  • You can't use recall foo, you have to write recall Foo.foo even though you are already in the namespace
  • The definition does not seem to be checked against the original in any way

Mario Carneiro (Apr 02 2024 at 21:34):

Also recall doesn't take a doc string. I would like to use it to gloss the declaration, it doesn't have to be stored or validated against the original

Damiano Testa (Apr 02 2024 at 22:00):

There was also this previous thread about it: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/.60recall.60.20strangeness

Mario Carneiro (Apr 02 2024 at 22:23):

oh look at that, past me already filed a bugfix PR

Mario Carneiro (Apr 02 2024 at 22:24):

seems to be failing though


Last updated: May 02 2025 at 03:31 UTC