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