author | Christian Urban <urbanc@in.tum.de> |
Fri, 21 Aug 2009 16:04:59 +0200 | |
changeset 319 | 6bce4acf7f2a |
child 321 | e450fa467e3f |
permissions | -rw-r--r-- |
theory Command imports Main begin ML {* let val do_nothing = Scan.succeed (LocalTheory.theory I) val kind = OuterKeyword.thy_goal in OuterSyntax.local_theory "foobar" "description of foobar" kind do_nothing end *} ML {* let val do_nothing = Scan.succeed (LocalTheory.theory I) val kind = OuterKeyword.thy_decl in OuterSyntax.local_theory "simple_induct" "description of foobar" kind do_nothing end *} end