aboutsummaryrefslogtreecommitdiff
path: root/src/Util/StringMap.v
blob: 8b45d81d4f55ee084895adf3e7a0e1133590aba2 (plain)
1
2
3
4
5
6
7
Require Import Coq.FSets.FMapInterface.
Require Import Coq.FSets.FMapList.
Require Import Coq.Structures.OrderedType.
Require Import Coq.Strings.String.
Require Import Crypto.Util.Strings.String_as_OT.

Module StringMap := FMapList.Make String_as_OT.