src/ZF/UNITY/Merge.thy
changeset 67443 3abf6a722518
parent 61798 27f3c10b0b50
child 76213 e44d86131648
--- a/src/ZF/UNITY/Merge.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/ZF/UNITY/Merge.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -64,10 +64,10 @@
 
 (** State definitions.  OUTPUT variables are locals **)
 locale merge =
-  fixes In   \<comment>\<open>merge's INPUT histories: streams to merge\<close>
-    and Out  \<comment>\<open>merge's OUTPUT history: merged items\<close>
-    and iOut \<comment>\<open>merge's OUTPUT history: origins of merged items\<close>
-    and A    \<comment>\<open>the type of items being merged\<close>
+  fixes In   \<comment> \<open>merge's INPUT histories: streams to merge\<close>
+    and Out  \<comment> \<open>merge's OUTPUT history: merged items\<close>
+    and iOut \<comment> \<open>merge's OUTPUT history: origins of merged items\<close>
+    and A    \<comment> \<open>the type of items being merged\<close>
     and M
  assumes var_assumes [simp]:
            "(\<forall>n. In(n):var) & Out \<in> var & iOut \<in> var"