test/Tools/isac/ADDTESTS/accumulate-val/Thy_2.thy
author wenzelm
Sat, 12 Jun 2021 18:22:07 +0200
changeset 60298 09106b85d3b4
parent 59852 ea7e6679080e
permissions -rw-r--r--
use more antiquotations;
     1 theory Thy_2 imports Thy_1 begin
     2 
     3 ML \<open>val test_list_rls =
     4   Rule_Set.append_rules "test_list_rls" Rule_Set.empty
     5     [\<^rule_thm>\<open>refl\<close>, \<^rule_thm>\<open>subst\<close>]\<close>
     6 
     7 setup \<open>Test_KEStore_Elems.add_rlss 
     8   [("test_list_rls", (Context.theory_name @{theory}, (*already added in Thy_1.thy*)
     9     test_list_rls))]\<close>
    10 
    11 ML \<open>(*test_ruleset' := overwritelthy @{theory} (! test_ruleset', 
    12   [("test_list_rls", test_list_rls)])*)
    13 \<close>
    14 
    15 end