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

16 lines
248 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 CSpace"
2014-07-14 19:32:44 +00:00
theory CSpaceDecls_H
imports FaultMonad_H
begin
#INCLUDE_HASKELL SEL4/Kernel/CSpace.lhs decls_only
end