https://gitlab.com/nomadic-labs/mi-cho-coq
Raw File
Tip revision: 6e53f26d9a0f048c38e674ded201a5890efe67dc authored by Raphaƫl Cauderlier on 19 September 2020, 19:17:41 UTC
Adapt to Bruno's template
Tip revision: 6e53f26
micheline_syntax.v
Require Import String ZArith.
Require Import location.

Inductive micheline : Set :=
| SEQ (_ : list loc_micheline)
| PRIM (_ : location * location * string)
       (_ : list loc_micheline)
| STR (_ : string)
| BYTES (_ : string)
| NUMBER (_ : Z)
with
loc_micheline : Set :=
| Mk_loc_micheline : location * location * micheline -> loc_micheline.

back to top