aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_3483.v
blob: 970363f00adc635ba839e3b1b5cdbea8b99f4eb5 (plain)
1
2
3
4
(* Check proper failing when using notation of non-constructors in
   pattern-bmatching *)

Fail Definition nonsense ( x : False ) := match x with y + 2 => 0 end.