test/Tools/isac/ADDTESTS/accumulate-val/Thy_2b.thy
changeset 60298 09106b85d3b4
parent 59852 ea7e6679080e
     1.1 --- a/test/Tools/isac/ADDTESTS/accumulate-val/Thy_2b.thy	Sat Jun 12 18:06:27 2021 +0200
     1.2 +++ b/test/Tools/isac/ADDTESTS/accumulate-val/Thy_2b.thy	Sat Jun 12 18:22:07 2021 +0200
     1.3 @@ -1,7 +1,7 @@
     1.4  theory Thy_2b imports Thy_1 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 ("False_def", @{thm False_def})]\<close>
     1.8 +  Rule_Set.append_rules "test_list_rls" Rule_Set.empty [\<^rule_thm>\<open>False_def\<close>]\<close>
     1.9  
    1.10  setup \<open>Test_KEStore_Elems.add_rlss [("test_list_rls", (Context.theory_name @{theory},
    1.11    test_list_rls))]\<close>