src/HOL/Map.thy
changeset 67780 7655e6369c9f
parent 67091 1393c2340eec
child 68450 41de07c7a0f3
--- a/src/HOL/Map.thy	Wed Mar 07 17:39:18 2018 +0100
+++ b/src/HOL/Map.thy	Wed Mar 07 19:02:22 2018 +0100
@@ -8,7 +8,8 @@
 section \<open>Maps\<close>
 
 theory Map
-imports List
+  imports List
+  abbrevs "(=" = "\<subseteq>\<^sub>m"
 begin
 
 type_synonym ('a, 'b) "map" = "'a \<Rightarrow> 'b option" (infixr "\<rightharpoonup>" 0)