test/Tools/isac/Knowledge/integrate.thy
author Walther Neuper <wneuper@ist.tugraz.at>
Thu, 22 Aug 2019 16:48:04 +0200
changeset 59585 0bb418c3855a
parent 59545 4035ec339062
child 59592 99c8d2ff63eb
permissions -rw-r--r--
lucin: rename Script --> Program
     1 
     2 theory integrate
     3 imports Isac.Build_Thydata
     4 begin
     5 
     6 ML \<open>
     7 "----------- method analog to rls 'integration' ---------";
     8 "----------- method analog to rls 'integration' ---------";
     9 "----------- method analog to rls 'integration' ---------";
    10 \<close>
    11 partial_function (tailrec) integration_test :: "real \<Rightarrow> real \<Rightarrow> real"
    12   where
    13 "integration_test f_f v_v =
    14   (((Rewrite_Set_Inst [(''bdv'',v_v)] ''integration_rules'' False) @@
    15     (Rewrite_Set_Inst [(''bdv'',v_v)] ''add_new_c'' False)         @@
    16     (Rewrite_Set_Inst [(''bdv'',v_v)] ''simplify_Integral'' False)) (f_f::real))"
    17 setup \<open>KEStore_Elems.add_mets
    18   [Specify.prep_met @{theory "Isac"} "met_testint" [] Celem.e_metID
    19 	    (["diff","integration","test"],
    20 	      [("#Given" ,["functionTerm f_f", "integrateBy v_v"]), ("#Find", ["antiDerivative F_F"])],
    21 	      {rew_ord'="tless_true", rls'=Atools_erls, calc = [], srls = Rule.e_rls, prls = Rule.e_rls,
    22 	        crls = Atools_erls, errpats = [], nrls = Rule.e_rls},
    23 	      @{thm integration_test.simps}
    24 	    (*"Program IntegrationScript (f_f::real) (v_v::real) =             \
    25   	      \  (((Rewrite_Set_Inst [(''bdv'',v_v)] ''integration_rules'' False) @@ \
    26           \    (Rewrite_Set_Inst [(''bdv'',v_v)] ''add_new_c'' False)         @@ \
    27           \    (Rewrite_Set_Inst [(''bdv'',v_v)] ''simplify_Integral'' False)) (f_f::real))"*))]
    28 \<close>
    29 
    30 end