diff --git a/lib/Monads/trace/Trace_More_RG.thy b/lib/Monads/trace/Trace_More_RG.thy index 0a5a8b5c4d..b409c3dffe 100644 --- a/lib/Monads/trace/Trace_More_RG.thy +++ b/lib/Monads/trace/Trace_More_RG.thy @@ -310,7 +310,7 @@ lemma ifM_throwError_returnOkI: lemmas state_unchanged_rg = in_inv_by_rgD [THEN sym] lemmas last_state_unchanged_rg = last_st_in_inv_by_rgD [THEN sym] -\ \FIXME MC: name? move (both this one and validI in More_VCG)\ +(*FIXME MC: name? move (both this one and validI in More_VCG)*) lemma validI_I: assumes px: "prefix_closed S" assumes gc: "\s0 s tr res. \ P s0 s; (tr, res) \ (rely S R s0 s)\ \ guar_cond G s0 tr" @@ -515,7 +515,7 @@ lemma rg_walk_assmsE: apply (auto simp: y split: sum.splits) done -\ \FIXME MC: it is not immediately obvious what the validI equivalent of these rules should be, so I +(*FIXME MC: it is not immediately obvious what the validI equivalent of these rules should be, so I think it is best to leave them until we have a specific use case. lemma univ_twp: "prefix_closed f \ \\s0 s. \(rv, s') \ mres (rely f R s0 s). Q rv s0 s'\,\R\ f -,\Q\" @@ -548,7 +548,7 @@ lemma other_rg_in_monad_post: apply clarsimp apply (drule bspec, assumption, simp) done - qed\ + qed*) lemma weak_if_twp: "\ \P\,\R\ f \G\,\Q\; \P'\,\R\ f \G\,\Q'\ \ \ diff --git a/lib/Monads/trace/Trace_RG.thy b/lib/Monads/trace/Trace_RG.thy index 3a5833a3ec..23d39732cd 100644 --- a/lib/Monads/trace/Trace_RG.thy +++ b/lib/Monads/trace/Trace_RG.thy @@ -289,12 +289,11 @@ lemma validIE_validE_no_trace_eq: apply (clarsimp simp: validI_valid_no_trace_eq) done -\ \FIXME MC: name\ +(*FIXME MC: name*) lemma validI_split: "\\P\,\R\ f -,\Q\; \P'\,\R\ f \G\,\\\\\\ \ \P and P'\,\R\ f \G\,\Q\" by (auto simp: validI_def) -\ \FIXME MC: name\ lemma validIE_split: "\\P\,\R\ f -,\Q\,\E\; \P'\,\R\ f \G\,\\\\\,\\\\\\ \ \P and P'\,\R\ f \G\,\Q\,\E\" by (auto simp: validIE_def validI_split) @@ -800,7 +799,7 @@ lemma validIE_eq_validI: subsection \@{const liftM}\ -\ \FIXME MC: make proof nicer\ +(*FIXME: make proof nicer*) lemma rg_liftM_subst: "\P\,\R\ liftM f m \G\,\Q\ = \P\,\R\ m \G\,\Q \ f\" apply (clarsimp simp: validI_def) @@ -1028,8 +1027,8 @@ lemma rg_vcg_const_imp_liftE_R: by (rule rg_strengthen_post) (fastforce intro!: rg_vcg_const_imp_lift split: sum.splits)+ -\ \FIXME MC: not clear whether we want these _T variants, and if we do whether they should be in the - wp set along with the above rules\ +(*FIXME MC: not clear whether we want these _T variants, and if we do whether they should be in the + wp set along with the above rules*) lemmas rg_vcg_const_imp_lift_T = rg_vcg_const_imp_lift[where G="\\" and P''="\\", simplified] lemmas rg_vcg_const_imp_liftE_E_T = rg_vcg_const_imp_liftE_E[where G="\\" and P''="\\", simplified] lemmas rg_vcg_const_imp_liftE_R_T = rg_vcg_const_imp_liftE_R[where G="\\" and P''="\\", simplified] @@ -1321,12 +1320,12 @@ lemma whenE_throwError_twp: "\\s0 s. \P \ Q s0 s\,\R\ whenE P (throwError e) \G\,\\_. Q\,-" by (simp add: whenE_def returnOk_def throwError_def return_def validIE_def validI_def prefix_closed_def) -\ \FIXME MC: not used, worth updating for validI or just delete? +(*FIXME MC: not used, worth updating for validI or just delete? lemma select_throwError_twp: "\\s0 s. \x\S. Q x s0 s\,\R\ select S >>= throwError \G\,-,\Q\" - by (simp add: bind_def throwError_def return_def select_def validIE_def validI_def prefix_closed_def)\ + by (simp add: bind_def throwError_def return_def select_def validIE_def validI_def prefix_closed_def)*) -\ \FIXME MC: explore adding a rely_preserves definition for the first part of this precondition\ +(*FIXME MC: explore adding a rely_preserves definition for the first part of this precondition*) lemma env_steps_twp[wp]: "\\s0 s. (\s'. R\<^sup>*\<^sup>* s0 s' \ Q () s' s') \ Q () s0 s\,\R\ env_steps \G\,\Q\" apply (simp add: env_steps_def)