test/Tools/isac/ADDTESTS/accumulate-val/Thy_2.thy
changeset 55359 73dc85c025ab
parent 52156 aa0884017d48
child 59410 2cbb98890190
equal deleted inserted replaced
55358:b1f0389ca11f 55359:73dc85c025ab
     1 theory Thy_2 imports Thy_1 begin
     1 theory Thy_2 imports Thy_1 begin
     2 
     2 
     3 ML {* val test_list_rls =
     3 ML {* val test_list_rls =
     4   append_rls "test_list_rls" e_rls [Thm ("refl", @{thm refl}), Thm ("subst", @{thm subst})] *}
     4   append_rls "test_list_rls" e_rls [Thm ("refl", @{thm refl}), Thm ("subst", @{thm subst})] *}
     5 
     5 
     6 setup {* KEStore_Elems.add_rlss 
     6 setup {* Test_KEStore_Elems.add_rlss 
     7   [("test_list_rls", (Context.theory_name @{theory}, (*already added in Thy_1.thy*)
     7   [("test_list_rls", (Context.theory_name @{theory}, (*already added in Thy_1.thy*)
     8     test_list_rls))] *}
     8     test_list_rls))] *}
     9 
     9 
    10 ML {* (*test_ruleset' := overwritelthy @{theory} (! test_ruleset', 
    10 ML {* (*test_ruleset' := overwritelthy @{theory} (! test_ruleset', 
    11   [("test_list_rls", test_list_rls)])*)
    11   [("test_list_rls", test_list_rls)])*)