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