Added tag Isabelle2014-RC4 for changeset 113b43b84412
(* Title: HOL/HOLCF/IOA/ABP/Action.thy Author: Olaf Müller*)header {* The set of all actions of the system *}theory Actionimports Packetbegindatatype 'm action = Next | S_msg 'm | R_msg 'm | S_pkt "'m packet" | R_pkt "'m packet" | S_ack bool | R_ack boolend