aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_9166.v
blob: cd594c660fb8dfce67addba1a00cca0fd59aa22e (plain)
1
2
3
4
5
6
7
8
9
10
Set Warnings "+deprecated".

#[deprecated(since = "X", note = "Y")]
Notation bar := option.

Definition foo (x: nat) : nat :=
  match x with
  | 0 => 0
  | S bar => bar
  end.