src/ZF/Arith.thy
changeset 9654 9754ba005b64
parent 9492 72e429c66608
child 9683 f87c8c449018
--- a/src/ZF/Arith.thy	Fri Aug 18 18:11:10 2000 +0200
+++ b/src/ZF/Arith.thy	Fri Aug 18 18:46:02 2000 +0200
@@ -1,4 +1,4 @@
-(*  Title:      ZF/arith.thy
+(*  Title:      ZF/Arith.thy
     ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1992  University of Cambridge
@@ -56,4 +56,7 @@
   mod  :: [i,i]=>i                    (infixl "mod" 70)
     "m mod n == raw_mod (natify(m), natify(n))"
 
+syntax (symbols)
+  "mult"      :: [i, i] => i               (infixr "#\\<times>" 70)
+
 end