test/Tools/isac/ADDTESTS/accumulate-val/Thy_3.thy
changeset 60298 09106b85d3b4
parent 59878 3163e63a5111
     1.1 --- a/test/Tools/isac/ADDTESTS/accumulate-val/Thy_3.thy	Sat Jun 12 18:06:27 2021 +0200
     1.2 +++ b/test/Tools/isac/ADDTESTS/accumulate-val/Thy_3.thy	Sat Jun 12 18:22:07 2021 +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_Set.append_rules "test_list_rls" Rule_Set.empty [Rule.Thm ("not_def", @{thm not_def})]\<close>
     1.8 +  Rule_Set.append_rules "test_list_rls" Rule_Set.empty [\<^rule_thm>\<open>not_def\<close>]\<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>