aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ZRange/Show.v
blob: 2fac57b16dddfd33337e4df504de7a17bbd44345 (plain)
1
2
3
4
5
6
7
8
Require Import Coq.Strings.String.
Require Import Crypto.Util.Strings.Show.
Require Import Crypto.Util.ZRange.
Local Open Scope string_scope.

Global Instance show_zrange : Show zrange
  := fun _ r
     => "[" ++ Hex.show_Z false (lower r) ++ " ~> " ++ Hex.show_Z false (upper r) ++ "]".