Fixed theory hierachy and includes.

This commit is contained in:
Achim D. Brucker 2017-01-02 13:16:48 +00:00
parent 17f828902e
commit dcc46bdad0
3 changed files with 6 additions and 5 deletions

View File

@ -35,7 +35,7 @@
* OF THIS SOFTWARE, EVEN IF ADVISED OF THE POSSIBILITY OF SUCH DAMAGE.
*****************************************************************************)
section {* Stateful Protocols *}
subsection {* Stateful Protocols: Foundations *}
theory
StatefulCore
imports
@ -103,4 +103,4 @@ fun ids where
definition applyPolicy:: "('i \<times> ('i \<mapsto> 'o)) \<mapsto> 'o"
where "applyPolicy = (\<lambda> (x,z). z x)"
end
end

View File

@ -35,10 +35,10 @@
* OF THIS SOFTWARE, EVEN IF ADVISED OF THE POSSIBILITY OF SUCH DAMAGE.
*****************************************************************************)
subsection {* Stateful Network Protocols *}
section {* Stateful Network Protocols *}
theory
StatefulFW
imports
FTPVOIP
begin
end
end

View File

@ -120,7 +120,8 @@
\input{NormalisationGenericProofs.tex}
\input{NormalisationIntegerPortProof.tex}
\input{NormalisationIPPProofs.tex}
\input{Stateful}
\input{StatefulFW}
\input{StatefulCore}
\input{FTP}
\input{FTP_WithPolicy}
\input{VOIP}