File tree 16 files changed +34
-34
lines changed
16 files changed +34
-34
lines changed Original file line number Diff line number Diff line change @@ -2812,10 +2812,10 @@ lemma ctes_of_ex_cte_cap_to':
2812
2812
2813
2813
2814
2814
lemma Arch_isFrameType_spec :
2815
- "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::ArchTypes_H. object_type)\<rbrace>
2815
+ "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::object_type)\<rbrace>
2816
2816
Call Arch_isFrameType_'proc
2817
2817
\<lbrace> \<acute>ret__unsigned_long =
2818
- from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::ArchTypes_H. object_type))\<rbrace>"
2818
+ from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::object_type))\<rbrace>"
2819
2819
apply vcg
2820
2820
apply ( simp add : toEnum_object_type_to_H )
2821
2821
apply ( frule object_type_from_to_H )
Original file line number Diff line number Diff line change @@ -5047,7 +5047,7 @@ lemma placeNewObject_user_data:
5047
5047
done
5048
5048
5049
5049
definition
5050
- createObject_hs_preconds :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
5050
+ createObject_hs_preconds :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
5051
5051
where
5052
5052
"createObject_hs_preconds regionBase newType userSize d \<equiv>
5053
5053
(invs' and pspace_no_overlap' regionBase (getObjectSize newType userSize)
@@ -5070,14 +5070,14 @@ abbreviation
5070
5070
5071
5071
(* these preconds actually used throughout the proof *)
5072
5072
abbreviation ( input )
5073
- createObject_c_preconds1 :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
5073
+ createObject_c_preconds1 :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
5074
5074
where
5075
5075
"createObject_c_preconds1 regionBase newType userSize deviceMemory \<equiv>
5076
5076
{s. region_actually_is_dev_bytes regionBase (2 ^ getObjectSize newType userSize) deviceMemory s}"
5077
5077
5078
5078
(* these preconds used at start of proof *)
5079
5079
definition
5080
- createObject_c_preconds :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
5080
+ createObject_c_preconds :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
5081
5081
where
5082
5082
"createObject_c_preconds regionBase newType userSize deviceMemory \<equiv>
5083
5083
(createObject_c_preconds1 regionBase newType userSize deviceMemory
Original file line number Diff line number Diff line change @@ -2623,10 +2623,10 @@ lemma ctes_of_ex_cte_cap_to':
2623
2623
2624
2624
2625
2625
lemma Arch_isFrameType_spec :
2626
- "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::ArchTypes_H. object_type)\<rbrace>
2626
+ "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::object_type)\<rbrace>
2627
2627
Call Arch_isFrameType_'proc
2628
2628
\<lbrace> \<acute>ret__unsigned_long =
2629
- from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::ArchTypes_H. object_type))\<rbrace>"
2629
+ from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::object_type))\<rbrace>"
2630
2630
apply vcg
2631
2631
apply ( simp add : toEnum_object_type_to_H )
2632
2632
apply ( frule object_type_from_to_H )
Original file line number Diff line number Diff line change @@ -4350,7 +4350,7 @@ lemma placeNewObject_user_data:
4350
4350
4351
4351
4352
4352
definition
4353
- createObject_hs_preconds :: "word32 \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
4353
+ createObject_hs_preconds :: "word32 \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
4354
4354
where
4355
4355
"createObject_hs_preconds regionBase newType userSize d \<equiv>
4356
4356
(invs' and pspace_no_overlap' regionBase (getObjectSize newType userSize)
@@ -4373,14 +4373,14 @@ abbreviation
4373
4373
4374
4374
(* these preconds actually used throughout the proof *)
4375
4375
abbreviation ( input )
4376
- createObject_c_preconds1 :: "word32 \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4376
+ createObject_c_preconds1 :: "word32 \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4377
4377
where
4378
4378
"createObject_c_preconds1 regionBase newType userSize deviceMemory \<equiv>
4379
4379
{s. region_actually_is_dev_bytes regionBase (2 ^ getObjectSize newType userSize) deviceMemory s}"
4380
4380
4381
4381
(* these preconds used at start of proof *)
4382
4382
definition
4383
- createObject_c_preconds :: "word32 \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4383
+ createObject_c_preconds :: "word32 \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4384
4384
where
4385
4385
"createObject_c_preconds regionBase newType userSize deviceMemory \<equiv>
4386
4386
(createObject_c_preconds1 regionBase newType userSize deviceMemory
Original file line number Diff line number Diff line change @@ -2828,10 +2828,10 @@ lemma ctes_of_ex_cte_cap_to':
2828
2828
2829
2829
2830
2830
lemma Arch_isFrameType_spec :
2831
- "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::ArchTypes_H. object_type)\<rbrace>
2831
+ "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::object_type)\<rbrace>
2832
2832
Call Arch_isFrameType_'proc
2833
2833
\<lbrace> \<acute>ret__unsigned_long =
2834
- from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::ArchTypes_H. object_type))\<rbrace>"
2834
+ from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::object_type))\<rbrace>"
2835
2835
apply vcg
2836
2836
apply ( simp add : toEnum_object_type_to_H )
2837
2837
apply ( frule object_type_from_to_H )
Original file line number Diff line number Diff line change @@ -4919,7 +4919,7 @@ lemma placeNewObject_user_data:
4919
4919
4920
4920
4921
4921
definition
4922
- createObject_hs_preconds :: "word32 \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
4922
+ createObject_hs_preconds :: "word32 \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
4923
4923
where
4924
4924
"createObject_hs_preconds regionBase newType userSize d \<equiv>
4925
4925
(invs' and pspace_no_overlap' regionBase (getObjectSize newType userSize)
@@ -4942,14 +4942,14 @@ abbreviation
4942
4942
4943
4943
(* these preconds actually used throughout the proof *)
4944
4944
abbreviation ( input )
4945
- createObject_c_preconds1 :: "word32 \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4945
+ createObject_c_preconds1 :: "word32 \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4946
4946
where
4947
4947
"createObject_c_preconds1 regionBase newType userSize deviceMemory \<equiv>
4948
4948
{s. region_actually_is_dev_bytes regionBase (2 ^ getObjectSize newType userSize) deviceMemory s}"
4949
4949
4950
4950
(* these preconds used at start of proof *)
4951
4951
definition
4952
- createObject_c_preconds :: "word32 \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4952
+ createObject_c_preconds :: "word32 \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4953
4953
where
4954
4954
"createObject_c_preconds regionBase newType userSize deviceMemory \<equiv>
4955
4955
(createObject_c_preconds1 regionBase newType userSize deviceMemory
Original file line number Diff line number Diff line change @@ -2774,10 +2774,10 @@ lemma ctes_of_ex_cte_cap_to':
2774
2774
2775
2775
2776
2776
lemma Arch_isFrameType_spec :
2777
- "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::ArchTypes_H. object_type)\<rbrace>
2777
+ "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::object_type)\<rbrace>
2778
2778
Call Arch_isFrameType_'proc
2779
2779
\<lbrace> \<acute>ret__unsigned_long =
2780
- from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::ArchTypes_H. object_type))\<rbrace>"
2780
+ from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::object_type))\<rbrace>"
2781
2781
apply vcg
2782
2782
apply ( simp add : toEnum_object_type_to_H )
2783
2783
apply ( frule object_type_from_to_H )
Original file line number Diff line number Diff line change @@ -4796,7 +4796,7 @@ lemma placeNewObject_user_data:
4796
4796
done
4797
4797
4798
4798
definition
4799
- createObject_hs_preconds :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
4799
+ createObject_hs_preconds :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
4800
4800
where
4801
4801
"createObject_hs_preconds regionBase newType userSize d \<equiv>
4802
4802
(invs' and pspace_no_overlap' regionBase (getObjectSize newType userSize)
@@ -4819,14 +4819,14 @@ abbreviation
4819
4819
4820
4820
(* these preconds actually used throughout the proof *)
4821
4821
abbreviation ( input )
4822
- createObject_c_preconds1 :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4822
+ createObject_c_preconds1 :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4823
4823
where
4824
4824
"createObject_c_preconds1 regionBase newType userSize deviceMemory \<equiv>
4825
4825
{s. region_actually_is_dev_bytes regionBase (2 ^ getObjectSize newType userSize) deviceMemory s}"
4826
4826
4827
4827
(* these preconds used at start of proof *)
4828
4828
definition
4829
- createObject_c_preconds :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4829
+ createObject_c_preconds :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
4830
4830
where
4831
4831
"createObject_c_preconds regionBase newType userSize deviceMemory \<equiv>
4832
4832
(createObject_c_preconds1 regionBase newType userSize deviceMemory
Original file line number Diff line number Diff line change @@ -2800,10 +2800,10 @@ lemma ctes_of_ex_cte_cap_to':
2800
2800
2801
2801
2802
2802
lemma Arch_isFrameType_spec :
2803
- "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::ArchTypes_H. object_type)\<rbrace>
2803
+ "\<forall>s. \<Gamma> \<turnstile> \<lbrace>s. unat \<acute>type \<le> fromEnum (maxBound::object_type)\<rbrace>
2804
2804
Call Arch_isFrameType_'proc
2805
2805
\<lbrace> \<acute>ret__unsigned_long =
2806
- from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::ArchTypes_H. object_type))\<rbrace>"
2806
+ from_bool (isFrameType ((toEnum (unat \<^bsup>s\<^esup> type))::object_type))\<rbrace>"
2807
2807
apply vcg
2808
2808
apply ( simp add : toEnum_object_type_to_H )
2809
2809
apply ( frule object_type_from_to_H )
Original file line number Diff line number Diff line change @@ -5628,7 +5628,7 @@ lemma placeNewObject_user_data:
5628
5628
done
5629
5629
5630
5630
definition
5631
- createObject_hs_preconds :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
5631
+ createObject_hs_preconds :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> kernel_state \<Rightarrow> bool"
5632
5632
where
5633
5633
"createObject_hs_preconds regionBase newType userSize d \<equiv>
5634
5634
(invs' and pspace_no_overlap' regionBase (getObjectSize newType userSize)
@@ -5651,14 +5651,14 @@ abbreviation
5651
5651
5652
5652
(* these preconds actually used throughout the proof *)
5653
5653
abbreviation ( input )
5654
- createObject_c_preconds1 :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
5654
+ createObject_c_preconds1 :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
5655
5655
where
5656
5656
"createObject_c_preconds1 regionBase newType userSize deviceMemory \<equiv>
5657
5657
{s. region_actually_is_dev_bytes regionBase (2 ^ getObjectSize newType userSize) deviceMemory s}"
5658
5658
5659
5659
(* these preconds used at start of proof *)
5660
5660
definition
5661
- createObject_c_preconds :: "machine_word \<Rightarrow> ArchTypes_H. object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
5661
+ createObject_c_preconds :: "machine_word \<Rightarrow> object_type \<Rightarrow> nat \<Rightarrow> bool \<Rightarrow> (globals myvars) set"
5662
5662
where
5663
5663
"createObject_c_preconds regionBase newType userSize deviceMemory \<equiv>
5664
5664
(createObject_c_preconds1 regionBase newType userSize deviceMemory
Original file line number Diff line number Diff line change @@ -535,7 +535,7 @@ crunch InterruptDecls_H.invokeIRQHandler
535
535
for typ_at' [ wp ]: "\<lambda>s. P (typ_at' T p s)"
536
536
537
537
lemmas invokeIRQHandler_typ_ats [ wp ] =
538
- typ_at_lifts [ OF InterruptDecls_H_invokeIRQHandler_typ_at ']
538
+ typ_at_lifts [ OF invokeIRQHandler_typ_at ']
539
539
540
540
crunch setDomain
541
541
for tcb_at' [ wp ]: "tcb_at' tptr"
Original file line number Diff line number Diff line change @@ -526,7 +526,7 @@ crunch InterruptDecls_H.invokeIRQHandler
526
526
for typ_at' [ wp ]: "\<lambda>s. P (typ_at' T p s)"
527
527
528
528
lemmas invokeIRQHandler_typ_ats [ wp ] =
529
- typ_at_lifts [ OF InterruptDecls_H_invokeIRQHandler_typ_at ']
529
+ typ_at_lifts [ OF invokeIRQHandler_typ_at ']
530
530
531
531
crunch setDomain
532
532
for tcb_at' [ wp ]: "tcb_at' tptr"
Original file line number Diff line number Diff line change @@ -1797,11 +1797,11 @@ lemma invokeIRQControl_no_orphans [wp]:
1797
1797
apply ( wp | clarsimp )+
1798
1798
done
1799
1799
1800
- lemma invokeIRQHandler_no_orphans [ wp ]:
1800
+ lemma arch_invokeIRQHandler_no_orphans [ wp ]:
1801
1801
"\<lbrace> \<lambda>s. no_orphans s \<and> invs' s \<rbrace>
1802
- invokeIRQHandler i
1802
+ ARM_H. invokeIRQHandler i
1803
1803
\<lbrace> \<lambda>reply s. no_orphans s \<rbrace>"
1804
- apply ( cases i , simp_all add : invokeIRQHandler_def )
1804
+ apply ( cases i , simp_all add : ARM_H. invokeIRQHandler_def)
1805
1805
apply ( wp | clarsimp | fastforce )+
1806
1806
done
1807
1807
@@ -1939,7 +1939,7 @@ lemma setDomain_no_orphans [wp]:
1939
1939
apply ( fastforce simp : tcb_at_typ_at' is_active_tcb_ptr_runnable' )
1940
1940
done
1941
1941
1942
- crunch InterruptDecls_H. invokeIRQHandler
1942
+ crunch invokeIRQHandler
1943
1943
for no_orphans [ wp ]: no_orphans
1944
1944
1945
1945
lemma performInvocation_no_orphans [ wp ]:
Original file line number Diff line number Diff line change @@ -536,7 +536,7 @@ crunch InterruptDecls_H.invokeIRQHandler
536
536
for typ_at'[wp]: "\<lambda>s. P (typ_at' T p s)"
537
537
538
538
lemmas invokeIRQHandler_typ_ats[wp] =
539
- typ_at_lifts [OF InterruptDecls_H_invokeIRQHandler_typ_at ']
539
+ typ_at_lifts [OF invokeIRQHandler_typ_at ']
540
540
541
541
crunch setDomain
542
542
for tcb_at'[wp]: "tcb_at' tptr"
Original file line number Diff line number Diff line change @@ -534,7 +534,7 @@ crunch InterruptDecls_H.invokeIRQHandler
534
534
for typ_at'[wp]: "\<lambda>s. P (typ_at' T p s)"
535
535
536
536
lemmas invokeIRQHandler_typ_ats[wp] =
537
- typ_at_lifts [OF InterruptDecls_H_invokeIRQHandler_typ_at ']
537
+ typ_at_lifts [OF invokeIRQHandler_typ_at ']
538
538
539
539
crunch setDomain
540
540
for tcb_at'[wp]: "tcb_at' tptr"
Original file line number Diff line number Diff line change @@ -535,7 +535,7 @@ crunch InterruptDecls_H.invokeIRQHandler
535
535
for typ_at'[wp]: "\<lambda>s. P (typ_at' T p s)"
536
536
537
537
lemmas invokeIRQHandler_typ_ats[wp] =
538
- typ_at_lifts [OF InterruptDecls_H_invokeIRQHandler_typ_at ']
538
+ typ_at_lifts [OF invokeIRQHandler_typ_at ']
539
539
540
540
crunch setDomain
541
541
for tcb_at'[wp]: "tcb_at' tptr"
You can’t perform that action at this time.
0 commit comments