src/HOL/Algebra/Bij.thy
changeset 67443 3abf6a722518
parent 67091 1393c2340eec
child 68687 2976a4a3b126
--- a/src/HOL/Algebra/Bij.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Algebra/Bij.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -10,7 +10,7 @@
 
 definition
   Bij :: "'a set \<Rightarrow> ('a \<Rightarrow> 'a) set"
-    \<comment>\<open>Only extensional functions, since otherwise we get too many.\<close>
+    \<comment> \<open>Only extensional functions, since otherwise we get too many.\<close>
    where "Bij S = extensional S \<inter> {f. bij_betw f S S}"
 
 definition