Module Qcert.Utils.Var
Require
Import
String
.
Section
Var
.
Variables are defined as strings
Definition
var
:=
string
.
End
Var
.