| author | wenzelm |
| Thu, 17 May 2012 15:23:00 +0200 | |
| changeset 47881 | 45a3a1c320d8 |
| parent 46950 | d0181abdbdac |
| child 48644 | 70a5d78e8326 |
| permissions | -rw-r--r-- |
(* Title: HOL/ex/Interpretation_with_Defs.thy Author: Florian Haftmann, TU Muenchen *) header {* Interpretation accompanied with mixin definitions. EXPERIMENTAL. *} theory Interpretation_with_Defs imports Pure keywords "interpretation" :: thy_goal uses "~~/src/Tools/interpretation_with_defs.ML" begin end