| author | wenzelm |
| Fri, 10 Nov 2000 19:11:51 +0100 | |
| changeset 10443 | 0a68dc9edba5 |
| parent 7322 | d16d7ddcc842 |
| child 12218 | 6597093b77e7 |
| permissions | -rw-r--r-- |
| 6008 | 1 |
(* Title: HOL/IOA/example/Sender.thy |
2 |
ID: $Id$ |
|
3 |
Author: Olaf Mueller |
|
4 |
Copyright 1997 TU Muenchen |
|
5 |
||
6 |
Impl |
|
7 |
*) |
|
8 |
||
9 |
Goal |
|
10 |
"New : actions(impl_sig) & \ |
|
11 |
\ Loc l : actions(impl_sig) & \ |
|
12 |
\ Free l : actions(impl_sig) "; |
|
| 7322 | 13 |
by (simp_tac (simpset() addsimps |
| 6008 | 14 |
(Impl.sig_def :: actions_def :: |
15 |
asig_projections)) 1); |
|
16 |
qed "in_impl_asig"; |