src/HOL/Set.thy
changeset 78258 71366be2c647
parent 78230 7ca11a7ace41
child 79099 05a753360b25
--- a/src/HOL/Set.thy	Wed Jul 05 16:50:07 2023 +0100
+++ b/src/HOL/Set.thy	Thu Jul 06 16:59:12 2023 +0100
@@ -719,6 +719,9 @@
 lemma Compl_eq_Diff_UNIV: "- A = (UNIV - A)"
   by blast
 
+abbreviation sym_diff :: "'a set \<Rightarrow> 'a set \<Rightarrow> 'a set" where
+  "sym_diff A B \<equiv> ((A - B) \<union> (B-A))"
+
 
 subsubsection \<open>Augmenting a set -- \<^const>\<open>insert\<close>\<close>