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