lh-l4v/spec/design/skel/ThreadDecls_H.thy

20 lines
330 B
Plaintext
Raw Normal View History

2014-07-14 19:32:44 +00:00
(*
* Copyright 2014, General Dynamics C4 Systems
*
2020-03-09 06:18:30 +00:00
* SPDX-License-Identifier: GPL-2.0-only
2014-07-14 19:32:44 +00:00
*)
2015-05-16 09:52:49 +00:00
chapter "Function Declarations for Threads"
2014-07-14 19:32:44 +00:00
theory ThreadDecls_H
imports
Structures_H
FaultMonad_H
KernelInitMonad_H
ArchThreadDecls_H
2014-07-14 19:32:44 +00:00
begin
#INCLUDE_HASKELL SEL4/Kernel/Thread.lhs decls_only NOT transferCapsToSlots
end