author | wenzelm |
Tue, 24 Jul 2012 23:01:55 +0200 | |
changeset 48494 | 00eb5be9e76b |
parent 46950 | d0181abdbdac |
child 48644 | 70a5d78e8326 |
permissions | -rw-r--r-- |
41582
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
1 |
(* Title: HOL/ex/Interpretation_with_Defs.thy |
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
2 |
Author: Florian Haftmann, TU Muenchen |
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
3 |
*) |
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
4 |
|
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
5 |
header {* Interpretation accompanied with mixin definitions. EXPERIMENTAL. *} |
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
6 |
|
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
7 |
theory Interpretation_with_Defs |
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
8 |
imports Pure |
46950
d0181abdbdac
declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents:
41582
diff
changeset
|
9 |
keywords "interpretation" :: thy_goal |
41582
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
10 |
uses "~~/src/Tools/interpretation_with_defs.ML" |
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
11 |
begin |
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
12 |
|
c34415351b6d
experimental variant of interpretation with simultaneous definitions, plus example
haftmann
parents:
diff
changeset
|
13 |
end |