src/HOL/Data_Structures/AA_Set.thy
changeset 68440 6826718f732d
parent 68431 b294e095f64c
child 69505 cc2d676d5395
--- a/src/HOL/Data_Structures/AA_Set.thy	Wed Jun 13 11:53:25 2018 +0200
+++ b/src/HOL/Data_Structures/AA_Set.thy	Wed Jun 13 15:24:20 2018 +0200
@@ -485,7 +485,7 @@
   (auto simp: del_list_simps inorder_adjust pre_adj_if_postL pre_adj_if_postR 
               post_split_max post_delete split_maxD split: prod.splits)
 
-interpretation I: Set_by_Ordered
+interpretation S: Set_by_Ordered
 where empty = empty and isin = isin and insert = insert and delete = delete
 and inorder = inorder and inv = invar
 proof (standard, goal_cases)