src/HOLCF/IOA/Storage/Impl.ML
author kleing
Tue, 13 May 2003 08:59:21 +0200
changeset 14024 213dcc39358f
parent 12218 6597093b77e7
child 14981 e73f8140af78
permissions -rw-r--r--
HOL-Real -> HOL-Complex

(*  Title:      HOL/IOA/example/Sender.thy
    ID:         $Id$
    Author:     Olaf Müller
    License:    GPL (GNU GENERAL PUBLIC LICENSE)

Impl.
*)
 
Goal 
 "New : actions(impl_sig)       &   \
\ Loc l : actions(impl_sig)       &   \
\ Free l : actions(impl_sig) ";
by (simp_tac (simpset() addsimps 
             (Impl.sig_def :: actions_def :: 
              asig_projections)) 1);
qed "in_impl_asig";