src/Tools/isac/TODO.thy
author Walther Neuper <walther.neuper@jku.at>
Tue, 21 Apr 2020 15:42:50 +0200
changeset 59898 68883c046963
parent 59887 4616b145b1cd
child 59901 07a042166900
permissions -rw-r--r--
replace Celem. with new struct.s in BaseDefinitions/

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