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

15 lines
273 B
Plaintext

(*
* Copyright 2014, General Dynamics C4 Systems
*
* SPDX-License-Identifier: GPL-2.0-only
*)
chapter "Function Declarations for Notifications"
theory NotificationDecls_H imports "FaultMonad_H"
begin
#INCLUDE_HASKELL SEL4/Object/Notification.lhs decls_only
end