mirror of
https://github.com/msgpack/msgpack-c.git
synced 2025-03-20 13:33:51 +01:00
4 lines
171 B
Coq
4 lines
171 B
Coq
![]() |
Require Import ExtrOcamlBasic ExtrOcamlIntConv ExtrOcamlNatInt.
|
||
|
Require Import SerializeImplement DeserializeImplement.
|
||
|
Extraction "msgpackCore.ml" serialize deserialize.
|