Skip to content

Commit

Permalink
trivial: rename arch_split -> arch-split
Browse files Browse the repository at this point in the history
Unifying the tag between Github labels, docs, and so on will make it
less confusing to grep for and deal with.

Signed-off-by: Rafal Kolanski <[email protected]>
  • Loading branch information
Xaphiosis committed Jul 26, 2024
1 parent 423e5d4 commit 0875edf
Show file tree
Hide file tree
Showing 320 changed files with 754 additions and 754 deletions.
12 changes: 6 additions & 6 deletions docs/arch-split.md
Original file line number Diff line number Diff line change
Expand Up @@ -111,7 +111,7 @@ theory Retype_R
imports VSpace_R
begin
context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)
lemma placeNewObject_def2:
"placeNewObject ptr val gb = createObjects' ptr 1 (injectKO val) gb"
Expand Down Expand Up @@ -199,7 +199,7 @@ architecture. If we saw such a reference in a generic theory, we would
immediately recognise that something was wrong.

The convention is that in architecture-specific theories, we initially
give *all* types, constants and lemmas with the architecture-specific
give *all* types, constants and lemmas the architecture-specific
`arch_global_naming` scheme. Then, in generic theories, we use
*requalification* to selectively extract just those types, constants and
facts which are expected to exist on all architectures.
Expand Down Expand Up @@ -339,7 +339,7 @@ available unqualified until the end of the context block. Indeed, in this case,
the only purpose of the anonymous context block is to limit the scope of this
`interpretation`.

Note: It is critical to the success of arch_split that we *never* interpret the
Note: It is critical to the success of arch-split that we *never* interpret the
Arch locale, *except* inside an appropriate context block.

In a generic theory, we typically only interpret the Arch locale to keep
Expand Down Expand Up @@ -770,7 +770,7 @@ will only ever look at the heap, so this proof will always work.

There are some considerations when using this strategy:

1. We use the Arch locale without a `global_naming`, as its performance better
1. We use the Arch locale without `global_naming`, as its performance is better
than entering the Arch locale and proving the lemma there. This means its
qualified name will be `Arch.valid_arch_cap_pspaceI`, but this is acceptable
since:
Expand Down Expand Up @@ -869,7 +869,7 @@ The workflow:
intra-theory dependencies" above.

- Look in the generic theory for a block of the form
`context Arch begin (* FIXME: arch_split *) ... end`.
`context Arch begin (* FIXME: arch-split *) ... end`.

- These indicate things that we've previously classified as belonging in an
arch-specific theory.
Expand All @@ -881,7 +881,7 @@ The workflow:
- Look for subsequent breakage in the generic theory.

