blob: a9e2c59ab0f7b27eb25d85aa07996da1a1a34c02 (
plain)
1
2
3
4
5
6
7
8
9
|
(* Check that "where" clause behaves as if given independently of the *)
(* definition (variant of bug #113? submitted by Assia Mahboubi) *)
Fixpoint plus1 (n m:nat) {struct n} : nat :=
match n with
| O => m
| S p => S (p+m)
end
where "n + m" := (plus1 n m) : nat_scope.
|