src/HOL/Library/Tree_Multiset.thy
changeset 60502 aa58872267ee
parent 60495 d7ff0a1df90a
parent 60500 903bb1495239
child 60506 83231b558ce4
--- a/src/HOL/Library/Tree_Multiset.thy	Wed Jun 17 17:33:22 2015 +0200
+++ b/src/HOL/Library/Tree_Multiset.thy	Wed Jun 17 17:54:09 2015 +0200
@@ -1,14 +1,14 @@
 (* Author: Tobias Nipkow *)
 
-section {* Multiset of Elements of Binary Tree *}
+section \<open>Multiset of Elements of Binary Tree\<close>
 
 theory Tree_Multiset
 imports Multiset Tree
 begin
 
-text{* Kept separate from theory @{theory Tree} to avoid importing all of
+text\<open>Kept separate from theory @{theory Tree} to avoid importing all of
 theory @{theory Multiset} into @{theory Tree}. Should be merged if
-@{theory Multiset} ever becomes part of @{theory Main}. *}
+@{theory Multiset} ever becomes part of @{theory Main}.\<close>
 
 fun mset_tree :: "'a tree \<Rightarrow> 'a multiset" where
 "mset_tree Leaf = {#}" |