author | wenzelm |
Mon, 18 Aug 2014 12:17:31 +0200 | |
changeset 57978 | 8f4a332500e4 |
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