tuned comments and whitespace (see also 589645894305);
authorwenzelm
Sun, 18 Aug 2024 15:41:55 +0200
changeset 80723 ac6a69b0f634
parent 80722 b7d051e25d9d
child 80724 f9b31d348fde
tuned comments and whitespace (see also 589645894305);
src/HOL/ex/Specifications_with_bundle_mixins.thy
--- a/src/HOL/ex/Specifications_with_bundle_mixins.thy	Sun Aug 18 15:29:18 2024 +0200
+++ b/src/HOL/ex/Specifications_with_bundle_mixins.thy	Sun Aug 18 15:41:55 2024 +0200
@@ -1,3 +1,9 @@
+(*  Title:      HOL/ex/Specifications_with_bundle_mixins.thy
+    Author:     Florian Haftmann
+
+Specifications with 'bundle' mixins.
+*)
+
 theory Specifications_with_bundle_mixins
   imports "HOL-Combinatorics.Perm"
 begin
@@ -7,8 +13,7 @@
   assumes involutory: \<open>\<And>x. f \<langle>$\<rangle> (f \<langle>$\<rangle> x) = x\<close>
 begin
 
-lemma
-  \<open>f * f = 1\<close>
+lemma \<open>f * f = 1\<close>
   using involutory
   by (simp add: perm_eq_iff apply_sequence)
 
@@ -17,7 +22,8 @@
 context involutory
 begin
 
-thm involutory (*syntax from permutation_syntax only present in locale specification and initial block*)
+thm involutory
+  \<comment> \<open>syntax from permutation_syntax only present in locale specification and initial block\<close>
 
 end
 
@@ -26,8 +32,7 @@
   assumes swap_distinct: \<open>a \<noteq> b \<Longrightarrow> \<langle>a \<leftrightarrow> b\<rangle> \<langle>$\<rangle> c \<noteq> c\<close>
 begin
 
-lemma
-  \<open>card (UNIV :: 'a set) \<le> 2\<close>
+lemma \<open>card (UNIV :: 'a set) \<le> 2\<close>
 proof (rule ccontr)
   fix a :: 'a
   assume \<open>\<not> card (UNIV :: 'a set) \<le> 2\<close>
@@ -48,11 +53,12 @@
   then have \<open>a \<noteq> c\<close> \<open>b \<noteq> c\<close>
     by auto
   with swap_distinct [of a b c] show False
-    by (simp add: \<open>a \<noteq> b\<close>) 
+    by (simp add: \<open>a \<noteq> b\<close>)
 qed
 
 end
 
-thm swap_distinct (*syntax from permutation_syntax only present in class specification and initial block*)
+thm swap_distinct
+  \<comment> \<open>syntax from permutation_syntax only present in class specification and initial block\<close>
 
-end
\ No newline at end of file
+end