src/Doc/Functions/Functions.thy
changeset 67443 3abf6a722518
parent 67406 23307fd33906
child 69505 cc2d676d5395
--- a/src/Doc/Functions/Functions.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/Doc/Functions/Functions.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -1095,11 +1095,11 @@
   let ?R = "measure (\<lambda>x. 101 - x)"
   show "wf ?R" ..
 
-  fix n :: nat assume "\<not> 100 < n" \<comment> "Assumptions for both calls"
+  fix n :: nat assume "\<not> 100 < n" \<comment> \<open>Assumptions for both calls\<close>
 
-  thus "(n + 11, n) \<in> ?R" by simp \<comment> "Inner call"
+  thus "(n + 11, n) \<in> ?R" by simp \<comment> \<open>Inner call\<close>
 
-  assume inner_trm: "f91_dom (n + 11)" \<comment> "Outer call"
+  assume inner_trm: "f91_dom (n + 11)" \<comment> \<open>Outer call\<close>
   with f91_estimate have "n + 11 < f91 (n + 11) + 11" .
   with \<open>\<not> 100 < n\<close> show "(f91 (n + 11), n) \<in> ?R" by simp
 qed