Zulip Chat Archive

Stream: mathlib4

Topic: Removing notation for `Function.combine`


Moritz Doll (Mar 14 2023 at 12:36):

In !4#2869 the notation for the segment clashes with the notation for Function.combine. According to the VSCode search for -[ the notation for Function.combine is never used. Is there anyone opposed to removing it?

Moritz Doll (Mar 14 2023 at 12:45):

mnwe:

import Mathlib.Init.Function

def foo (a b c : Type _) : Type := sorry

notation "[" a "-[" c "]" b "]" => foo a b c

theorem foo_blubb : [a -[c] b] = foo a b c := sorry

Eric Wieser (Mar 14 2023 at 12:50):

In Lean 3 the notation was

notation f ` -[` op `]- ` g  := combine f op g

Is it the same in Lean 4 for docs4#Function.combine ?

Moritz Doll (Mar 14 2023 at 12:50):

yes, this is the notation that causes the above code to fail

Moritz Doll (Mar 14 2023 at 12:51):

it is defined in Mathlib.Init.Function


Last updated: Dec 20 2023 at 11:08 UTC