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