aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Strings/Ascii.v
blob: 93ea9b749df6e1003e9ec1d8bddc6248e7d20738 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
Require Import Crypto.Util.Strings.Equality.
Require Import Coq.Strings.Ascii.

Local Open Scope char_scope.

(** Special characters *)

Example Null := "000".
Example Backspace := "008".
Example Tab := "009".
Example LF := "010".
Example NewPage := "012".
Example CR := "013".
Example Escape := "027".
Example NewLine := "010".