- If this is in a subsequent Arch block (`context Arch begin (* FIXME:
arch_split *) ... end`), just move that block.
arch-split *) ... end`), just move that block.

- Otherwise, if it's not obvious what to do, have a conversation with someone.
We'll add more tips here as the process becomes clearer.
Expand Down
2 changes: 1 addition & 1 deletion proof/access-control/ARM/ArchIpc_AC.thy
Original file line number Diff line number Diff line change
Expand Up @@ -192,7 +192,7 @@ declare arch_get_sanitise_register_info_inv[Ipc_AC_assms]
end


context is_extended begin interpretation Arch . (*FIXME: arch_split*)
context is_extended begin interpretation Arch . (*FIXME: arch-split*)

lemma list_integ_lift_in_ipc[Ipc_AC_assms]:
assumes li:
Expand Down
2 changes: 1 addition & 1 deletion proof/access-control/ARM/ExampleSystem.thy
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ theory ExampleSystem
imports ArchAccess_AC
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
nat_to_bl :: "nat \<Rightarrow> nat \<Rightarrow> bool list option"
Expand Down
2 changes: 1 addition & 1 deletion proof/access-control/RISCV64/ExampleSystem.thy
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ theory ExampleSystem
imports ArchAccess_AC
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
nat_to_bl :: "nat \<Rightarrow> nat \<Rightarrow> bool list option"
Expand Down
2 changes: 1 addition & 1 deletion proof/bisim/Syscall_S.thy
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ theory Syscall_S
imports Separation
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma syscall_bisim:
assumes bs:
Expand Down
6 changes: 3 additions & 3 deletions proof/crefine/AARCH64/ADT_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -220,7 +220,7 @@ end
consts
Init_C' :: "unit observable \<Rightarrow> cstate global_state set"

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition "Init_C \<equiv> \<lambda>((tc,s),m,e). Init_C' ((tc, truncate_state s),m,e)"

Expand Down Expand Up @@ -345,7 +345,7 @@ lemma cint_rel_to_H:

end

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
"cstate_to_machine_H s \<equiv>
Expand Down Expand Up @@ -630,7 +630,7 @@ lemma carch_state_to_H_correct:

end

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma tcb_queue_rel_unique:
"hp NULL = None \<Longrightarrow>
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/Arch_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@ begin

unbundle l4v_word_context

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

crunch unmapPageTable
for gsMaxObjectSize[wp]: "\<lambda>s. P (gsMaxObjectSize s)"
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/CLevityCatch.thy
Original file line number Diff line number Diff line change
Expand Up @@ -73,7 +73,7 @@ qed
(* end holding area *)


context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

(* Short-hand for unfolding cumbersome machine constants *)
(* FIXME MOVE these should be in refine, and the _eq forms should NOT be declared [simp]! *)
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/DetWP.thy
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,7 @@ theory DetWP
imports "Lib.DetWPLib" "CBaseRefine.Include_C"
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma det_wp_doMachineOp [wp]:
"det_wp (\<lambda>_. P) f \<Longrightarrow> det_wp (\<lambda>_. P) (doMachineOp f)"
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/Fastpath_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,7 @@ imports
"CLib.MonadicRewrite_C"
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma setCTE_obj_at'_queued:
"\<lbrace>obj_at' (\<lambda>tcb. P (tcbQueued tcb)) t\<rbrace> setCTE p v \<lbrace>\<lambda>rv. obj_at' (\<lambda>tcb. P (tcbQueued tcb)) t\<rbrace>"
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/Fastpath_Defs.thy
Original file line number Diff line number Diff line change
Expand Up @@ -15,7 +15,7 @@ theory Fastpath_Defs
imports ArchMove_C
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
"fastpaths sysc \<equiv> case sysc of
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/Fastpath_Equiv.thy
Original file line number Diff line number Diff line change
Expand Up @@ -45,7 +45,7 @@ lemma setCTE_tcbContext:
apply (rule setObject_cte_obj_at_tcb', simp_all)
done

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma setThreadState_tcbContext:
"setThreadState st tptr \<lbrace>obj_at' (\<lambda>tcb. P ((atcbContextGet o tcbArch) tcb)) t\<rbrace>"
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/Invoke_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -1382,7 +1382,7 @@ lemma decodeCNodeInvocation_ccorres:

end

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemmas setCTE_def3 = setCTE_def2[THEN eq_reflection]

Expand Down
8 changes: 4 additions & 4 deletions proof/crefine/AARCH64/Ipc_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ imports
IsolatedThreadAction
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
"replyFromKernel_success_empty thread \<equiv> do
Expand Down Expand Up @@ -292,7 +292,7 @@ lemma ccap_relation_reply_helpers:
cap_reply_cap_lift_def word_size
elim!: ccap_relationE)

(*FIXME: arch_split: C kernel names hidden by Haskell names *)
(*FIXME: arch-split: C kernel names hidden by Haskell names *)
(*FIXME: fupdate simplification issues for 2D arrays *)
abbreviation "syscallMessageC \<equiv> kernel_all_global_addresses.fault_messages.[unat MessageID_Syscall]"
lemmas syscallMessageC_def = kernel_all_substitute.fault_messages_def
Expand All @@ -315,7 +315,7 @@ lemma syscallMessage_ccorres:

end

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
"handleArchFaultReply' f sender receiver tag \<equiv>
Expand Down Expand Up @@ -1041,7 +1041,7 @@ lemma setMR_ccorres_dc:
end

(* FIXME: move *)
context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)
crunch setMR
for valid_pspace'[wp]: "valid_pspace'"
crunch setMR
Expand Down
4 changes: 2 additions & 2 deletions proof/crefine/AARCH64/IsolatedThreadAction.thy
Original file line number Diff line number Diff line change
Expand Up @@ -156,7 +156,7 @@ lemma partial_overwrite_fun_upd:
apply (clarsimp split: if_split)
done

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma get_tcb_state_regs_ko_at':
"ko_at' ko p s \<Longrightarrow> get_tcb_state_regs (ksPSpace s p)
Expand Down Expand Up @@ -1349,7 +1349,7 @@ lemma bind_assoc:
= do x \<leftarrow> m; y \<leftarrow> f x; g y od"
by (rule bind_assoc)

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma setObject_modify_assert:
"\<lbrakk> updateObject v = updateObject_default v \<rbrakk>
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/Recycle_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -533,7 +533,7 @@ lemma heap_to_user_data_in_user_mem'[simp]:
apply simp+
done

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma setObject_asidpool_gs[wp]:
"setObject ptr (vcpu::asidpool) \<lbrace>\<lambda>s. P (gsMaxObjectSize s)\<rbrace>"
Expand Down
4 changes: 2 additions & 2 deletions proof/crefine/AARCH64/Retype_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -41,7 +41,7 @@ lemma zero_le_sint: "\<lbrakk> 0 \<le> (a :: machine_word); a < 0x80000000000000
apply simp
done

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma map_option_byte_to_word_heap:
assumes disj: "\<And>(off :: 9 word) x. x<8 \<Longrightarrow> p + ucast off * 8 + x \<notin> S " (*9=page table index*)
Expand Down Expand Up @@ -7833,7 +7833,7 @@ lemma APIType_capBits_min:

end

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma createNewCaps_1_gsCNodes_p:
"\<lbrace>\<lambda>s. P (gsCNodes s p) \<and> p \<noteq> ptr\<rbrace> createNewCaps newType ptr 1 n dev\<lbrace>\<lambda>rv s. P (gsCNodes s p)\<rbrace>"
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/SR_lemmas_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@ imports
"Refine.Invariants_H"
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

section "vm rights"

Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/Schedule_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@ begin

instance tcb :: no_vcpu by intro_classes auto

(*FIXME: arch_split: move up?*)
(*FIXME: arch-split: move up?*)
context Arch begin
context begin global_naming global
requalify_facts
Expand Down
8 changes: 4 additions & 4 deletions proof/crefine/AARCH64/StateRelation_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ theory StateRelation_C
imports Wellformed_C
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
"lifth p s \<equiv> the (clift (t_hrs_' s) p)"
Expand Down Expand Up @@ -81,7 +81,7 @@ text \<open>
which can subsequently be instantiated for
@{text kernel_all_global_addresses} as well as @{text kernel_all_substitute}.
\<close>
locale state_rel = Arch + substitute_pre + (*FIXME: arch_split*)
locale state_rel = Arch + substitute_pre + (*FIXME: arch-split*)
fixes armKSKernelVSpace_C :: "machine_word \<Rightarrow> arm_vspace_region_use"

locale kernel = kernel_all_substitute + state_rel
Expand Down Expand Up @@ -133,7 +133,7 @@ definition carch_state_relation :: "Arch.kernel_state \<Rightarrow> globals \<Ri

end

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
cmachine_state_relation :: "machine_state \<Rightarrow> globals \<Rightarrow> bool"
Expand Down Expand Up @@ -709,7 +709,7 @@ where
((\<not> (d \<le> maxDomain \<and> i < l2BitmapSize))
\<longrightarrow> abitmap2 (d, i) = 0)"

end (* interpretation Arch . (*FIXME: arch_split*) *)
end (* interpretation Arch . (*FIXME: arch-split*) *)

definition
region_is_bytes' :: "machine_word \<Rightarrow> nat \<Rightarrow> heap_typ_desc \<Rightarrow> bool"
Expand Down
6 changes: 3 additions & 3 deletions proof/crefine/AARCH64/SyscallArgs_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -13,13 +13,13 @@ imports
StoreWord_C DetWP
begin

(*FIXME: arch_split: C kernel names hidden by Haskell names *)
(*FIXME: arch-split: C kernel names hidden by Haskell names *)
context kernel_m begin
abbreviation "msgRegistersC \<equiv> kernel_all_substitute.msgRegisters"
lemmas msgRegistersC_def = kernel_all_substitute.msgRegisters_def
end

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

declare word_neq_0_conv[simp del]

Expand Down Expand Up @@ -1201,7 +1201,7 @@ lemma getSyscallArg_ccorres_foo:

end

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma invocation_eq_use_type:
"\<lbrakk> value \<equiv> (value' :: 32 signed word);
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/Syscall_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -15,7 +15,7 @@ imports
Arch_C
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)
crunch replyFromKernel
for sch_act_wf[wp]: "\<lambda>s. sch_act_wf (ksSchedulerAction s) s"
end
Expand Down
4 changes: 2 additions & 2 deletions proof/crefine/AARCH64/Tcb_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -59,7 +59,7 @@ lemma doMachineOp_sched:
apply fastforce
done

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)
crunch restart
for curThread[wp]: "\<lambda>s. P (ksCurThread s)"
(wp: crunch_wps simp: crunch_simps)
Expand Down Expand Up @@ -1105,7 +1105,7 @@ lemma Arch_performTransfer_ccorres:
apply simp+
done

(*FIXME: arch_split: C kernel names hidden by Haskell names *)
(*FIXME: arch-split: C kernel names hidden by Haskell names *)
abbreviation "frameRegistersC \<equiv> kernel_all_substitute.frameRegisters"
lemmas frameRegistersC_def = kernel_all_substitute.frameRegisters_def
abbreviation "gpRegistersC \<equiv> kernel_all_substitute.gpRegisters"
Expand Down
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/VSpace_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -19,7 +19,7 @@ autocorres
c_locale = kernel_all_substitute
] "../c/build/$L4V_ARCH/kernel_all.c_pp"

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

lemma ccorres_name_pre_C:
"(\<And>s. s \<in> P' \<Longrightarrow> ccorres_underlying sr \<Gamma> r xf arrel axf P {s} hs f g)
Expand Down
4 changes: 2 additions & 2 deletions proof/crefine/AARCH64/Wellformed_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -15,7 +15,7 @@ imports
"CSpec.Substitute"
begin

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

(* Takes an address and ensures it can be given to a function expecting a canonical address.
Canonical addresses on 64-bit machines aren't really 64-bit, due to bus sizes. Hence, structures
Expand Down Expand Up @@ -303,7 +303,7 @@ record cte_CL =
cap_CL :: cap_CL
cteMDBNode_CL :: mdb_node_CL

context begin interpretation Arch . (*FIXME: arch_split*)
context begin interpretation Arch . (*FIXME: arch-split*)

definition
cte_lift :: "cte_C \<rightharpoonup> cte_CL"
Expand Down
Loading

0 comments on commit 0875edf

Please sign in to comment.