src/Doc/IsarImplementation/Base.thy
author blanchet
Wed, 12 Feb 2014 08:37:06 +0100
changeset 55417 01fbfb60c33e
parent 48985 5386df44a037
child 56059 2390391584c2
permissions -rw-r--r--
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems * * * more transition of 'xxx_rec' to 'rec_xxx' and same for case * * * compile * * * 'rename_tac's to avoid referring to generated names * * * more robust scripts with 'rename_tac' * * * 'where' -> 'of' * * * 'where' -> 'of' * * * renamed 'xxx_rec' to 'rec_xxx'

theory Base
imports Main
begin

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

end