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

18 lines
220 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 "Kernel"
2014-07-14 19:32:44 +00:00
theory Kernel_H
imports
KernelInit_H
Thread_H
FaultHandler_H
CSpace_H
Hypervisor_H
2014-07-14 19:32:44 +00:00
begin
end