src/HOL/Algebra/Congruence.thy
changeset 61382 efac889fccbc
parent 44471 3c2b2c4a7c1c
child 63167 0909deb8059b
--- a/src/HOL/Algebra/Congruence.thy	Sat Oct 10 16:21:34 2015 +0200
+++ b/src/HOL/Algebra/Congruence.thy	Sat Oct 10 16:26:23 2015 +0200
@@ -7,15 +7,15 @@
 imports Main
 begin
 
-section {* Objects *}
+section \<open>Objects\<close>
 
-subsection {* Structure with Carrier Set. *}
+subsection \<open>Structure with Carrier Set.\<close>
 
 record 'a partial_object =
   carrier :: "'a set"
 
 
-subsection {* Structure with Carrier and Equivalence Relation @{text eq} *}
+subsection \<open>Structure with Carrier and Equivalence Relation @{text eq}\<close>
 
 record 'a eq_object = "'a partial_object" +
   eq :: "'a \<Rightarrow> 'a \<Rightarrow> bool" (infixl ".=\<index>" 50)