test/Tools/isac/ADDTESTS/accumulate-val/Thy_2.thy
changeset 60298 09106b85d3b4
parent 59852 ea7e6679080e
equal deleted inserted replaced
60297:73e7175a7d3f 60298:09106b85d3b4
     1 theory Thy_2 imports Thy_1 begin
     1 theory Thy_2 imports Thy_1 begin
     2 
     2 
     3 ML \<open>val test_list_rls =
     3 ML \<open>val test_list_rls =
     4   Rule_Set.append_rules "test_list_rls" Rule_Set.empty
     4   Rule_Set.append_rules "test_list_rls" Rule_Set.empty
     5     [Rule.Thm ("refl", @{thm refl}), Rule.Thm ("subst", @{thm subst})]\<close>
     5     [\<^rule_thm>\<open>refl\<close>, \<^rule_thm>\<open>subst\<close>]\<close>
     6 
     6 
     7 setup \<open>Test_KEStore_Elems.add_rlss 
     7 setup \<open>Test_KEStore_Elems.add_rlss 
     8   [("test_list_rls", (Context.theory_name @{theory}, (*already added in Thy_1.thy*)
     8   [("test_list_rls", (Context.theory_name @{theory}, (*already added in Thy_1.thy*)
     9     test_list_rls))]\<close>
     9     test_list_rls))]\<close>
    10 
    10