src/HOL/Data_Structures/Tree2.thy
changeset 62390 842917225d56
parent 62160 ff20b44b2fc8
child 62650 7e6bb43e7217
--- a/src/HOL/Data_Structures/Tree2.thy	Tue Feb 23 15:37:18 2016 +0100
+++ b/src/HOL/Data_Structures/Tree2.thy	Tue Feb 23 16:25:08 2016 +0100
@@ -14,4 +14,4 @@
 "height Leaf = 0" |
 "height (Node _ l a r) = max (height l) (height r) + 1"
 
-end
\ No newline at end of file
+end