src/HOL/Library/Structure_Syntax.thy
author haftmann
Mon, 08 Feb 2010 10:36:02 +0100
changeset 35029 22aab1c5e5a8
permissions -rw-r--r--
separate theory for index structures

(* Author: Florian Haftmann, TU Muenchen *)

header {* Index syntax for structures *}

theory Structure_Syntax
imports Pure
begin

syntax
  "_index1"  :: index    ("\<^sub>1")
translations
  (index) "\<^sub>1" => (index) "\<^bsub>\<struct>\<^esub>"

end