summaryrefslogtreecommitdiff
path: root/tests/lean/External/FunsExternal_Template.lean
diff options
context:
space:
mode:
authorRyan Lahfa2024-04-17 00:01:34 +0200
committerRyan Lahfa2024-04-24 11:04:11 +0200
commit18484e28ef7b13b95dc3af0b1e34c2181e1778e5 (patch)
treef9480db9b7b00df8a2c4eae43c9705be5b8e2928 /tests/lean/External/FunsExternal_Template.lean
parentc264b08cfb9beb5fe34d872b02a8f4cd1e12d45e (diff)
compiler: map `core::mem::swap` to the pure swap
In the pure functional model, `swap` is mostly about borrow checking and should simplify to the pure swap in our backends. Other backends than Lean are not done in this commit. Signed-off-by: Ryan Lahfa <ryan.lahfa@inria.fr>
Diffstat (limited to '')
-rw-r--r--tests/lean/External/FunsExternal_Template.lean6
1 files changed, 0 insertions, 6 deletions
diff --git a/tests/lean/External/FunsExternal_Template.lean b/tests/lean/External/FunsExternal_Template.lean
index 38151dc9..f0e771f7 100644
--- a/tests/lean/External/FunsExternal_Template.lean
+++ b/tests/lean/External/FunsExternal_Template.lean
@@ -6,12 +6,6 @@ import External.Types
open Primitives
open external
-/- [core::mem::swap]:
- Source: '/rustc/d59363ad0b6391b7fc5bbb02c9ccf9300eef3753/library/core/src/mem/mod.rs', lines 726:0-726:42
- Name pattern: core::mem::swap -/
-axiom core.mem.swap
- (T : Type) : T → T → State → Result (State × (T × T))
-
/- [core::num::nonzero::{core::num::nonzero::NonZeroU32#14}::new]:
Source: '/rustc/d59363ad0b6391b7fc5bbb02c9ccf9300eef3753/library/core/src/num/nonzero.rs', lines 79:16-79:57
Name pattern: core::num::nonzero::{core::num::nonzero::NonZeroU32}::new -/