author | wenzelm |
Mon, 29 Nov 1999 15:52:49 +0100 | |
changeset 8039 | a901bafe4578 |
parent 2907 | 0e272e4c7cb2 |
permissions | -rw-r--r-- |
1247 | 1 |
(* Title: HOL/AxClasses/Tutorial/Sigs.thy |
2 |
ID: $Id$ |
|
3 |
Author: Markus Wenzel, TU Muenchen |
|
4 |
||
5 |
Some polymorphic constants for the 'signature' parts of axclasses. |
|
6 |
*) |
|
7 |
||
8 |
Sigs = HOL + |
|
9 |
||
10 |
consts |
|
11 |
"<*>" :: "['a, 'a] => 'a" (infixl 70) |
|
2907 | 12 |
inverse :: "'a => 'a" |
1247 | 13 |
"1" :: "'a" ("1") |
14 |
||
15 |
end |