src/HOL/HOL.thy
changeset 13456 42601eb7553f
parent 13438 527811f00c56
child 13550 5a176b8dda84
--- a/src/HOL/HOL.thy	Mon Aug 05 14:35:33 2002 +0200
+++ b/src/HOL/HOL.thy	Mon Aug 05 21:16:36 2002 +0200
@@ -163,6 +163,11 @@
   uminus        :: "['a::minus] => 'a"              ("- _" [81] 80)
   *             :: "['a::times, 'a] => 'a"          (infixl 70)
 
+syntax
+  "_index1"  :: index    ("\<^sub>1")
+translations
+  (index) "\<^sub>1" == "_index 1"
+
 local
 
 typed_print_translation {*