https://gitlab.com/nomadic-labs/mi-cho-coq
Raw File
Tip revision: e8f74dfd815040efcf6d88ce32a1f14ab9f83263 authored by Colin González on 05 March 2021, 14:06:39 UTC
Proof for updateTokenPool
Tip revision: e8f74df
micheline_syntax.v
Require Import String ZArith.
Require Import location.

Inductive annotation := Mk_annot : location * location * string -> annotation.

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