lh-l4v/proof/sep-capDL/AbstractSeparationHelpers_S...

26 lines
447 B
Plaintext

(*
* Copyright 2014, NICTA
*
* This software may be distributed and modified according to the terms of
* the GNU General Public License version 2. Note that NO WARRANTY is provided.
* See "LICENSE_GPLv2.txt" for details.
*
* @TAG(NICTA_GPL)
*)
theory AbstractSeparationHelpers_SD
imports
"Sep_Algebra.Sep_Algebra_L4v"
begin
(*
* Lemmas that should be moved into the abstract separation logic.
*)
context sep_algebra
begin
end
end