| author | wenzelm |
| Thu, 03 Aug 2000 19:28:37 +0200 | |
| changeset 9516 | 72b5d28aae58 |
| parent 9102 | c7ba07e3bbe8 |
| child 9771 | 54c6a2c6e569 |
| permissions | -rw-r--r-- |
| 5261 | 1 |
(* Title: HOL/Lambda/ListApplication.thy |
2 |
ID: $Id$ |
|
3 |
Author: Tobias Nipkow |
|
4 |
Copyright 1998 TU Muenchen |
|
5 |
||
6 |
Application of a term to a list of terms |
|
7 |
*) |
|
8 |
||
| 9102 | 9 |
ListApplication = Lambda + |
| 5261 | 10 |
|
11 |
syntax "$$" :: dB => dB list => dB (infixl 150) |
|
12 |
translations "t $$ ts" == "foldl op$ t ts" |
|
13 |
||
14 |
end |