(* Title: HOLCF/IOA/ABP/Action.thy ID: $Id$ Author: Olaf Müller*)header {* The set of all actions of the system *}theory Actionimports Mainbegindatatype action = New | Loc nat | Free natlemma [cong]: "!!x. x = y ==> action_case a b c x = action_case a b c y" by simpend