changeset 61585 | a9599d3d7610 |
parent 60808 | fd26519b1a6a |
child 62160 | ff20b44b2fc8 |
--- a/src/HOL/Library/Tree.thy Thu Nov 05 10:35:37 2015 +0100 +++ b/src/HOL/Library/Tree.thy Thu Nov 05 10:39:49 2015 +0100 @@ -146,7 +146,7 @@ (heap l \<and> heap r \<and> (\<forall>x \<in> set_tree l \<union> set_tree r. m \<le> x))" -subsection "Function @{text mirror}" +subsection "Function \<open>mirror\<close>" fun mirror :: "'a tree \<Rightarrow> 'a tree" where "mirror \<langle>\<rangle> = Leaf" |