From 18b79f83ce6c947eaa49baf586cc475d50e3d9ca Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Wed, 22 Jun 2016 13:34:00 -0700 Subject: Aggregate all level specifications not in Spec/* This prevents notation conflicts (see comment in Notations.v for more explanation). --- src/BaseSystemProofs.v | 3 ++- 1 file changed, 2 insertions(+), 1 deletion(-) (limited to 'src/BaseSystemProofs.v') diff --git a/src/BaseSystemProofs.v b/src/BaseSystemProofs.v index 4414877b4..85835aabe 100644 --- a/src/BaseSystemProofs.v +++ b/src/BaseSystemProofs.v @@ -3,9 +3,10 @@ Require Import Util.ListUtil Util.CaseUtil Util.ZUtil. Require Import ZArith.ZArith ZArith.Zdiv. Require Import Omega NPeano Arith. Require Import Crypto.BaseSystem. +Require Import Crypto.Util.Notations. Local Open Scope Z. -Local Infix ".+" := add (at level 50). +Local Infix ".+" := add. Local Hint Extern 1 (@eq Z _ _) => ring. -- cgit v1.2.3