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