Skip to content

Commit

Permalink
lib+spec+proof+tools: update for reader_option refactor
Browse files Browse the repository at this point in the history
Signed-off-by: Corey Lewis <[email protected]>
  • Loading branch information
corlewis committed Feb 29, 2024
1 parent d08f849 commit cf75dfb
Show file tree
Hide file tree
Showing 11 changed files with 11 additions and 18 deletions.
3 changes: 1 addition & 2 deletions lib/HaskellLib_H.thy
Original file line number Diff line number Diff line change
Expand Up @@ -14,8 +14,7 @@ imports
Lib
More_Numeral_Type
Monads.Nondet_VCG
Monads.Reader_Option_Monad
Monads.Reader_Option_VCG
Monads.Nondet_Reader_Option
begin

abbreviation (input) "flip \<equiv> swp"
Expand Down
2 changes: 1 addition & 1 deletion lib/NonDetMonadLemmaBucket.thy
Original file line number Diff line number Diff line change
Expand Up @@ -19,7 +19,7 @@ imports
Injection_Handler
Monads.Nondet_While_Loop_Rules_Completeness
"Word_Lib.Distinct_Prop" (* for distinct_tuple_helper *)
Monads.Reader_Option_VCG
Monads.Nondet_Reader_Option
begin

lemma distinct_tuple_helper:
Expand Down
2 changes: 1 addition & 1 deletion lib/clib/Corres_UL_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ imports
CParser.LemmaBucket_C
Lib.LemmaBucket
SIMPL_Lemmas
Monads.Reader_Option_VCG
Monads.Nondet_Reader_Option
begin

declare word_neq_0_conv [simp del]
Expand Down
2 changes: 1 addition & 1 deletion proof/sep-capDL/Lookups_D.thy
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@
theory Lookups_D
imports
"DSpec.Syscall_D"
"Monads.Reader_Option_ND"
"Monads.Nondet_Reader_Option"
begin

type_synonym 'a lookup = "cdl_state \<Rightarrow> 'a option"
Expand Down
3 changes: 1 addition & 2 deletions spec/design/m-skel/AARCH64/MachineTypes.thy
Original file line number Diff line number Diff line change
Expand Up @@ -9,8 +9,7 @@ theory MachineTypes
imports
Word_Lib.WordSetup
Monads.Nondet_Empty_Fail
Monads.Nondet_No_Fail
Monads.Reader_Option_ND
Monads.Nondet_Reader_Option
Lib.HaskellLib_H
Platform
begin
Expand Down
3 changes: 1 addition & 2 deletions spec/design/m-skel/ARM/MachineTypes.thy
Original file line number Diff line number Diff line change
Expand Up @@ -10,8 +10,7 @@ theory MachineTypes
imports
Word_Lib.WordSetup
Monads.Nondet_Empty_Fail
Monads.Nondet_No_Fail
Monads.Reader_Option_ND
Monads.Nondet_Reader_Option
Setup_Locale
Platform
begin
Expand Down
3 changes: 1 addition & 2 deletions spec/design/m-skel/ARM_HYP/MachineTypes.thy
Original file line number Diff line number Diff line change
Expand Up @@ -10,8 +10,7 @@ theory MachineTypes
imports
Word_Lib.WordSetup
Monads.Nondet_Empty_Fail
Monads.Nondet_No_Fail
Monads.Reader_Option_ND
Monads.Nondet_Reader_Option
Setup_Locale
Platform
begin
Expand Down
3 changes: 1 addition & 2 deletions spec/design/m-skel/RISCV64/MachineTypes.thy
Original file line number Diff line number Diff line change
Expand Up @@ -10,8 +10,7 @@ theory MachineTypes
imports
Word_Lib.WordSetup
Monads.Nondet_Empty_Fail
Monads.Nondet_No_Fail
Monads.Reader_Option_ND
Monads.Nondet_Reader_Option
Lib.HaskellLib_H
Platform
begin
Expand Down
3 changes: 1 addition & 2 deletions spec/design/m-skel/X64/MachineTypes.thy
Original file line number Diff line number Diff line change
Expand Up @@ -10,8 +10,7 @@ theory MachineTypes
imports
Word_Lib.WordSetup
Monads.Nondet_Empty_Fail
Monads.Nondet_No_Fail
Monads.Reader_Option_ND
Monads.Nondet_Reader_Option
Lib.HaskellLib_H
Platform
begin
Expand Down
4 changes: 2 additions & 2 deletions tools/autocorres/NonDetMonadEx.thy
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,7 @@ imports
"Monads.Nondet_More_VCG"
"Monads.Nondet_No_Throw"
"Monads.Nondet_No_Fail"
"Monads.Reader_Option_ND"
"Monads.Nondet_Reader_Option"
begin

(*
Expand Down Expand Up @@ -276,7 +276,7 @@ lemma whileLoop_to_fold:
(\<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"
(is "?LHS s = return (?RHS x) s")
apply (subst Reader_Option_ND.gets_the_return [symmetric])
apply (subst gets_the_return [symmetric])
apply (subst gets_the_whileLoop)
apply (rule gets_the_to_return)
apply (subst owhile_to_fold)
Expand Down
1 change: 0 additions & 1 deletion tools/autocorres/TypeStrengthen.thy
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,6 @@
theory TypeStrengthen
imports
L2Defs
"Monads.Reader_Option_ND"
ExecConcrete
begin

Expand Down

0 comments on commit cf75dfb

Please sign in to comment.