aboutsummaryrefslogtreecommitdiff
path: root/test-suite/success/NumberNotationsNoLocal.v
blob: e19d06cfa7017496e2feb5cb6b382933ca8521b8 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
(* Test that number notations don't work on proof-local variables, especially not ones containing evars *)
Inductive unit11 := tt11.
Declare Scope unit11_scope.
Delimit Scope unit11_scope with unit11.
Goal True.
  evar (to_uint : unit11 -> Decimal.uint).
  evar (of_uint : Decimal.uint -> unit11).
  Fail Number Notation unit11 of_uint to_uint : uint11_scope.
  exact I.
  Unshelve.
  all: solve [ constructor ].
Qed.