src/Tools/Spec_Check/Examples.thy
changeset 69593 3dda49e08b9d
parent 62020 5d208fd2507d
--- a/src/Tools/Spec_Check/Examples.thy	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/Tools/Spec_Check/Examples.thy	Fri Jan 04 23:22:53 2019 +0100
@@ -76,7 +76,7 @@
 
 
 ML_command \<open>
-val thy = @{theory};
+val thy = \<^theory>;
 check_property "ALL t u. if Pattern.matches thy (t, u) then Term.could_unify (t, u) else true"
 \<close>