src/HOL/Library/More_List.thy
changeset 60500 903bb1495239
parent 58881 b9556a055632
child 63040 eb4ddd18d635
--- a/src/HOL/Library/More_List.thy	Wed Jun 17 10:57:11 2015 +0200
+++ b/src/HOL/Library/More_List.thy	Wed Jun 17 11:03:05 2015 +0200
@@ -304,7 +304,7 @@
       with last_conv_nth_default [of ?ys dflt]
       have "last ?ys = nth_default dflt ?ys (length ?ys - 1)"
         by auto
-      moreover from `?ys \<noteq> []` no_trailing_strip_while [of "HOL.eq dflt" ys]
+      moreover from \<open>?ys \<noteq> []\<close> no_trailing_strip_while [of "HOL.eq dflt" ys]
         have "last ?ys \<noteq> dflt" by (simp add: no_trailing_unfold)
       ultimately have "nth_default dflt ?xs (length ?ys - 1) \<noteq> dflt"
         using eq by simp