aboutsummaryrefslogtreecommitdiff
path: root/test-suite/output/bug_9180.v
blob: f221a94a501c14b7915e090516831a5a5e0c06fc (plain)
1
2
3
4
5
6
7
8
9
10
11
Notation succn := (Datatypes.S).

Notation "n .+1" := (succn n) (at level 2, left associativity,
  format "n .+1") : nat_scope.

Locate ".+1".
(* Notation *)
(* "n .+1" := S n : nat_scope (default interpretation) *)
(** so Coq does not apply succn notation *)

Check forall x : nat, x.+1 = x.+1.