src/HOL/ex/Quicksort.thy
changeset 61343 5b5656a63bd6
parent 60515 484559628038
child 62430 9527ff088c15
--- a/src/HOL/ex/Quicksort.thy	Tue Oct 06 17:46:07 2015 +0200
+++ b/src/HOL/ex/Quicksort.thy	Tue Oct 06 17:47:28 2015 +0200
@@ -2,7 +2,7 @@
     Copyright   1994 TU Muenchen
 *)
 
-section {* Quicksort with function package *}
+section \<open>Quicksort with function package\<close>
 
 theory Quicksort
 imports "~~/src/HOL/Library/Multiset"