test/Tools/isac/ADDTESTS/accumulate-val/Thy_3.thy
changeset 59850 f3cac3053e7b
parent 59773 d88bb023c380
child 59851 4dd533681fef
     1.1 --- a/test/Tools/isac/ADDTESTS/accumulate-val/Thy_3.thy	Wed Apr 01 19:20:05 2020 +0200
     1.2 +++ b/test/Tools/isac/ADDTESTS/accumulate-val/Thy_3.thy	Sat Apr 04 12:11:32 2020 +0200
     1.3 @@ -1,7 +1,7 @@
     1.4  theory Thy_3 imports Thy_2 Thy_2b begin
     1.5  
     1.6  ML \<open>val test_list_rls =
     1.7 -  Rule.append_rls "test_list_rls" Rule.e_rls [Rule.Thm ("not_def", @{thm not_def})]\<close>
     1.8 +  Rule_Set.append_rls "test_list_rls" Rule_Set.e_rls [Rule.Thm ("not_def", @{thm not_def})]\<close>
     1.9  
    1.10  setup \<open>Test_KEStore_Elems.add_rlss (*already added in Thy_1.thy and Thy_2.thy*)
    1.11    [("test_list_rls", (Context.theory_name @{theory}, test_list_rls))]\<close>
    1.12 @@ -16,7 +16,7 @@
    1.13  (*if length (Test_KEStore_Elems.get_rlss @{theory}) = length (! test_ruleset')
    1.14    then () else error "Test_KEStore_Elems.get_rlss = test_ruleset': changed"*)
    1.15    ;
    1.16 -  val SOME (_, Rule.Rls {rules, ...}) =
    1.17 +  val SOME (_, Rule_Set.Rls {rules, ...}) =
    1.18      AList.lookup op= (Test_KEStore_Elems.get_rlss @{theory}) "test_list_rls"
    1.19    ;
    1.20    case rules of