Theory M_07_Implementation

(*************************************************************************
 * Copyright (C) 
 *               2019-2022 University of Exeter 
 *               2018-2022 University of Paris-Saclay
 *               2018      The University of Sheffield
 *
 * License:
 *   This program can be redistributed and/or modified under the terms
 *   of the 2-clause BSD-style license.
 *
 *   SPDX-License-Identifier: BSD-2-Clause
 *************************************************************************)

(*<*)
theory "M_07_Implementation"
  imports "M_06_RefMan"
begin           
(*>*)


chapter*[isadof_developers::text_section]‹Extending isadof
text‹
  In this chapter, we describe the basic implementation aspects of isadof, which is based on 
  the following design-decisions:
   the entire isadof is a ``pure add-on,'' ie, we deliberately resign to the possibility to 
    modify Isabelle itself,
   isadof has been organized as an AFP entry and a form of an Isabelle component that is
    compatible with this goal,
   we decided to make the markup-generation by itself to adapt it as well as possible to the 
    needs of tracking the linking in documents,
   isadof is deeply integrated into the Isabelle's IDE (PIDE) to give immediate feedback during 
    editing and other forms of document evolution.
›
text‹
  Semantic macros, as required by our document model, are called ‹document antiquotations›
  in the Isabelle literature~cite"wenzel:isabelle-isar:2020". While Isabelle's code-antiquotations 
  are an old concept going back to Lisp and having found via SML and OCaml their ways into modern 
  proof systems, special annotation syntax inside documentation comments have their roots in 
  documentation generators such as Javadoc. Their use, however, as a mechanism to embed 
  machine-checked ‹formal content› is usually very limited and also lacks 
  IDE support.
›

sectionisadof: A User-Defined Plugin in Isabelle/Isar›
text‹ 
  A plugin in Isabelle starts with defining the local data and registering it in the framework. As 
  mentioned before, contexts are structures with independent cells/compartments having three
  primitives boxed_sml‹init›,  boxed_sml‹extend› and  boxed_sml‹merge›. Technically this is done by 
  instantiating a functor  boxed_sml‹Theory_Data›, and the following fairly typical code-fragment 
  is drawn from isadof:

@{boxed_sml [display]
‹structure Onto_Classes = Theory_Data
  (
    type T =  onto_class Name_Space.table;
    val empty : T = Name_Space.empty_table onto_classN;
    fun merge data : T = Name_Space.merge_tables data;
  );›}
  where the table  boxed_sml‹Name_Space.table› manages
  the environment for class definitions (boxed_sml‹onto_class›), inducing the inheritance relation,
  using a boxed_sml‹Name_Space› table. Other tables capture, \eg, 
  the class instances, class invariants, inner-syntax antiquotations.
  Operations follow the MVC-pattern, where 
  Isabelle/Isar provides the controller part. A typical model operation has the type:

@{boxed_sml [display]
‹val opn :: <args_type> -> theory -> theory›}
  representing a transformation on system contexts. For example, the operation of defining a class
  in the context is presented as follows:

