https://gitlab.com/nomadic-labs/mi-cho-coq
Revision d116674d67eca4b4b15d7c08efd878a8c8aa864b authored by kristinas on 11 May 2021, 09:41:59 UTC, committed by kristinas on 11 May 2021, 09:41:59 UTC
1 parent f70493e
Raw File
Tip revision: d116674d67eca4b4b15d7c08efd878a8c8aa864b authored by kristinas on 11 May 2021, 09:41:59 UTC
Added README
Tip revision: d116674
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