src/HOL/Library/Saturated.thy
changeset 60500 903bb1495239
parent 60011 3eef7a43cd51
child 60679 ade12ef2773c
--- a/src/HOL/Library/Saturated.thy	Wed Jun 17 10:57:11 2015 +0200
+++ b/src/HOL/Library/Saturated.thy	Wed Jun 17 11:03:05 2015 +0200
@@ -4,13 +4,13 @@
     Author:     Florian Haftmann
 *)
 
-section {* Saturated arithmetic *}
+section \<open>Saturated arithmetic\<close>
 
 theory Saturated
 imports Numeral_Type "~~/src/HOL/Word/Type_Length"
 begin
 
-subsection {* The type of saturated naturals *}
+subsection \<open>The type of saturated naturals\<close>
 
 typedef ('a::len) sat = "{.. len_of TYPE('a)}"
   morphisms nat_of Abs_sat
@@ -116,7 +116,7 @@
     proof(cases "c = 0")
       case True thus ?thesis by (simp add: sat_eq_iff)
     next
-      case False with `a \<noteq> 0` show ?thesis
+      case False with \<open>a \<noteq> 0\<close> show ?thesis
         by (simp add: sat_eq_iff nat_mult_min_left nat_mult_min_right mult.assoc min.assoc min.absorb2)
     qed
   qed