Zulip Chat Archive
Stream: mathlib4
Topic: Deprecated & namespace
Andrew Yang (Jul 02 2024 at 23:00):
In the following example, lean marks foo
deprecated despite it is using the non-deprecated Foo.foo
.
theorem Foo.foo : True := trivial
@[deprecated] def Bar.foo : Nat := 3
open Foo Bar
example : True := foo
Damiano Testa (Jul 03 2024 at 00:46):
Is https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/Misfiring.20deprecation related?
Kim Morrison (Jul 03 2024 at 00:57):
Related to, but not exactly, lean#2132.
Would you mind opening an issue? (Perhaps link to lean#2132 in it.)
Andrew Yang (Jul 03 2024 at 02:10):
Ah didn't see that stream when searching. I opened #4636.
Damiano Testa (Jul 03 2024 at 03:46):
Last updated: May 02 2025 at 03:31 UTC