Neue commands, import RegExp, …

This commit is contained in:
Burkhart Wolff 2018-05-14 15:47:16 +02:00
parent 93bad550ef
commit 2acc4ea222
2 changed files with 9 additions and 6 deletions

View File

@ -11,6 +11,7 @@ that provide direct support in the PIDE framework. *}
theory Isa_DOF (* Isabelle Document Ontology Framework *)
imports Main (* Isa_MOF *)
RegExp
Assert
keywords "+=" ":="
and "section*" "subsection*" "subsubsection*"
@ -19,7 +20,7 @@ theory Isa_DOF (* Isabelle Document Ontology Framework *)
and "open_monitor*" "close_monitor*" "declare_reference*"
"update_instance*" "doc_class" ::thy_decl
and "lemma*" ::thy_decl
and "lemma*" "assert*"::thy_decl
begin
@ -553,6 +554,11 @@ val _ =
"close a document reference monitor"
(attributes >> (fn (((oid,pos),cid),doc_attrs) =>
(Toplevel.theory (I)))); (* dummy/fake so far *)
val _ =
Outer_Syntax.command @{command_keyword "assert*"}
"close a document reference monitor"
(attributes >> (fn (((oid,pos),cid),doc_attrs) =>
(Toplevel.theory (I)))); (* dummy/fake so far *)
val _ =
Outer_Syntax.command @{command_keyword "update_instance*"}
@ -563,7 +569,6 @@ end (* struct *)
*}
lemma murx : "XXX" sorry
section{* Syntax for Ontological Antiquotations (the '' View'' Part II) *}

View File

@ -10,13 +10,11 @@ Common Criteria identifies:
order of category instances in the overall document as a regular language)
*}
text_raw{*\snip{appendix.tex}{1}{1}{%*}
(*<<*)
theory CENELEC_50126
imports "../Isa_DOF"
begin
text_raw{*}%endsnip*}
(*>>*)
text{* Excerpt of the BE EN 50128:2011 *}