https://gitlab.com/nomadic-labs/mi-cho-coq
Raw File
Tip revision: 10d93ac9f34335b1ebe8b7ee15b4281ddb9e4a7a authored by Arvid Jakobsson on 02 February 2021, 18:38:48 UTC
tmp: remove dexter to make pipeline leaner
Tip revision: 10d93ac
contract_components.v
Require Import String ZArith.
Require Import syntax macros semantics comparable util.
Import error.
Require tez.
Require map.


Module Contract_components (C : ContractContext).

Module semantics := Semantics C. Import semantics.



End Contract_components.
back to top