summaryrefslogtreecommitdiff
path: root/tests/coq/misc/External__Opaque.v
blob: 19111a373b56ebd57c2eca7e1440ea9ca2b27896 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
(** [external]: opaque function definitions *)
Require Import Primitives.
Import Primitives.
Require Import Coq.ZArith.ZArith.
Local Open Scope Primitives_scope.
Require Export External__Types .
Import External__Types .
Module External__Opaque .

(** [core::mem::swap] *)
Axiom core_mem_swap_fwd :
  forall(T : Type) , T -> T -> state -> result (state * unit)
  .

(** [core::mem::swap] *)
Axiom core_mem_swap_back0 :
  forall(T : Type) , T -> T -> state -> state -> result (state * T)
  .

(** [core::mem::swap] *)
Axiom core_mem_swap_back1 :
  forall(T : Type) , T -> T -> state -> state -> result (state * T)
  .

(** [core::num::nonzero::NonZeroU32::{14}::new] *)
Axiom core_num_nonzero_non_zero_u32_new_fwd
  : u32 -> state -> result (state * (option Core_num_nonzero_non_zero_u32_t))
  .

(** [core::option::Option::{0}::unwrap] *)
Axiom core_option_option_unwrap_fwd :
  forall(T : Type) , option T -> state -> result (state * T)
  .

End External__Opaque .