src/HOL/AxClasses/Tutorial/Sigs.thy
changeset 1247 18b1441fb603
child 2907 0e272e4c7cb2
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/AxClasses/Tutorial/Sigs.thy	Fri Sep 01 14:27:36 1995 +0200
@@ -0,0 +1,15 @@
+(*  Title:      HOL/AxClasses/Tutorial/Sigs.thy
+    ID:         $Id$
+    Author:     Markus Wenzel, TU Muenchen
+
+Some polymorphic constants for the 'signature' parts of axclasses.
+*)
+
+Sigs = HOL +
+
+consts
+  "<*>"         :: "['a, 'a] => 'a"             (infixl 70)
+  "inv"         :: "'a => 'a"
+  "1"           :: "'a"                         ("1")
+
+end