| author | paulson |
| Sun, 23 Jun 2002 10:14:13 +0200 | |
| changeset 13240 | bb5f4faea1f3 |
| parent 12218 | 6597093b77e7 |
| child 14981 | e73f8140af78 |
| permissions | -rw-r--r-- |
| 6008 | 1 |
(* Title: HOL/IOA/example/Sender.thy |
2 |
ID: $Id$ |
|
| 12218 | 3 |
Author: Olaf Müller |
4 |
License: GPL (GNU GENERAL PUBLIC LICENSE) |
|
| 6008 | 5 |
|
| 12218 | 6 |
Impl. |
| 6008 | 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"; |