summaryrefslogtreecommitdiff
path: root/tests/coq/misc/External_FunsExternal_Template.v
blob: 31e69c398740a7ff58e2a93c864cc8d31d84eb2b (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
37
38
39
40
41
42
43
44
(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
(** [external]: external functions.
-- This is a template file: rename it to "FunsExternal.lean" and fill the holes. *)
Require Import Primitives.
Import Primitives.
Require Import Coq.ZArith.ZArith.
Require Import List.
Import ListNotations.
Local Open Scope Primitives_scope.
Require Import External_Types.
Include External_Types.
Module External_FunsExternal_Template.

(** [core::mem::swap]: forward function
    Source: '/rustc/d59363ad0b6391b7fc5bbb02c9ccf9300eef3753/library/core/src/mem/mod.rs', lines 726:0-726:42 *)
Axiom core_mem_swap :
  forall(T : Type), T -> T -> state -> result (state * unit)
.

(** [core::mem::swap]: backward function 0
    Source: '/rustc/d59363ad0b6391b7fc5bbb02c9ccf9300eef3753/library/core/src/mem/mod.rs', lines 726:0-726:42 *)
Axiom core_mem_swap_back0 :
  forall(T : Type), T -> T -> state -> state -> result (state * T)
.

(** [core::mem::swap]: backward function 1
    Source: '/rustc/d59363ad0b6391b7fc5bbb02c9ccf9300eef3753/library/core/src/mem/mod.rs', lines 726:0-726:42 *)
Axiom core_mem_swap_back1 :
  forall(T : Type), T -> T -> state -> state -> result (state * T)
.

(** [core::num::nonzero::{core::num::nonzero::NonZeroU32#14}::new]: forward function
    Source: '/rustc/d59363ad0b6391b7fc5bbb02c9ccf9300eef3753/library/core/src/num/nonzero.rs', lines 79:16-79:57 *)
Axiom core_num_nonzero_NonZeroU32_new
  : u32 -> state -> result (state * (option core_num_nonzero_NonZeroU32_t))
.

(** [core::option::{core::option::Option<T>}::unwrap]: forward function
    Source: '/rustc/d59363ad0b6391b7fc5bbb02c9ccf9300eef3753/library/core/src/option.rs', lines 932:4-932:34 *)
Axiom core_option_Option_unwrap :
  forall(T : Type), option T -> state -> result (state * T)
.

End External_FunsExternal_Template.