aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_11816.v
blob: 82a317b2504efb39d7b81ac4baf3d7f9c69e3288 (plain)
1
2
(* This should be an error, not an anomaly *)
Fail Definition foo := fix foo (n : nat) { wf n n } := 0.