doc-src/IsarImplementation/Thy/Syntax.thy
author huffman
Fri, 12 Jun 2009 16:23:07 -0700
changeset 31590 776d6a4c1327
parent 30272 2d612824e642
child 34924 520727474bbe
permissions -rw-r--r--
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]

theory Syntax
imports Base
begin

chapter {* Syntax and type-checking *}

text FIXME

end