src/HOL/Library/Disjoint_Sets.thy
changeset 63145 703edebd1d92
parent 63100 aa5cffd8a606
child 63148 6a767355d1a9
--- a/src/HOL/Library/Disjoint_Sets.thy	Tue May 24 22:46:23 2016 +0200
+++ b/src/HOL/Library/Disjoint_Sets.thy	Wed May 25 11:49:40 2016 +0200
@@ -168,7 +168,7 @@
   proof (rule inj_onI, rule ccontr)
     fix x y assume A: "x \<in> A" "y \<in> A" "g x = g y" "x \<noteq> y"
     with g[of x] g[of y] have "g x \<in> f x" "g x \<in> f y" by auto
-    with A `x \<noteq> y` assms show False
+    with A \<open>x \<noteq> y\<close> assms show False
       by (auto simp: disjoint_family_on_def inj_on_def)
   qed
   from g have "g ` A \<subseteq> UNION A f" by blast