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