@{boxed_sml [display]
‹fun add_onto_class name onto_class thy =
    thy |> Onto_Classes.map
      (Name_Space.define (Context.Theory thy) true (name, onto_class) #> #2);
›}
  This code fragment uses operations from the library structure boxed_sml‹Name_Space›
  that were used to update the appropriate table for document objects in
  the plugin-local state.
  A name space manages a collection of long names, together with a mapping
  between partially qualified external names and fully qualified internal names
  (in both directions).
  It can also keep track of the declarations and updates position of objects,
  and then allows a simple markup-generation.
  Possible exceptions to the update operation are automatically triggered.

  Finally, the view-aspects were handled by an API for parsing-combinators. The library structure 
   boxed_sml‹Scan› provides the operators:

@{boxed_sml [display]
‹op ||     : ('a -> 'b) * ('a -> 'b) -> 'a -> 'b
op --     : ('a -> 'b * 'c) * ('c -> 'd * 'e) -> 'a -> ('b * 'd) * 'e
op >>     : ('a -> 'b * 'c) * ('b -> 'd) -> 'a -> 'd * 'c
op option : ('a -> 'b * 'a) -> 'a -> 'b option * 'a
op repeat : ('a -> 'b * 'a) -> 'a -> 'b list * 'a ›}
  for alternative, sequence, and piping, as well as combinators for option and repeat. Parsing 
  combinators have the advantage that they can be integrated into standard programs, 
  and they enable the dynamic extension of the grammar. There is a more high-level structure 
  boxed_sml‹Parse› providing specific combinators for the command-language Isar:

@{boxed_sml [display]
‹val attribute = Parse.position Parse.name 
              -- Scan.optional(Parse.$$$ "=" |-- Parse.!!! Parse.name)"";
val reference = Parse.position Parse.name 
              -- Scan.option (Parse.$$$ "::" |-- Parse.!!!
                              (Parse.position Parse.name));
val attributes =(Parse.$$$ "[" |-- (reference 
               -- (Scan.optional(Parse.$$$ ","
                   |--(Parse.enum ","attribute)))[]))--| Parse.$$$ "]"              
›}                                          

  The ``model'' boxed_sml‹create_and_check_docitem› and ``new''
  boxed_sml‹ODL_Meta_Args_Parser.attributes› parts were 
  combined via the piping operator and registered in the Isar toplevel:

@{boxed_sml [display]
‹val _ = 
  let fun create_and_check_docitem (((oid, pos),cid_pos),doc_attrs) 
                 = (Value_Command.Docitem_Parser.create_and_check_docitem
                          {is_monitor = false} {is_inline=true}
                          {define = false} oid pos (cid_pos) (doc_attrs))
  in  Outer_Syntax.command @{command_keyword "declare_reference*"}
                       "declare document reference"
                       (ODL_Meta_Args_Parser.attributes 
                        >> (Toplevel.theory o create_and_check_docitem))
  end;›}

  Altogether, this gives the extension of Isabelle/HOL with Isar syntax and semantics for the 
  new \emph{command}:

@{boxed_theory_text [display]declare_reference* [lal::requirement, alpha="main", beta=42]}

  The construction also generates implicitly some markup information; for example, when hovering
  over the boxed_theory_textdeclare_reference* command in the IDE, a popup window with the text: 
  ``declare document reference'' will appear.
›

section‹Programming Antiquotations›
text‹
  The definition and registration of text antiquotations and ML-antiquotations is similar in 
  principle: based on a number of combinators, new user-defined antiquotation syntax and semantics
  can be added to the system that works on the internal plugin-data freely. For example, in

@{boxed_sml [display]
‹val _ = Theory.setup
         (docitem_antiquotation  @{binding "docitem"}  DOF_core.default_cid #>
            
        ML_Antiquotation.inline @{binding "docitem_value"} 
              ML_antiquotation_docitem_value)›}
  the text antiquotation boxed_sml‹docitem› is declared and bounded to a parser for the argument 
  syntax and the overall semantics. This code defines a generic antiquotation to be used in text 
  elements such as

@{boxed_theory_text [display]text‹as defined in @{docitem ‹d1›} ...›}

  The subsequent registration boxed_sml‹docitem_value› binds code to a ML-antiquotation usable 
  in an ML context for user-defined extensions; it permits the access to the current ``value'' 
  of document element, ie, a term with the entire update history.

  It is possible to generate antiquotations \emph{dynamically}, as a consequence of a class 
  definition in ODL. The processing of the ODL class typdefinition also \emph{generates}
  a text antiquotation boxed_theory_text‹@{"definition" ‹d1›}, which works similar to 
  boxed_theory_text‹@{docitem ‹d1›} except for an additional type-check that assures that 
  boxed_theory_text‹d1› is a reference to a definition. These type-checks support the subclass hierarchy.
›

section‹Implementing Second-level Type-Checking›

text‹
  On expressions for attribute values, for which we chose to use HOL syntax to avoid that users 
  need to learn another syntax, we implemented an own pass over type-checked terms. Stored in the 
  late-binding table boxed_sml‹ISA_transformer_tab›, we register for each term-annotation 
  (ISA's), a function of type

@{boxed_sml [display]
‹   theory -> term * typ * Position.T -> term option›}

  Executed in a second pass of term parsing, ISA's may just return boxed_theory_text‹None›. This is 
  adequate for ISA's just performing some checking in the logical context boxed_theory_texttheory; 
  ISA's of this kind report errors  by exceptions. In contrast, ‹transforming› ISA's will 
  yield a term; this is adequate, for example, by replacing a string-reference to some term denoted 
  by it. This late-binding table is also used to generate standard inner-syntax-antiquotations from 
  a boxed_theory_textdoc_class.
›

section‹Programming Class Invariants›
text‹
  See technicalsec_low_level_inv.
›

section‹Implementing Monitors›

text‹
  Since monitor-clauses have a regular expression syntax, it is natural to implement them as 
  deterministic automata. These are stored in the  boxed_sml‹docobj_tab› for monitor-objects 
  in the isadof component. We implemented the functions:

@{boxed_sml [display]
‹  val  enabled : automaton -> env -> cid list
   val  next    : automaton -> env -> cid -> automaton›}
  where boxed_sml‹env› is basically a map between internal automaton states and class-id's 
  (boxed_sml‹cid›'s). An automaton is said to be ‹enabled› for a class-id, 
  iff it either occurs in its accept-set or its reject-set (see @{docitem "sec_monitors"}). During 
  top-down document validation, whenever a text-element is encountered, it is checked if a monitor 
  is \emph{enabled} for this class; in this case, the boxed_sml‹next›-operation is executed. The 
  transformed automaton recognizing the suffix is stored in boxed_sml‹docobj_tab› if
  possible;
  otherwise, if boxed_sml‹next› fails, an error is reported. The automata implementation
  is, in large parts, generated from a formalization of functional automata
  cite"nipkow.ea:functional-Automata-afp:2004".
›

section‹The LaTeX-Core of isadof
text‹
  The LaTeX-implementation of isadof heavily relies on the 
  ``keycommand''~cite"chervet:keycommand:2010" package. In fact, the core isadof LaTeX-commands
  are just wrappers for the corresponding commands from the keycommand package:

@{boxed_latex [display]
‹\newcommand\newisadof[1]{%
  \expandafter\newkeycommand\csname isaDof.#1\endcsname}%
\newcommand\renewisadof[1]{%
  \expandafter\renewkeycommand\csname isaDof.#1\endcsname}%
\newcommand\provideisadof[1]{%
  \expandafter\providekeycommand\csname isaDof.#1\endcsname}%›}

  The LaTeX-generator of isadof maps each boxed_theory_text‹doc_item› to an LaTeX-environment (recall
  @{docitem "text_elements"}). As generic boxed_theory_text‹doc_item›s are derived from the text element, 
  the environment \inlineltx|isamarkuptext*| builds the core of isadof's LaTeX implementation. 

›
(*<*)
end
(*>*)