Coq is a formal proof management system. It provides a formal language to write mathematical definitions, executable algorithms and theorems together with an environment for semi-interactive development of machine-checked proofs.
Inductive t : Set := C : t -> t -> t.
Reserved Notation "a $ b" (at level 200, right associativity).
Infix "$" := C.
Variables (a b : t).
Check (a $ b).
(* Error: Syntax error: ',' or ')' expected after [term level 200] (in [term]). *)
Description of the problem
Other levels don't seem to have this problem.
Coq Version
master
cc. @Alizter