src/FOL/ex/Natural_Numbers.thy
changeset 60770 240563fbf41d
parent 58889 5b7a9633cfa8
child 69587 53982d5ec0bb
--- a/src/FOL/ex/Natural_Numbers.thy	Thu Jul 23 14:20:51 2015 +0200
+++ b/src/FOL/ex/Natural_Numbers.thy	Thu Jul 23 14:25:05 2015 +0200
@@ -2,16 +2,16 @@
     Author:     Markus Wenzel, TU Munich
 *)
 
-section {* Natural numbers *}
+section \<open>Natural numbers\<close>
 
 theory Natural_Numbers
 imports FOL
 begin
 
-text {*
+text \<open>
   Theory of the natural numbers: Peano's axioms, primitive recursion.
   (Modernized version of Larry Paulson's theory "Nat".)  \medskip
-*}
+\<close>
 
 typedecl nat
 instance nat :: "term" ..