Zulip Chat Archive
Stream: mathlib4
Topic: alias is noncomputable
Mario Carneiro (Mar 29 2023 at 09:40):
MWE?
Eric Wieser (Mar 29 2023 at 09:42):
import Mathlib.Tactic.Alias
def foo : ℕ → ℕ := id
alias foo ← bar
-- failed to compile definition, consider marking it as 'noncomputable' because it depends on 'bar', and it does not have executable code
def baz (n : ℕ) := bar n
Notification Bot (Mar 29 2023 at 10:25):
2 messages were moved here from #mathlib4 > !4#3169 by Eric Wieser.
Alex J. Best (Apr 28 2023 at 20:54):
I made !4#3719 for this
Last updated: Dec 20 2023 at 11:08 UTC