src/HOL/Library/AList_Mapping.thy
changeset 46238 9ace9e5b79be
parent 46171 19f68d7671f0
child 49929 70300f1b6835
--- a/src/HOL/Library/AList_Mapping.thy	Tue Jan 17 09:38:30 2012 +0100
+++ b/src/HOL/Library/AList_Mapping.thy	Tue Jan 17 10:45:42 2012 +0100
@@ -5,7 +5,7 @@
 header {* Implementation of mappings with Association Lists *}
 
 theory AList_Mapping
-imports AList_Impl Mapping
+imports AList Mapping
 begin
 
 definition Mapping :: "('a \<times> 'b) list \<Rightarrow> ('a, 'b) mapping" where
@@ -30,11 +30,11 @@
   by (cases xs) (simp_all add: is_empty_def null_def)
 
 lemma update_Mapping [code]:
-  "Mapping.update k v (Mapping xs) = Mapping (AList_Impl.update k v xs)"
+  "Mapping.update k v (Mapping xs) = Mapping (AList.update k v xs)"
   by (rule mapping_eqI) (simp add: update_conv')
 
 lemma delete_Mapping [code]:
-  "Mapping.delete k (Mapping xs) = Mapping (AList_Impl.delete k xs)"
+  "Mapping.delete k (Mapping xs) = Mapping (AList.delete k xs)"
   by (rule mapping_eqI) (simp add: delete_conv')
 
 lemma ordered_keys_Mapping [code]: