Checked style.

This commit is contained in:
Achim D. Brucker 2016-12-28 00:01:00 +00:00
parent 61cdc4efcf
commit 1ab1f96579
7 changed files with 81 additions and 100 deletions

View File

@ -39,7 +39,7 @@ subsection {* The File Transfer Prototol (ftp) *}
theory
FTP
imports
Stateful
StatefulCore
begin
subsubsection{* The protocol syntax *}
@ -213,28 +213,19 @@ definition
(is_ftp S0 s2 d2 i2 p2 (packet_with_id x i2))}"
lemma subnetOf_lemma: "(a::int) \<noteq> (c::int) \<Longrightarrow> \<forall>x\<in>subnet_of (a, b::port). (c, d) \<notin> x"
apply (rule ballI)
apply (simp add: subnet_of_int_def)
done
by (rule ballI, simp add: subnet_of_int_def)
lemma subnetOf_lemma2: " \<forall>x\<in>subnet_of (a::int, b::port). (a, b) \<in> x"
apply (rule ballI)
apply (simp add: subnet_of_int_def)
done
by (rule ballI, simp add: subnet_of_int_def)
lemma subnetOf_lemma3: "(\<exists>x. x \<in> subnet_of (a::int, b::port))"
apply (rule exI)
apply (simp add: subnet_of_int_def)
done
by (rule exI, simp add: subnet_of_int_def)
lemma subnetOf_lemma4: "\<exists>x\<in>subnet_of (a::int, b::port). (a, c::port) \<in> x"
apply (rule bexI)
apply (simp_all add: subnet_of_int_def)
done
by (rule bexI, simp_all add: subnet_of_int_def)
lemma port_open_lemma: "\<not> (Ex (port_open [] (x::port)))"
apply (simp add: port_open_def)
done
by (simp add: port_open_def)
lemmas FTPLemmas = TRPolicy_def applyPolicy_def policy2MON_def
Let_def in_subnet_def src_def
@ -245,4 +236,3 @@ lemmas FTPLemmas = TRPolicy_def applyPolicy_def policy2MON_def
NetworkCore.id_def adr\<^sub>i\<^sub>pLemmas port_open_lemma
bind_SE_def unit_SE_def valid_SE_def
end

View File

@ -73,5 +73,3 @@ where
then Some (allow (POL (snd x)),((fst x),snd x))
else Some (deny (POL (snd x)),(fst x,snd x)))"
end

View File

@ -36,8 +36,10 @@
*****************************************************************************)
subsection {* Termporal Combinators *}
theory LTL_alike
imports Main
theory
LTL_alike
imports
Main
begin
text{*

View File

@ -37,7 +37,7 @@
section {* Stateful Protocols *}
theory
Stateful
StatefulCore
imports
"../PacketFilter/PacketFilter"
LTL_alike
@ -74,7 +74,7 @@ type_synonym ('\<alpha>,'\<beta>,'\<gamma>) FWState = "'\<alpha> \<times> (('\<b
text{* Having a state, we need of course some state transitions. Such
a transition can happen every time a new packet arrives. State
transitions can be modelled using a state-exception monad.
We provide two types of firewall monads: one *}
*}
type_synonym ('\<alpha>,'\<beta>,'\<gamma>) FWStateTransitionP =

View File

@ -37,7 +37,7 @@
subsection {* A simple voice-over-ip model *}
theory VOIP
imports Stateful
imports StatefulCore
begin
text{*
@ -59,13 +59,6 @@ text{*
\item Calls can be initiated from outside the firewall.
\end{itemize}
% \begin{figure}
% \centering
% \includegraphics[scale=0.4]{voip}
% \caption {The modelled VoIP-Protocol}
% \label{voip}
% \end{figure}
Again we only consider a simplified VoIP scenario with the following
seven messages which are grouped into four subprotocols (see Figure
\ref{voip}):
@ -273,8 +266,6 @@ text{*
*}
datatype voip_states = S0 | S1 | S2 | S3 | S4 | S5
text{*
The constant @{text "is_voip"} checks if a trace corresponds to a
legal VoIP protocol, given the IP-addresses of the three entities,