diff --git a/proof/crefine/ARM/IsolatedThreadAction.thy b/proof/crefine/ARM/IsolatedThreadAction.thy index de6f61a0c21..40156e314b4 100644 --- a/proof/crefine/ARM/IsolatedThreadAction.thy +++ b/proof/crefine/ARM/IsolatedThreadAction.thy @@ -247,12 +247,12 @@ lemma zipWithM_setRegister_simple: simpler_modify_def fun_upd_def[symmetric]) done -(* these variant used in fastpath rewrite proof *) +(* this variant used in fastpath rewrite proof *) lemma setRegister_simple_modify_registers: "setRegister r v = (\con. ({((), modify_registers (\f. f(r := v)) con)}, False))" by (simp add: modify_registers_def setRegister_simple) -(* these variant used in fastpath rewrite proof *) +(* this variant used in fastpath rewrite proof *) lemma zipWithM_setRegister_simple_modify_registers: "zipWithM_x setRegister rs vs = (\con. ({((), modify_registers (\regs. foldl (\f (r,v). f(r := v)) regs (zip rs vs)) con)}, diff --git a/proof/crefine/ARM_HYP/IsolatedThreadAction.thy b/proof/crefine/ARM_HYP/IsolatedThreadAction.thy index d071752830e..939a16a2e9f 100644 --- a/proof/crefine/ARM_HYP/IsolatedThreadAction.thy +++ b/proof/crefine/ARM_HYP/IsolatedThreadAction.thy @@ -244,12 +244,12 @@ lemma zipWithM_setRegister_simple: simpler_modify_def fun_upd_def[symmetric]) done -(* these variant used in fastpath rewrite proof *) +(* this variant used in fastpath rewrite proof *) lemma setRegister_simple_modify_registers: "setRegister r v = (\con. ({((), modify_registers (\f. f(r := v)) con)}, False))" by (simp add: modify_registers_def setRegister_simple) -(* these variant used in fastpath rewrite proof *) +(* this variant used in fastpath rewrite proof *) lemma zipWithM_setRegister_simple_modify_registers: "zipWithM_x setRegister rs vs = (\con. ({((), modify_registers (\regs. foldl (\f (r,v). f(r := v)) regs (zip rs vs)) con)}, diff --git a/proof/drefine/Schedule_DR.thy b/proof/drefine/Schedule_DR.thy index 14476b1d8b6..3b469648092 100644 --- a/proof/drefine/Schedule_DR.thy +++ b/proof/drefine/Schedule_DR.thy @@ -625,7 +625,6 @@ lemma transform_tcb_NextIP: = transform_tcb m t tcb" apply (rule ext) apply (simp add: transform_tcb_def transform_full_intent_def Let_def) - by (auto simp add: transform_tcb_def transform_full_intent_def Let_def cap_register_def ARM.capRegister_def arch_tcb_context_get_def) diff --git a/proof/refine/ARM/TcbAcc_R.thy b/proof/refine/ARM/TcbAcc_R.thy index 73377a464a3..932ff1dc4f3 100644 --- a/proof/refine/ARM/TcbAcc_R.thy +++ b/proof/refine/ARM/TcbAcc_R.thy @@ -4255,7 +4255,7 @@ proof - show ?thesis using m unfolding setMRs_def set_mrs_def - apply (clarsimp cong: option.case_cong split del: if_split) + apply (clarsimp cong: option.case_cong split del: if_split) apply (subst bind_assoc[symmetric]) apply (fold thread_set_def[simplified]) apply (subst thread_set_as_user_registers) diff --git a/proof/refine/ARM_HYP/TcbAcc_R.thy b/proof/refine/ARM_HYP/TcbAcc_R.thy index 839b3698ccb..9ffb18e7650 100644 --- a/proof/refine/ARM_HYP/TcbAcc_R.thy +++ b/proof/refine/ARM_HYP/TcbAcc_R.thy @@ -4306,7 +4306,7 @@ proof - show ?thesis using m unfolding setMRs_def set_mrs_def - apply (clarsimp cong: option.case_cong split del: if_split) + apply (clarsimp cong: option.case_cong split del: if_split) apply (subst bind_assoc[symmetric]) apply (fold thread_set_def[simplified]) apply (subst thread_set_as_user_registers) diff --git a/spec/machine/ARM/MachineOps.thy b/spec/machine/ARM/MachineOps.thy index 5f7c64252cd..52bc600c454 100644 --- a/spec/machine/ARM/MachineOps.thy +++ b/spec/machine/ARM/MachineOps.thy @@ -504,7 +504,7 @@ type_synonym 'a user_monad = "(user_context, 'a) nondet_monad" definition getRegister :: "register \ machine_word user_monad" where "getRegister r \ gets (\s. user_regs s r)" -definition +definition modify_registers :: "(user_regs \ user_regs) \ user_context \ user_context" where "modify_registers f uc \ UserContext (f (user_regs uc))" definition setRegister :: "register \ machine_word \ unit user_monad" where diff --git a/spec/machine/ARM_HYP/MachineOps.thy b/spec/machine/ARM_HYP/MachineOps.thy index 49c9434c6f6..d08071e0cd6 100644 --- a/spec/machine/ARM_HYP/MachineOps.thy +++ b/spec/machine/ARM_HYP/MachineOps.thy @@ -729,7 +729,7 @@ type_synonym 'a user_monad = "(user_context, 'a) nondet_monad" definition getRegister :: "register \ machine_word user_monad" where "getRegister r \ gets (\s. user_regs s r)" -definition +definition modify_registers :: "(user_regs \ user_regs) \ user_context \ user_context" where "modify_registers f uc \ UserContext (f (user_regs uc))" definition setRegister :: "register \ machine_word \ unit user_monad" where