Module ForeignTypeToJSON


Require Import List String.

Require Import Utils ForeignType.

Local Open Scope string_scope.

Section ForeignTypeToJSON.


Class foreign_type_to_JSON {ftype:foreign_type}: Type
  := mk_foreign_type_to_JSON {
         foreign_to_string_to_type
           (s:string) : option foreign_type_type
         ; foreign_to_string_from_type
             (fd:foreign_type_type) : string
       }.

End ForeignTypeToJSON.