playground/coq/unfinished/notation-scope.v

11 lines
203 B
Coq

Require Import List.
Import ListNotations.
Module EgNotations.
Declare Scope eg_scope.
Delimit Scope eg_scope with eg.
Print Visibility.
Notation "[ ]" := 3
(at level 30) : eg_scope.
End EgNotations.