aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ZUtil/Notations.v
blob: 9a07435243106ce4acaa4f2ee14c19cf8e24f5d9 (plain)
1
2
3
4
5
6
Require Import Coq.ZArith.BinInt.
Require Import Crypto.Util.Notations.

Infix ">>" := Z.shiftr : Z_scope.
Infix "<<" := Z.shiftl : Z_scope.
Infix "&'" := Z.land : Z_scope.