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