Isabelle_DOF/examples/conceptual/InnerSyntaxAntiquotations.thy

23 lines
590 B
Plaintext
Raw Normal View History

theory InnerSyntaxAntiquotations
imports "../../ontologies/Conceptual"
begin
ML\<open>
val ({tab = x, ...},y,z)= DOF_core.get_data @{context};
Symtab.dest z;
\<close>
lemma murks : "T = {ert,dfg}" sorry
text*[xcv::F, u="@{file ''./examples/conceptual/Attributes.thy''}"]\<open>Lorem ipsum ...\<close>
text*[xcv1::F, r="[@{thm ''HOL.refl''},
@{thm ''InnerSyntaxAntiquotations.murks''}]",
b="{(@{docitem ''xcv''},@{docitem ''xcv''})}", (* lamentable ! No typecheck.*)
s="[@{typ ''int list''}]"]\<open>Lorem ipsum ...\<close>
2018-09-11 10:08:25 +00:00
end