src/HOL/Data_Structures/Tree234_Map.thy
changeset 61686 e6784939d645
parent 61640 44c9198f210c
child 61790 0494964bb226
--- a/src/HOL/Data_Structures/Tree234_Map.thy	Mon Nov 16 12:37:46 2015 +0100
+++ b/src/HOL/Data_Structures/Tree234_Map.thy	Mon Nov 16 13:08:52 2015 +0100
@@ -165,7 +165,7 @@
 
 interpretation T234_Map: Map_by_Ordered
 where empty = Leaf and lookup = lookup and update = update and delete = delete
-and inorder = inorder and wf = bal
+and inorder = inorder and inv = bal
 proof (standard, goal_cases)
   case 2 thus ?case by(simp add: lookup)
 next