aboutsummaryrefslogtreecommitdiff
path: root/test-suite/interactive
diff options
context:
space:
mode:
authorPierre Roux2020-09-09 23:33:05 +0200
committerPierre Roux2020-09-11 22:23:24 +0200
commit6551f14196784e323688e682877229bc7f901659 (patch)
tree18fd2fd9da90095327498f0de309beb6d409c77a /test-suite/interactive
parentd5eb564a1ae46409e90a2c6bd6af5b77aa37773e (diff)
Rename Numeral Notation command to Number Notation
Keep Numeral Notation wit a deprecation warning.
Diffstat (limited to 'test-suite/interactive')
-rw-r--r--test-suite/interactive/PrimNotation.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/test-suite/interactive/PrimNotation.v b/test-suite/interactive/PrimNotation.v
index 07986b0df3..55116dc78b 100644
--- a/test-suite/interactive/PrimNotation.v
+++ b/test-suite/interactive/PrimNotation.v
@@ -21,7 +21,7 @@ Local Set Universe Polymorphism.
Delimit Scope punit_scope with punit.
Delimit Scope pcunit_scope with pcunit.
Delimit Scope int_scope with int.
-Numeral Notation Decimal.int Decimal.int_of_int Decimal.int_of_int : int_scope.
+Number Notation Decimal.int Decimal.int_of_int Decimal.int_of_int : int_scope.
Module A.
NonCumulative Inductive punit@{u} : Type@{u} := ptt.
Cumulative Inductive pcunit@{u} : Type@{u} := pctt.
@@ -31,10 +31,10 @@ Module A.
:= fun v => match v with 0%int => Some pctt | _ => None end.
Definition of_punit : punit -> Decimal.uint := fun _ => Nat.to_uint 0.
Definition of_pcunit : pcunit -> Decimal.uint := fun _ => Nat.to_uint 0.
- Numeral Notation punit to_punit of_punit : punit_scope.
+ Number Notation punit to_punit of_punit : punit_scope.
Check let v := 0%punit in v : punit.
Back 2.
- Numeral Notation pcunit to_pcunit of_pcunit : punit_scope.
+ Number Notation pcunit to_pcunit of_pcunit : punit_scope.
Check let v := 0%punit in v : pcunit.
End A.
Reset A.
@@ -44,7 +44,7 @@ Module A.
Definition to_punit : Decimal.int -> option punit
:= fun v => match v with 0%int => Some ptt | _ => None end.
Definition of_punit : punit -> Decimal.uint := fun _ => Nat.to_uint 0.
- Numeral Notation punit to_punit of_punit : punit_scope.
+ Number Notation punit to_punit of_punit : punit_scope.
Check let v := 0%punit in v : punit.
End A.
Local Set Universe Polymorphism.
@@ -52,7 +52,7 @@ Inductive punit@{u} : Type@{u} := ptt.
Definition to_punit : Decimal.int -> option punit
:= fun v => match v with 0%int => Some ptt | _ => None end.
Definition of_punit : punit -> Decimal.uint := fun _ => Nat.to_uint 0.
-Numeral Notation punit to_punit of_punit : punit_scope.
+Number Notation punit to_punit of_punit : punit_scope.
Check let v := 0%punit in v : punit.
Back 6. (* check backtracking of registering universe polymorphic constants *)
Local Unset Universe Polymorphism.
@@ -60,5 +60,5 @@ Inductive punit : Set := ptt.
Definition to_punit : Decimal.int -> option punit
:= fun v => match v with 0%int => Some ptt | _ => None end.
Definition of_punit : punit -> Decimal.uint := fun _ => Nat.to_uint 0.
-Numeral Notation punit to_punit of_punit : punit_scope.
+Number Notation punit to_punit of_punit : punit_scope.
Check let v := 0%punit in v : punit.