src/HOL/Sum_Type.thy
changeset 67443 3abf6a722518
parent 63575 b9bd9e61fd63
--- a/src/HOL/Sum_Type.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Sum_Type.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -212,7 +212,7 @@
 definition Plus :: "'a set \<Rightarrow> 'b set \<Rightarrow> ('a + 'b) set"  (infixr "<+>" 65)
   where "A <+> B = Inl ` A \<union> Inr ` B"
 
-hide_const (open) Plus \<comment> "Valuable identifier"
+hide_const (open) Plus \<comment> \<open>Valuable identifier\<close>
 
 lemma InlI [intro!]: "a \<in> A \<Longrightarrow> Inl a \<in> A <+> B"
   by (simp add: Plus_def)