| author | urbanc |
| Wed, 11 Jan 2006 17:10:11 +0100 | |
| changeset 18655 | 73cebafb9a89 |
| parent 17244 | 0b2ff9541727 |
| child 19740 | 6b38551d0798 |
| permissions | -rw-r--r-- |
(* Title: HOLCF/IOA/ABP/Action.thy ID: $Id$ Author: Olaf Müller *) header {* The set of all actions of the system *} theory Action imports Main begin datatype action = New | Loc nat | Free nat lemma [cong]: "!!x. x = y ==> action_case a b c x = action_case a b c y" by simp ML {* use_legacy_bindings (the_context ()) *} end