src/Doc/IsarImplementation/Base.thy
author wenzelm
Wed, 05 Mar 2014 18:26:35 +0100
changeset 55922 710bc66f432c
parent 48985 5386df44a037
child 56059 2390391584c2
permissions -rw-r--r--
more markup for inner syntax class/type names (notably for completion); explicit reports result without broadcast yet, which is important for brute-force disambiguation;

theory Base
imports Main
begin

ML_file "../antiquote_setup.ML"
setup {* Antiquote_Setup.setup *}

end