diff options
author | Son HO | 2024-06-17 23:30:10 +0200 |
---|---|---|
committer | GitHub | 2024-06-17 23:30:10 +0200 |
commit | 878be6d051f2f920fdc6c90add8423fa6f489492 (patch) | |
tree | c967637249ea1c9001983e09e1f04f17b8e0a1d4 /tests/coq/misc/External_Funs.v | |
parent | 820916ca6d5b247417b18bb8b9d981b7ef0a9195 (diff) | |
parent | 76ab141814644a94bffc8497e5845436d86b1083 (diff) |
Merge branch 'main' into son/cleanup
Diffstat (limited to '')
-rw-r--r-- | tests/coq/misc/External_Funs.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/tests/coq/misc/External_Funs.v b/tests/coq/misc/External_Funs.v index 6c5bbdd2..699db6a7 100644 --- a/tests/coq/misc/External_Funs.v +++ b/tests/coq/misc/External_Funs.v @@ -13,7 +13,7 @@ Include External_FunsExternal. Module External_Funs. (** Trait implementation: [core::marker::{(core::marker::Copy for u32)#61}] - Source: '/rustc/65ea825f4021eaf77f1b25139969712d65b435a4/library/core/src/marker.rs', lines 47:29-47:65 + Source: '/rustc/library/core/src/marker.rs', lines 47:29-47:65 Name pattern: core::marker::Copy<u32> *) Definition core_marker_CopyU32 : core_marker_Copy_t u32 := {| core_marker_Copy_tcore_marker_Copy_t_cloneCloneInst := core_clone_CloneU32; |