(* * Copyright 2014, General Dynamics C4 Systems * * This software may be distributed and modified according to the terms of * the GNU General Public License version 2. Note that NO WARRANTY is provided. * See "LICENSE_GPLv2.txt" for details. * * @TAG(GD_GPL) *) (* Kernel init refinement. Currently axiomatised. *) theory KernelInit_R imports IncKernelInit "AInvs.KernelInit_AI" begin (* Axiomatisation of the rest of the initialisation code *) axiomatization where init_refinement: "Init_H \ lift_state_relation state_relation `` Init_A" axiomatization where ckernel_init_valid_duplicates': "\((tc,s),x) \ Init_H. vs_valid_duplicates' (ksPSpace s)" axiomatization where ckernel_init_invs: "\((tc,s),x) \ Init_H. invs' s" axiomatization where ckernel_init_sch_norm: "((tc,s),x) \ Init_H \ ksSchedulerAction s = ResumeCurrentThread" axiomatization where ckernel_init_ctr: "((tc,s),x) \ Init_H \ ct_running' s" axiomatization where ckernel_init_domain_time: "((tc,s),x) \ Init_H \ ksDomainTime s \ 0" axiomatization where ckernel_init_domain_list: "((tc,s),x) \ Init_H \ length (ksDomSchedule s) > 0 \ (\(d,time) \ set (ksDomSchedule s). time > 0)" end