(** 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#10}::get]: Source: '/rustc/ad963232d9b987d66a6f8e6ec4141f672b8b9900/library/core/src/cell.rs', lines 497:4-497: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#11}::get_mut]: Source: '/rustc/ad963232d9b987d66a6f8e6ec4141f672b8b9900/library/core/src/cell.rs', lines 574:4-574: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.