lib+proof+tools: move LemmaBucket_C into CParser

Signed-off-by: Gerwin Klein <gerwin.klein@proofcraft.systems>
This commit is contained in:
Gerwin Klein 2023-01-24 14:55:01 +11:00
parent cb34fc3c4c
commit 2d2cadb86b
No known key found for this signature in database
GPG Key ID: 20A847CE6AB7F5F3
12 changed files with 14 additions and 14 deletions

View File

@ -85,7 +85,6 @@ session CLib (lib) in clib = CParser +
Simpl_Rewrite
MonadicRewrite_C
CTranslationNICTA
LemmaBucket_C
SIMPL_Lemmas
SimplRewrite
BitFieldProofsLib

View File

@ -11,9 +11,9 @@
theory Corres_UL_C
imports
"LemmaBucket_C"
"Lib.LemmaBucket"
"SIMPL_Lemmas"
CParser.LemmaBucket_C
Lib.LemmaBucket
SIMPL_Lemmas
begin
declare word_neq_0_conv [simp del]

View File

@ -7,7 +7,7 @@
theory ShowTypes_Test
imports
Lib.ShowTypes
CLib.LemmaBucket_C
CParser.LemmaBucket_C
CParser.CTranslation
begin

View File

@ -8,7 +8,7 @@ theory CLevityCatch
imports
"CBaseRefine.Include_C"
ArchMove_C
"CLib.LemmaBucket_C"
"CParser.LemmaBucket_C"
"Lib.LemmaBucket"
begin

View File

@ -8,7 +8,7 @@ theory CLevityCatch
imports
"CBaseRefine.Include_C"
ArchMove_C
"CLib.LemmaBucket_C"
"CParser.LemmaBucket_C"
"Lib.LemmaBucket"
begin

View File

@ -8,7 +8,7 @@ theory CLevityCatch
imports
"CBaseRefine.Include_C"
ArchMove_C
"CLib.LemmaBucket_C"
"CParser.LemmaBucket_C"
"Lib.LemmaBucket"
begin

View File

@ -8,7 +8,7 @@ theory CLevityCatch
imports
"CBaseRefine.Include_C"
ArchMove_C
"CLib.LemmaBucket_C"
"CParser.LemmaBucket_C"
"Lib.LemmaBucket"
begin

View File

@ -7,7 +7,7 @@
theory FieldAccessors
imports
Lib.Lib
CLib.LemmaBucket_C
CParser.LemmaBucket_C
begin
lemma h_val_mono:

View File

@ -10,7 +10,7 @@ imports
TailrecPre
GraphLangLemmas
Lib.Lib
"CLib.LemmaBucket_C"
"CParser.LemmaBucket_C"
ExtraSpecs
begin

View File

@ -11,7 +11,7 @@ imports
L2Defs
ExecConcrete
AbstractArrays
"CLib.LemmaBucket_C"
"CParser.LemmaBucket_C"
begin
definition "L2Tcorres st A C = corresXF st (\<lambda>r _. r) (\<lambda>r _. r) \<top> A C"

View File

@ -7,7 +7,7 @@
theory LemmaBucket_C
imports
Basics.CLib
CParser.TypHeapLib
TypHeapLib
begin
lemma Ptr_not_null_pointer_not_zero: "(Ptr p \<noteq> NULL)=(p\<noteq>0)"

View File

@ -16,9 +16,10 @@ session CParser = "Simpl-VCG" +
sessions
"HOL-Library"
"ML_Utils"
"Basics"
directories
"umm_heap"
"umm_heap/$L4V_ARCH"
theories
"CTranslation"
"TypHeapLib"
"LemmaBucket_C"