summaryrefslogtreecommitdiff
path: root/tests/coq/misc/External_FunsExternal_Template.v
blob: 7be1240a76174062afd06fbf89aa05dcfb12230e (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
(** 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::cell::{core::cell::Cell<T>#10}::get]:
    Source: '/rustc/library/core/src/cell.rs', lines 533:4-533:26
    Name pattern: core::cell::{core::cell::Cell<@T>}::get *)
Axiom core_cell_Cell_get :
  forall(T : Type) (markerCopyInst : core_marker_Copy_t T),
        core_cell_Cell_t T -> state -> result (state * T)
.

(** [core::cell::{core::cell::Cell<T>#11}::get_mut]:
    Source: '/rustc/library/core/src/cell.rs', lines 611:4-611:39
    Name pattern: core::cell::{core::cell::Cell<@T>}::get_mut *)
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_Template.