aboutsummaryrefslogtreecommitdiff
path: root/src/BaseSystem.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jagro@google.com>2016-06-22 13:34:00 -0700
committerGravatar Jason Gross <jagro@google.com>2016-06-22 13:34:00 -0700
commit18b79f83ce6c947eaa49baf586cc475d50e3d9ca (patch)
treedc20511c7507aec0dc8656d30f9388d906ab664b /src/BaseSystem.v
parentacd8d172e3112372be930544af57c36bf085e6c2 (diff)
Aggregate all level specifications not in Spec/*
This prevents notation conflicts (see comment in Notations.v for more explanation).
Diffstat (limited to 'src/BaseSystem.v')
-rw-r--r--src/BaseSystem.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/src/BaseSystem.v b/src/BaseSystem.v
index c07aad759..1985520f0 100644
--- a/src/BaseSystem.v
+++ b/src/BaseSystem.v
@@ -2,6 +2,7 @@ Require Import Coq.Lists.List.
Require Import Coq.ZArith.ZArith Coq.ZArith.Zdiv.
Require Import Coq.omega.Omega Coq.Numbers.Natural.Peano.NPeano Coq.Arith.Arith.
Require Import Crypto.Util.ListUtil Crypto.Util.CaseUtil Crypto.Util.ZUtil.
+Require Import Crypto.Util.Notations.
Import Nat.
Local Open Scope Z.
@@ -47,7 +48,7 @@ Section BaseSystem.
| _, nil => us
| _, _ => vs
end.
- Infix ".+" := add (at level 50).
+ Infix ".+" := add.
Hint Extern 1 (@eq Z _ _) => ring.