thys/Paper/Paper.thy
changeset 165 ca4dcfd912cb
parent 162 aa4fdba769ea
child 169 072a701bb153
equal deleted inserted replaced
164:15294ac95e47 165:ca4dcfd912cb
   855   @{term "simp_SEQ (r\<^sub>1, f\<^sub>1) (r\<^sub>2, f\<^sub>2)"} & $\dn$ & @{term "(SEQ r\<^sub>1 r\<^sub>2, F_SEQ f\<^sub>1 f\<^sub>2)"}\\
   855   @{term "simp_SEQ (r\<^sub>1, f\<^sub>1) (r\<^sub>2, f\<^sub>2)"} & $\dn$ & @{term "(SEQ r\<^sub>1 r\<^sub>2, F_SEQ f\<^sub>1 f\<^sub>2)"}\\
   856   \end{tabular}
   856   \end{tabular}
   857   \end{center}
   857   \end{center}
   858 
   858 
   859   \noindent
   859   \noindent
   860   The functions @{text "simp\<^bsub>ALT\<^esub>"} and @{text "simp\<^bsub>SEQ\<^esub>"} encode the simplification rules
   860   The functions @{text "simp\<^bsub>Alt\<^esub>"} and @{text "simp\<^bsub>Seq\<^esub>"} encode the simplification rules
   861   and compose the rectification functions. The main simplification function is then 
   861   and compose the rectification functions. The main simplification function is then 
   862 
   862 
   863   \begin{center}
   863   \begin{center}
   864   \begin{tabular}{lcl}
   864   \begin{tabular}{lcl}
   865   @{term "simp (ALT r\<^sub>1 r\<^sub>2)"} & $\dn$ & @{term "simp_ALT (simp r\<^sub>1) (simp r\<^sub>2)"}\\
   865   @{term "simp (ALT r\<^sub>1 r\<^sub>2)"} & $\dn$ & @{term "simp_ALT (simp r\<^sub>1) (simp r\<^sub>2)"}\\