lib+spec+proof+autocorres: update for renamed Reader_Option_Monad

Signed-off-by: Corey Lewis <corey.lewis@proofcraft.systems>
This commit is contained in:
Corey Lewis 2023-07-07 15:03:17 +10:00 committed by Corey Lewis
parent 26f41e1764
commit 9b90b9e34a
14 changed files with 15 additions and 15 deletions

View File

@ -14,7 +14,7 @@ imports
Lib Lib
More_Numeral_Type More_Numeral_Type
Monads.NonDetMonadVCG Monads.NonDetMonadVCG
Monads.OptionMonad Monads.Reader_Option_Monad
begin begin
abbreviation (input) "flip \<equiv> swp" abbreviation (input) "flip \<equiv> swp"

View File

@ -19,7 +19,7 @@ imports
Injection_Handler Injection_Handler
Monads.WhileLoopRulesCompleteness Monads.WhileLoopRulesCompleteness
"Word_Lib.Distinct_Prop" (* for distinct_tuple_helper *) "Word_Lib.Distinct_Prop" (* for distinct_tuple_helper *)
Monads.OptionMonadWP Monads.Reader_Option_VCG
begin begin
lemma distinct_tuple_helper: lemma distinct_tuple_helper:

View File

@ -14,7 +14,7 @@ imports
CParser.LemmaBucket_C CParser.LemmaBucket_C
Lib.LemmaBucket Lib.LemmaBucket
SIMPL_Lemmas SIMPL_Lemmas
Monads.OptionMonadWP Monads.Reader_Option_VCG
begin begin
declare word_neq_0_conv [simp del] declare word_neq_0_conv [simp del]

View File

@ -7,7 +7,7 @@
theory Lookups_D theory Lookups_D
imports imports
"DSpec.Syscall_D" "DSpec.Syscall_D"
"Monads.OptionMonadND" "Monads.Reader_Option_ND"
begin begin
type_synonym 'a lookup = "cdl_state \<Rightarrow> 'a option" type_synonym 'a lookup = "cdl_state \<Rightarrow> 'a option"

View File

@ -10,7 +10,7 @@ imports
Word_Lib.WordSetup Word_Lib.WordSetup
Monads.Empty_Fail Monads.Empty_Fail
Monads.No_Fail Monads.No_Fail
Monads.OptionMonadND Monads.Reader_Option_ND
Lib.HaskellLib_H Lib.HaskellLib_H
Platform Platform
begin begin

View File

@ -11,7 +11,7 @@ imports
Word_Lib.WordSetup Word_Lib.WordSetup
Monads.Empty_Fail Monads.Empty_Fail
Monads.No_Fail Monads.No_Fail
Monads.OptionMonadND Monads.Reader_Option_ND
Setup_Locale Setup_Locale
Platform Platform
begin begin

View File

@ -11,7 +11,7 @@ imports
Word_Lib.WordSetup Word_Lib.WordSetup
Monads.Empty_Fail Monads.Empty_Fail
Monads.No_Fail Monads.No_Fail
Monads.OptionMonadND Monads.Reader_Option_ND
Setup_Locale Setup_Locale
Platform Platform
begin begin

View File

@ -11,7 +11,7 @@ imports
Word_Lib.WordSetup Word_Lib.WordSetup
Monads.Empty_Fail Monads.Empty_Fail
Monads.No_Fail Monads.No_Fail
Monads.OptionMonadND Monads.Reader_Option_ND
Lib.HaskellLib_H Lib.HaskellLib_H
Platform Platform
begin begin

View File

@ -11,7 +11,7 @@ imports
Word_Lib.WordSetup Word_Lib.WordSetup
Monads.Empty_Fail Monads.Empty_Fail
Monads.No_Fail Monads.No_Fail
Monads.OptionMonadND Monads.Reader_Option_ND
Lib.HaskellLib_H Lib.HaskellLib_H
Platform Platform
begin begin

View File

@ -21,7 +21,7 @@ imports
TypHeapSimple TypHeapSimple
HeapLift HeapLift
WordAbstract WordAbstract
"Monads.OptionMonadWP" "Monads.Reader_Option_VCG"
"Eisbach_Tools.Apply_Trace" "Eisbach_Tools.Apply_Trace"
AutoCorresSimpset AutoCorresSimpset
"ML_Utils.MkTermAntiquote" "ML_Utils.MkTermAntiquote"

View File

@ -13,7 +13,7 @@ theory MonadMono
imports imports
NonDetMonadEx NonDetMonadEx
Monads.WhileLoopRulesCompleteness Monads.WhileLoopRulesCompleteness
Monads.OptionMonadWP Monads.Reader_Option_VCG
begin begin
(* (*

View File

@ -16,7 +16,7 @@ imports
"Monads.More_NonDetMonadVCG" "Monads.More_NonDetMonadVCG"
"Monads.No_Throw" "Monads.No_Throw"
"Monads.No_Fail" "Monads.No_Fail"
"Monads.OptionMonadND" "Monads.Reader_Option_ND"
begin begin
(* (*
@ -276,7 +276,7 @@ lemma whileLoop_to_fold:
(\<lambda>r. return (Q r)) (\<lambda>r. return (Q r))
i s) = return (if P i \<le> x then fold (\<lambda>i r. (Q r)) [unat (P i) ..< unat x] i else i) s" i s) = return (if P i \<le> x then fold (\<lambda>i r. (Q r)) [unat (P i) ..< unat x] i else i) s"
(is "?LHS s = return (?RHS x) s") (is "?LHS s = return (?RHS x) s")
apply (subst OptionMonadND.gets_the_return [symmetric]) apply (subst Reader_Option_ND.gets_the_return [symmetric])
apply (subst gets_the_whileLoop) apply (subst gets_the_whileLoop)
apply (rule gets_the_to_return) apply (rule gets_the_to_return)
apply (subst owhile_to_fold) apply (subst owhile_to_fold)

View File

@ -14,7 +14,7 @@
theory TypeStrengthen theory TypeStrengthen
imports imports
L2Defs L2Defs
"Monads.OptionMonadND" "Monads.Reader_Option_ND"
ExecConcrete ExecConcrete
begin begin

View File

@ -10,7 +10,7 @@ Termination for recursive functions.
theory FactorialTest theory FactorialTest
imports imports
"AutoCorres.AutoCorres" "AutoCorres.AutoCorres"
"Monads.OptionMonadWP" "Monads.Reader_Option_VCG"
begin begin
external_file "factorial.c" external_file "factorial.c"