src/HOL/List.thy
changeset 69349 7cef9e386ffe
parent 69312 e0f68a507683
child 69593 3dda49e08b9d
--- a/src/HOL/List.thy	Tue Nov 27 16:22:12 2018 +0100
+++ b/src/HOL/List.thy	Tue Nov 27 21:07:39 2018 +0100
@@ -508,7 +508,7 @@
     fun check s1 s2 =
       read s1 aconv read s2 orelse
         error ("Check failed: " ^
-          quote (Input.source_content s1) ^ Position.here_list [Input.pos_of s1, Input.pos_of s2]);
+          quote (#1 (Input.source_content s1)) ^ Position.here_list [Input.pos_of s1, Input.pos_of s2]);
   in
     check \<open>[(x,y,z). b]\<close> \<open>if b then [(x, y, z)] else []\<close>;
     check \<open>[(x,y,z). (x,_,y)\<leftarrow>xs]\<close> \<open>map (\<lambda>(x,_,y). (x, y, z)) xs\<close>;