src/Tools/isac/TODO.thy
author Walther Neuper <walther.neuper@jku.at>
Fri, 10 Apr 2020 18:32:36 +0200
changeset 59868 d77aa0992e0f
parent 59865 75a9d629ea53
child 59872 cea2815f65ed
permissions -rw-r--r--
use "UnparseC" for renaming identifiers
     1 (* Title:  todo's for isac core
     2    Author: Walther Neuper 111013
     3    (c) copyright due to lincense terms.
     4 *)
     5 theory TODO
     6 imports "~~/src/Doc/Prog_Prove/LaTeXsugar"
     7 begin
     8 
     9 text \<open>
    10 Legend: here + code since 200120
    11   \<open>(*DOC\<close> identifies stuff dedicated for isac/Doc/Lucas_Interpreter
    12   \<open>(*?!?\<close> identifies a design question
    13 
    14 Distillation of "rounds of reforms":
    15   \<open>TODOs from current changesets\<close> \<rightarrow> \<open>Postponed from current changeset\<close> \<rightarrow>
    16   (*to be removed..*) \<rightarrow> \<open>Separated tasks\<close> (*.. to be removed*)
    17   \<rightarrow> subsection of \<open>Major reforms\<close>
    18 \<close>
    19 
    20 section \<open>TODOs from current changesets\<close>
    21 text\<open>
    22   Shift more complicated issues from  \<open>Current changeset\<close> to \<open>Postponed from current changeset\<close>
    23 \<close>
    24 subsection \<open>Current changeset\<close>
    25 text \<open>
    26   \begin{itemize}
    27   \item xxx
    28   \item xxx
    29   \item xxx
    30   \item xxx
    31   \item xxx
    32   \item xxx
    33   \item xxx
    34   \item xxx
    35   \end{itemize}
    36 \<close>
    37 subsection \<open>Postponed from current changeset\<close>
    38 text \<open>
    39   \item see "TODO CLEANUP Thm" in code
    40     (* TODO CLEANUP Thm:
    41     Thm (string, thm): (a) needs string to identify sym_thmID for handling in front-end;
    42                        (b) investigate if ""RS sym" attaches a [.]" still occurs: ThmC_Def.string_of_thmI
    43     thmID            : type for data from user input + program
    44     thmDeriv         : type for thy_hierarchy ONLY
    45     obsolete types   : thm' (SEE "ad thm'"), thm''. 
    46     revise funs      : id_of_thm, thm_of_thm, rep_thm_G', eq_thmI, eq_thmI', thm''_of_thm thm.
    47     activate         : thmID_of_derivation_name'
    48     *)
    49   \item xxx
    50   \item use "Exec_Def" for renaming identifiers
    51   \item xxx
    52   \item xxx
    53   \item xxx
    54   \item xxx
    55   \begin{itemize}
    56   \item LI.do_next (*TODO RM..*) ???
    57   \item generate.sml: RM datatype edit TOGETHER WITH datatype inout
    58   \item TermC.list2isalist: typ -> term list -> term  .. should NOT requires typ
    59   \item get_ctxt_LI should replace get_ctxt
    60   \item ALL CODE: rename spec(ification) --> know(ledge), in Specification: Relation -> Knowledge
    61   \item rename   Base_Tool.thy  <---         Base_Tools
    62   \item adopt naming conventions in Knowledge: EqSystem --> Equation_System, etc
    63   \item rename field scr in meth
    64   \item DEL double code: nxt_specify_init_calc IN specify.sml + step-specify.sml
    65   \item xxx
    66   \item xxx
    67   \item xxx
    68   \item xxx
    69   \item xxx
    70   \item xxx
    71   \item xxx
    72   \item clarify Tactic.Subproblem (domID, pblID) as term in Pstate {act_arg, ...}
    73      there it is Free ("Subproblem", "char list \<times> ..
    74      instead of  Const (|???.Subproblem", "char list \<times> ..
    75      AND THE STRING REPRESENTATION IS STRANGE: 
    76        Subproblem (''Test'',
    77         ??.\ <^const> String.char.Char ''LINEAR'' ''univariate'' ''equation''
    78          ''test'')
    79      ML \<open>
    80      \<close> ML \<open>
    81      term2str; (*defined by..*)
    82      fun term_to_string''' thy t =
    83        let
    84          val ctxt' = Config.put show_markup false (Proof_Context.init_global thy)
    85        in Print_Mode.setmp [] (Syntax.string_of_term ctxt') t end;
    86      \<close> ML \<open>
    87      val t = @{term "aaa + bbb"}
    88      val t = @{term "Subproblem (''Test'', [''LINEAR'', ''univariate'', ''equation''])"};
    89      \<close> ML \<open>
    90      val sss = Print_Mode.setmp [] (Syntax.string_of_term @{context}) t
    91      \<close> ML \<open>
    92      writeln sss (*.. here perfect: Subproblem (''Test'', [''LINEAR'', ''univariate'', ''equation'']) *)
    93      \<close> ML \<open>
    94      \<close>
    95   \item xxx
    96   \item xxx
    97   \item cleanup fun me:
    98     fun me (*(_, Empty_Tac) p _ _ = raise ERROR ("me:  Empty_Tac at " ^ pos'2str p)
    99       | me*) (_, tac) p _(*NEW remove*) pt =
   100     + -------------------------^^^^^^
   101     # see test-code.sml fun me_trace
   102       use this also for me, not only for me_ist_ctxt; del. me
   103       this requires much updating in all test/*
   104   \item xxx
   105   \item xxx
   106   \item generate, generate1: NO thy as arg.
   107         Generate.generate1 thy is redundant: is the same during pbl, thus lookup spec
   108         redesign return value (originally for output by fun me?)
   109   \item xxx
   110   \item shift tests into NEW model.sml (upd, upds_envv, ..)
   111   \item xxx
   112   \item xxx
   113   \item clarify handling of contexts ctxt ContextC
   114     \begin{itemize}
   115     \item xxx
   116     \item Specify/ works with thy | Interpret/ works with ctxt | MathEngine.step works with ?!?ctxt
   117     \item xxx
   118     \item Check_Elementwise "Assumptions": prerequisite for ^^goal
   119       rm tactic Check_elementwise "Assumptions" in a way, which keeps it for Minisubpbl
   120       rm Assumptions  :: bool  (* TODO: remove with making ^^^ idle *)
   121     \item xxx
   122     \item xxx
   123     \end{itemize}
   124   \item xxx
   125   \item xxx
   126   \item complete mstools.sml (* survey on handling contexts:
   127   \item xxx
   128   \item xxx
   129   \item xxx
   130   \item xxx
   131   \item librarys.ml --> libraryC.sml + text from termC.sml
   132   \item xxx
   133   \item xxx
   134   \item xxx
   135   \item xxx
   136   \item xxx
   137   \item xxx
   138   \item concentrate "insert_assumptions" for locate_input_tactic in "associate", ?OR? Tactic.insert_assumptions
   139                                    DONE  for find_next_step by Tactic.insert_assumptions m' ctxt 
   140     \begin{itemize}
   141     \item rm from "generate1" ("Detail_Set_Inst'", Tactic.Detail_Set' ?)
   142     \item shift from "applicable_in..Apply_Method" to ? ? ? (is ONLY use-case in appl.sml))
   143     \item ?"insert_assumptions" necessary in "init_pstate" ?+++? in "applicable_in" ?+++? "associate"
   144     \item xxx
   145     \item xxx
   146     \item DO DELETIONS AFTER analogous concentrations in find_next_step
   147     \end{itemize}
   148   \item xxx
   149   \item ? what is the difference headline <--> cascmd in
   150     Subproblem' (spec, oris, headline, fmz_, context, cascmd)
   151   \item xxx
   152   \item inform: TermC.parse (Celem.assoc_thy "Isac_Knowledge") istr --> parseNEW context istr
   153   \item xxx
   154   \item unify/clarify stac2tac_ | 
   155     \begin{itemize}
   156     \item xxx
   157     \item extract common code from associate.. stac2tac_xxx
   158     \item rename LItool.tac_from_prog -> Tactic.from_prog_tac ? Solve_Tac.from_prog_tac,
   159     \item xxx
   160     \item xxx
   161     \end{itemize}
   162   \item xxx
   163   \item unify in signature LANGUAGE_TOOLS =\\
   164     val pblterm: ThyC.domID -> Celem.pblID -> term     vvv        vvv\\
   165     val subpbl: string -> string list -> term          unify with ^^^
   166   \item xxx
   167   \item Telem.safe is questionable: has it been replaced by Safe_Step, Not_Derivable, Helpless, etc?
   168     Note: replacement of Istate.safe by Istate.appy_ didn't care much about Telem.safe.
   169     If Telem.safe is kept, consider merge with CTbasic.ostate
   170   \item xxx
   171   \item remove find_next_step from solve Apply_Method';
   172     this enforces Pos.at_first_tactic, which should be dropped, too.
   173   \item xxx
   174   \item xxx
   175   \item xxx
   176   \end{itemize}
   177 \<close>
   178 subsection \<open>Postponed --> Major reforms\<close>
   179 text \<open>
   180   \begin{itemize}
   181   \item xxx          
   182   \item revisit bootstrap Calcelements. rule->calcelems->termC
   183     would be nice, but is hard: UnparseC.terms -> TermC.s_to_string
   184   \item xxx
   185   \item replace all Ctree.update_* with Ctree.cupdate_problem
   186   \item xxx
   187   \item rename (ist as {eval, ...}) -> (ist as {eval_rls, ...})
   188   \item xxx
   189   \item exception PROG analogous to TERM
   190   \item xxx
   191   \item sig/struc ..elems --> ..elem
   192   \item xxx          
   193   \item distille CAS-command, CAScmd, etc into a struct
   194   \item xxx          
   195   \item check location of files:
   196         test/Tools/isac/Interpret/ptyps.thy
   197         test/Tools/isac/Specify.ptyps.sml
   198   \item xxx
   199   \item check occurences of Atools in src/ test/
   200   \item Const ("Atools.pow", _) ---> Const ("Base_Tool.pow", _) 
   201   \item xxx          
   202   \item rm Float
   203   \item xxx
   204   \item Diff.thy: differentiateX --> differentiate after removal of script-constant
   205   \item Test.thy: met_test_sqrt2: deleted?!
   206   \item xxx          
   207   \item Rewrite_Ord.rew_ord' := overwritel (! Rewrite_Ord.rew_ord', (*<<<---- use KEStore.xxx, too*)
   208   \item xxx
   209     \item automatically extrac rls from program-code 
   210       ? take ["SignalProcessing", "Z_Transform", "Inverse_sub"] as an example ?
   211   \item xxx          
   212   \item finish output of trace_LI with Check_Postcond (useful for SubProblem)
   213   \item xxx
   214   \item replace Rule_Set.empty by Rule_Set.Empty
   215     latter is more clear, but replacing ***breaks rewriting over all examples***,
   216     e.g. see ERROR: rewrite__set_ called with 'Erls' for 'precond_rootpbl x'
   217     in Minisubplb/200-start-method-NEXT_STEP.sml:
   218      (*+* )------- in f3cac3053e7b (Rule_Set.empty just renamed, NOT deleted) we had
   219      (*+*)  prls =
   220      (*+*)    Rls {calc = [], erls = Erls, errpatts = [], id = "empty", preconds = [], rew_ord =
   221      (*+*)      ("dummy_ord", fn), rules = [], scr = EmptyScr, srls = Erls}:
   222      (*+*).. THIS IS Rule_Set.empty, BUT IT DID not CAUSE ANY ERROR !
   223      (*+*)------- WITH Rule_Set.empty REMOVED (based on f3cac3053e7b) we had
   224      (*+*)val Empty = prls (* <---ERROR: rewrite__set_ called with 'Erls' for 'precond_rootpbl x' *)
   225      ( *+*)val ["sqroot-test", "univariate", "equation", "test"] = cpI
   226     THAT INDICATES, that much rewriting/evaluating JUST WORKED BY CHANCE?!?
   227   \item xxx          
   228   \item xxx
   229   \item xxx          
   230   \item xxx
   231   \item xxx          
   232   \item xxx
   233   \item xxx          
   234   \end{itemize}
   235 \<close>
   236 
   237 section \<open>Major reforms\<close>
   238 text \<open>
   239 \<close>
   240 subsection \<open>Exception Size raised\<close>
   241 text \<open>
   242   During update Isabelle2018 --> Isabelle2019 we noticed, that
   243   "isabelle build" uses resources more efficiently than "isabelle jedit".
   244   The former works, but the latter causes 
   245   \begin{itemize}
   246   \item "Exception- Size raised"
   247     in Build_Thydata.thy
   248   \item "exception Size raised (line 169 of "./basis/LibrarySupport.sml")"
   249     in test/../biegelinie-*.xml.
   250   \end{itemize}
   251   This has been detected after changeset (30cd47104ad7) "lucin: reorganise theories in ProgLang".
   252 
   253   Find tools to investigate the Exception, and find ways around it eventually.
   254 \<close>
   255 subsection \<open>Cleanup & review signatures wrt. implementation.pdf canonical argument order\<close>
   256 text \<open>
   257   \begin{itemize}
   258   \item there are comments in several signatures
   259   \item ML_file "~~/src/Tools/isac/Interpret/specification-elems.sml" can be (almost) deleted
   260   \item src/../Frontend/: signatures missing
   261   \item xxx
   262   \end{itemize}
   263 \<close>
   264 subsection \<open>overall structure of code\<close>
   265 text \<open>
   266   \begin{itemize}
   267   \item try to separate Isac_Knowledge from MathEngine
   268     common base: Knowledge_Author / ..??
   269   \item xxx
   270   \item  ML_file "~~/src/Tools/isac/Interpret/ctree.sml" (*shift to base in common with Interpret*)
   271   \item xxx
   272   \item xxx
   273   \item xxx
   274   \end{itemize}
   275 \<close>
   276 subsection \<open>Separate MathEngineBasic/ Specify/ Interpret/ MathEngine/\<close>
   277 text \<open>
   278   \begin{itemize}
   279   \item xxx
   280   \item xxx
   281   \item re-organise code for Interpret
   282     \begin{itemize}
   283     \item Step*: Step_Specify | Step_Solve | Step
   284       \begin{itemize}
   285       \item *.check | *.add ARE TOO LATE IN BUILD with Step_Specify | Step_Solve
   286         Specify_Step.check | Specify_Step.add <-- Applicable.applicable_in
   287         Solve_Step.check   | Solve_Step.add   <-- Generate.generate1
   288       \item xxx
   289       \end{itemize}
   290     \item xxx
   291     \item Prog_Tac: fun get_first_argument takes both Prog_Tac + Program --- wait for separate Tactical
   292       then shift into common descendant
   293     \item xxx
   294     \end{itemize}
   295   \item xxx
   296   \item xxx
   297   \item ??????????? WHY CAN LI.by_tactic NOT BE REPLACED BY Step_Solve.by_tactic ???????????
   298   \item xxx
   299   \item xxx
   300   \end{itemize}
   301 \<close>
   302 subsection \<open>Review modelling- + specification-phase\<close>
   303 text \<open>
   304   \begin{itemize}
   305   \item xxx
   306   \item xxx
   307   \item xxx
   308   \item check match between args of partial_function and model-pattern of meth;
   309      provide error message.
   310   \item xxx
   311   \item "--- hack for funpack: generalise handling of meths which extend problem items ---"
   312     \begin{itemize}
   313     \item see several locations of hack in code
   314     \item these locations are NOT sufficient, see
   315       test/../biegelinie-3.sml --- IntegrierenUndKonstanteBestimmen2: Bsp.7.70. auto ---
   316     \item "fun associate" "match_ags ..dI" instead "..pI" breaks many tests, however,
   317       this would be according to survey Notes (3) in src/../calchead.sml.
   318     \end{itemize}
   319   \item see "failed trial to generalise handling of meths"98298342fb6d
   320   \item abstract specify + nxt_specif to common aux-funs;
   321     see e.g. "--- hack for funpack: generalise handling of meths which extend problem items ---"
   322   \item xxx
   323   \item type model = itm list ?
   324   \item review survey Notes in src/../calchead.sml: they are questionable
   325   \item review copy-named, probably two issues commingled 
   326     \begin{itemize}
   327     \item special handling of "#Find#, because it is not a formal argument of partial_function
   328     \item special naming for solutions of equation solving: x_1, x_2, ...
   329     \end{itemize}
   330   \item xxx
   331   \item structure Tactic Specify -?-> Proglang (would require Model., Selem.)
   332   \item xxx
   333   \item this has been written in one go:
   334     \begin{itemize}
   335     \item reconsidering Model.max_vt, use problem with meth ["DiffApp","max_by_calculus"]
   336     \item reconsider add_field': where is it used for what? Shift into mk_oris
   337     \item reconsider match_itms_oris: where is it used for what? max_vt ONLY???
   338     \item in Specify_Method search root-oris for items (e.g. "errorBound"), #1# in survey
   339     \item Specify_Problem, Specify_Method: check respective identifiers after re-Specify_
   340       (relevant for pre-condition)
   341     \item unify match_ags to mk_oris1..N with different args (fmz | pat list, pbl | meth
   342     \item 
   343     \end{itemize}
   344   \end{itemize}
   345 \<close>
   346 subsection \<open>taci list, type step\<close>
   347 text \<open>
   348 taci was, most likely, invented to make "fun me" more efficient by avoiding duplicate rewrite,
   349 and probably, because the Kernel interface separated setNextTactic and applyTactic.
   350 Both are no good reasons to make code more complicated.
   351 
   352 !!! taci list is used in do_next !!!
   353 
   354   \begin{itemize}
   355   \item xxx
   356   \item can lev_on_total replace lev_on ? ..Test_Isac_Short + rename lev_on_total -> lev_on
   357   \item xxx
   358   \item Step* functions should return Calc.T instead of Chead.calcstate'
   359   \item xxx
   360   \item states.sml: check, when "length tacis > 1"
   361   \item in Test_Isac.thy there is only 1 error in Interpret/inform.sml
   362   \item (*WN190713 REMOVE: "creating a new node" was never implemented for more than one node?!?
   363   \item xxx
   364   \item brute force setting all empty ([], [], ptp) works!?! but ptp causes errors -- investigate!
   365   \item xxx
   366   \end{itemize}
   367 \<close>
   368 subsection \<open>Ctree\<close>
   369 text \<open>
   370 analysis
   371 # mixture pos' .. pos in cappend_*, append_* is confusing
   372 # existpt p pt andalso Tactic.is_empty DIFFERENT IN append_*, cappend_* is confusing
   373   "exception PTREE "get_obj: pos =" ^^^^^: ^^^^ due to cut !!!
   374   NOTE: exn IN if..andalso.. IS NOT!!! DETECTED, THIS                       is confusing
   375   see test/../--- Minisubpbl/800-append-on-Frm.sml ---
   376 # ?!? "cut branches below cannot be decided here" in append_atomic
   377 # sign. of functions too different ?!?canonical arg.order ?!?
   378   \begin{itemize}
   379   \item xxx
   380   \item remove update_branch, update_*? -- make branch, etc args of append_*
   381   \item xxx
   382   \item close sig Ctree, contains cappend_* ?only? --- ?make parallel to ?Pide_Store?
   383   \item xxx
   384   \item unify args to Ctree.state (pt, p)
   385   \item  fun update_env       .. repl_env                   \<rightarrow>updatempty
   386   \item xxx
   387   \item xxx
   388   \item xxx
   389   \item xxx
   390   \end{itemize}
   391 \<close>
   392 subsection \<open>replace theory/thy by context/ctxt\<close>
   393 text \<open>
   394   \begin{itemize}
   395   \item xxx
   396   \item Specify/ works with thy | Interpret/ works with ctxt | MathEngine.step works with ?!?ctxt
   397     special case: Tactic.Refine_Problem
   398   \item xxx
   399   \item theory can be retrieved from ctxt by Proof_Context.theory_of
   400   \item xxx
   401   \item cleaup the many conversions string -- theory
   402   \item make dest_spec --> (theory, pblID, metID) ?+ common_subthy ?
   403   \item 1. Rewrite.eval_true_, then
   404     LItool.check_leaf, Rewrite.eval_prog_expr, Generate.generate1, LItool.tac_from_prog.
   405   \item fun associate
   406     let val thy = Celem.assoc_thy "Isac_Knowledge";(*TODO*)
   407   \item xxx
   408   \item xxx
   409   \item in locate_input_tactic .. ?scan_dn1?; Program.is_eval_expr   .use  Term.exists_Const
   410   \item push srls into pstate
   411   \item lucas-intrpreter.locate_input_tactic: scan_to_tactic1 srls tac cstate (progr, Rule_Set.Empty)
   412                                                                                       ^^^^^^^^^^^^^^^
   413   \item xxx
   414   \end{itemize}
   415 \<close>
   416 subsection \<open>Rfuns, Begin_/End_Detail', Rrls, Istate\<close>
   417 text \<open>
   418 remove refactor Rfuns, Rule.Prog, Rule.EmptyScr, RrlsState: this is a concept never brought to work.
   419   Clarify relation to reverse rewriting!
   420   \begin{itemize}
   421   \item separate mut.recursion program with rule and rls by deleting fild scr in rls
   422     (possible since CS 43160c1e775a
   423   ` "replace Prog. in prep_rls by Auto_Prog.gen, which generates Prog. on the fly" )
   424   \item xxx
   425   \item probably only "normal_form" seems to be needed
   426   \item deleted Rfuns in NEW "locate_input_tactic": no active test for "locate_rule"
   427     but that seems desirable
   428   \item ?how is the relation to reverse-rewriting ???
   429   \item "Rfuns" markers in test/../rational
   430   \item xxx
   431   \item datatype istate (Istate.T): remove RrlsState, pstate: use Rrls only for creating results beyond
   432     rewriting and/or respective intermediate steps (e.g. cancellation of fractions).
   433     Thus we get a 1-step-action which does NOT require a state beyond istate/pstate.
   434     Thus we drastically reduce complexity, also get rid of "fun from_pblobj_or_detail_calc" , etc.
   435   \item debug ^^^ related: is there an occurence of Steps with more than 1 element?
   436   \item xxx
   437   \item and do_next (* WN1907: ?only for Begin_/End_Detail' DEL!!!*)
   438   \item xxx
   439   \item shouldn't go Rfuns from Rewrite --> Rewrite_Set; they behave similar to "fun interSteps" ?
   440   \item xxx
   441   \item ?finally Prog could go from Calcelems to ProgLang?
   442   \end{itemize}
   443 \<close>
   444 subsection \<open>Inverse_Z_Transform.thy\<close>
   445 text \<open>
   446   \begin{itemize}
   447   \item\label{new-var-rhs} rule1..6, ruleZY introduce new variables on the rhs of the rewrite-rule.
   448   ? replace rewriting with substitution ?!?
   449   The problem is related to the decision of typing for "d_d" and making bound variables free (while
   450   shifting specific handling in equation solving etc. to the meta-logic). 
   451   \item Find "stepResponse (x[n::real]::bool)" is superfluous, because immediately used by
   452     rewrite-rules; see \ref{new-var-rhs}.
   453   \item Reconsider whole problem:
   454     input only the polynomial as argument of partial_function, in ([1], Frm) compile lhs "X z" ?
   455   \end{itemize}
   456 \<close>
   457 subsection \<open>Adopt Isabelle's numerals for Isac\<close>
   458 text \<open>
   459   \begin{itemize}
   460   \item replace numerals of type "real" by "nat" in some specific functions from ListC.thy
   461     and have both representations in parallel for "nat".
   462   \item xxx
   463   \item xxx
   464   \end{itemize}
   465 \<close>
   466 subsection \<open>Redesign equation solver\<close>
   467 text \<open>
   468   Existing solver is structured along the WRONG assumption,
   469   that Poly.thy must be the LAST thy among all thys involved -- while the opposite is the case.
   470 
   471   Preliminary solution: all inappropriately located thms are collected in Base_Tools.thy
   472 \<close>
   473 subsection \<open>Finetunig required for xmldata in kbase\<close>
   474 text \<open>
   475   See xmldata https://intra.ist.tugraz.at/hg/isac/rev/5b222a649390
   476   and in kbase html-representation generated from these xmldata.
   477   Notes in ~~/xmldata/TODO.txt.
   478 \<close>
   479 
   480 section \<open>Hints for further development\<close>
   481 text \<open>
   482 \<close>
   483 subsection \<open>Coding standards & some explanations for math-authors\<close>
   484 text \<open>copy from doc/math-eng.tex WN.28.3.03
   485 WN071228 extended\<close>
   486 
   487 subsubsection \<open>Identifiers\<close>
   488 text \<open>Naming is particularily crucial, because Isabelles name space is global, and isac does
   489   not yet use the novel locale features introduces by Isar. For instance, {\tt probe} sounds
   490   reasonable as (1) a description in the model of a problem-pattern, (2) as an element of the
   491   problem hierarchies key, (3) as a socalled CAS-command, (4) as the name of a related script etc.
   492   However, all the cases (1)..(4) require different typing for one and the same
   493   identifier {\tt probe} which is impossible, and actually leads to strange errors
   494   (for instance (1) is used as string, except in a script addressing a Subproblem).
   495 
   496   These are the preliminary rules for naming identifiers>
   497   \begin{description}
   498   \item [elements of a key] into the hierarchy of problems or methods must not contain
   499     capital letters and may contain underscrores, e.g. {\tt probe, for_polynomials}.
   500   \item [descriptions in problem-patterns] must contain at least 1 capital letter and
   501     must not contain underscores, e.g. {\tt Probe, forPolynomials}.
   502   \item [CAS-commands] follow the same rules as descriptions in problem-patterns above, thus
   503     beware of conflicts~!
   504   \item [script identifiers] always end with {\tt Program}, e.g. {\tt ProbeScript}.
   505   \item [???] ???
   506   \item [???] ???
   507   \end{description}
   508 %WN071228 extended\<close>
   509 
   510 subsubsection \<open>Rule sets\<close>
   511 text \<open>The actual version of the coding standards for rulesets is in {\tt /IsacKnowledge/Atools.ML
   512   where it can be viewed using the knowledge browsers.
   513 
   514   There are rulesets visible to the student, and there are rulesets visible (in general) only for
   515   math authors. There are also rulesets which {\em must} exist for {\em each} theory;
   516   these contain the identifier of the respective theory (including all capital letters) 
   517   as indicated by {\it Thy} below.
   518 
   519   \begin{description}
   520   \item [norm\_{\it Thy}] exists for each theory, and {\em efficiently} calculates a
   521     normalform for all terms which can be expressed by the definitions of the respective theory
   522     (and the respective parents).
   523   \item [simplify\_{\it Thy}] exists for each theory, and calculates a normalform for all terms
   524     which can be expressed by the definitions of the respective theory (and the respective parents)
   525     such, that the rewrites can be presented to the student.
   526   \item [calculate\_{\it Thy}] exists for each theory, and evaluates terms with 
   527     numerical constants only (i.e. all terms which can be expressed by the definitions of
   528     the respective theory and the respective parent theories). In particular, this ruleset includes
   529     evaluating in/equalities with numerical constants only.
   530     WN.3.7.03: may be dropped due to more generality: numericals and non-numericals
   531     are logically equivalent, where the latter often add to the assumptions
   532     (e.g. in Check_elementwise).
   533   \end{description}
   534 
   535   The above rulesets are all visible to the user, and also may be input; 
   536   thus they must be contained in {\tt Theory_Data} (KEStore_Elems.add_rlss,
   537   KEStore_Elems.get_rlss). All these rulesets must undergo a preparation
   538   using the function {\tt prep_rls'}, which generates a script for stepwise rewriting etc.
   539   The following rulesets are used for internal purposes and usually invisible to the (naive) user:
   540 
   541   \begin{description}
   542   \item [*\_erls] TODO
   543   \item [*\_prls] 
   544   \item [*\_srls] 
   545   \end{description}
   546 {\tt Rule_Set.append_rules, Rule_Set.merge, remove_rls} TODO
   547 \<close>
   548 
   549 subsection \<open>get proof-state\<close>
   550 text \<open>
   551   Re: [isabelle] Programatically get "this"
   552   ----------------------------------------------------
   553   So here is my (Makarius') version of your initial example, following these principles:
   554   begin{verbatim}
   555     notepad
   556     begin
   557       assume a: A
   558       ML_val \<open>
   559         val ctxt = @{context};
   560     
   561         val this_name =
   562           Name_Space.full_name (Proof_Context.naming_of ctxt) (Binding.name Auto_Bind.thisN);
   563         val this = #thms (the (Proof_Context.lookup_fact ctxt this_name));
   564       \<close>
   565     end
   566   end{verbatim}
   567 \<close>
   568 subsection \<open>write Specification to jEdit\<close>
   569 text \<open>
   570   Re: [isabelle] Printing terms with type annotations
   571   ----------------------------------------------------
   572   On 06/02/2019 17:52, Moa Johansson wrote:
   573   >
   574   > I’m writing some code that should create a snippet of Isar script.
   575   
   576   This is how Sledgehammer approximates this:
   577   
   578   http://isabelle.in.tum.de/repos/isabelle/file/Isabelle2018/src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML#l299
   579   
   580   (The module name already shows that the proper terminology is "Isar
   581   proof" (or "Isar proof text").  Proof scripts are a thing from the past,
   582   before Isar. You can emulate old-style proof scripts via a sequence of
   583   'apply' commands, but this is improper Isar.)
   584   
   585   Note that there is no standard function in Isabelle/Pure, because the
   586   problem to print just the right amount of type information is very
   587   complex and not fully solved. One day, after 1 or 2 rounds of
   588   refinements over the above approach, it might become generally available.
   589 \<close>
   590 subsection \<open>follow Isabelle conventions (*Does not yet work in Isabelle2018\<close>
   591 text \<open>
   592   isabelle update -u path_cartouches
   593   isabelle update -u inner_syntax_cartouches
   594 \<close>
   595 section \<open>Questions to Isabelle experts\<close>
   596 text \<open>
   597 \begin{itemize}
   598 \item ad ERROR Undefined fact "all_left"        in Test_Isac: error-pattern.sml
   599                Undefined fact: "xfoldr_Nil"                   inssort.sml
   600 \item xxx
   601 \item xxx
   602 \item ?OK Test_Isac_Short with
   603     LI.by_tactic tac (get_istate_LI pt p, get_ctxt_LI pt p) ptp
   604   instead
   605     LI.by_tactic tac (Istate.empty, ContextC.empty) ptp
   606   in step-solve ?
   607 \item xxx
   608 \item test from last CS with outcommented re-def of code -> 
   609   -> \<open>further tests additional to src/.. files\<close>
   610       ADDTESTS/redefined-code.sml
   611 \item xxx
   612 \item efb749b79361 Test_Some_Short.thy has 2 errors, which disappear in thy ?!?:
   613   ML_file "Interpret/error-pattern.sml" Undefined fact: "all_left"
   614   ML_file "Knowledge/inssort.sml" Undefined fact: "xfoldr_Nil"
   615 \item xxx
   616 \item what is the actual replacement of "hg log --follow" ?
   617 \item xxx
   618 \item how HANDLE these exceptions, e.g.:
   619     Syntax.read_term ctxt "Randbedingungen y 0 = (0::real), y L = 0, M_b 0 = 0, M_b L = 0]"
   620   GIVES
   621     "Inner syntax error
   622      Failed to parse term"
   623 \item xxx
   624 \item how cope with "exception Size raised (line 171 of "./basis/LibrarySupport.sml")"
   625   e.g. in test/Interpret/lucas-interpreter.sml
   626 \item xxx
   627 \item xxx
   628 \end{itemize}
   629 \<close>
   630 
   631 section \<open>For copy & paste\<close>
   632 text \<open>
   633 \begin{itemize}
   634 \item xxx
   635   \begin{itemize}
   636   \item xxx
   637     \begin{itemize}
   638     \item xxx
   639       \begin{itemize}
   640       \item xxx
   641         \begin{itemize}
   642         \item xxx
   643         \end{itemize}
   644       \end{itemize}
   645     \end{itemize}
   646   \end{itemize}
   647 \end{itemize}
   648 \<close>
   649 subsection \<open>xxx\<close>
   650 subsubsection \<open>xxx\<close>
   651 end