author | wenzelm |
Wed, 12 Aug 2015 13:53:51 +0200 | |
changeset 60916 | a6e2a667b0a8 |
parent 58889 | 5b7a9633cfa8 |
permissions | -rw-r--r-- |
(* Title: Tools/Permanent_Interpretation.thy Author: Florian Haftmann, TU Muenchen *) section {* 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