src/HOL/ex/AVL.thy
changeset 11701 3d51fbf81c17
parent 8797 b55e2354d71e
child 11908 82f68fd05094
--- a/src/HOL/ex/AVL.thy	Fri Oct 05 21:50:37 2001 +0200
+++ b/src/HOL/ex/AVL.thy	Fri Oct 05 21:52:39 2001 +0200
@@ -6,7 +6,7 @@
 AVL trees: at the moment only insertion.
 This version works exclusively with nat.
 Balance check could be simplified by working with int:
-"isbal (MKT n l r) = (abs(int(height l) - int(height r)) <= #1 &
+"isbal (MKT n l r) = (abs(int(height l) - int(height r)) <= Numeral1 &
                       isbal l & isbal r)"
 *)