blob: a25d9c334dc2bf3b2d3d61cacf52ab8a41822d16 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
|
(** [external]: external function declarations *)
Require Import Primitives.
Import Primitives.
Require Import Coq.ZArith.ZArith.
Require Import List.
Import ListNotations.
Local Open Scope Primitives_scope.
Require Export External_Types.
Include External_Types.
Module External_FunsExternal.
Axiom core_cell_Cell_get :
forall(T : Type) (markerCopyInst : core_marker_Copy_t T),
core_cell_Cell_t T -> state -> result (state * T)
.
Axiom core_cell_Cell_get_mut :
forall(T : Type),
core_cell_Cell_t T -> state -> result (state * (T * (T -> state ->
result (state * (core_cell_Cell_t T)))))
.
End External_FunsExternal.
|