author | wenzelm |
Wed, 09 Apr 2014 16:22:06 +0200 | |
changeset 56497 | 0c63f3538639 |
parent 55601 | b7f4da504b75 |
child 58889 | 5b7a9633cfa8 |
permissions | -rw-r--r-- |
(* Title: Tools/Permanent_Interpretation.thy Author: Florian Haftmann, TU Muenchen *) header {* Permanent interpretation accompanied with mixin definitions. *} theory Permanent_Interpretation imports Pure keywords "defining" and "permanent_interpretation" :: thy_goal begin ML_file "~~/src/Tools/permanent_interpretation.ML" end