aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Scopes.v
blob: 997fedd38ffb19426e961d924732e411a41e14e6 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
(* Check exportation of Argument Scopes even without import of modules *)

Require Import ZArith.

Module A.
Definition opp := Z.opp.
End A.
Check (A.opp 3).

(* Test extra scopes to be used in the presence of coercions *)

Record B := { f :> Z -> Z }.
Variable a:B.
Arguments Scope a [Z_scope].
Check a 0.