diff -r b7d051e25d9d -r ac6a69b0f634 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: \\x. f \$\ (f \$\ x) = x\ begin -lemma - \f * f = 1\ +lemma \f * f = 1\ 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 + \ \syntax from permutation_syntax only present in locale specification and initial block\ end @@ -26,8 +32,7 @@ assumes swap_distinct: \a \ b \ \a \ b\ \$\ c \ c\ begin -lemma - \card (UNIV :: 'a set) \ 2\ +lemma \card (UNIV :: 'a set) \ 2\ proof (rule ccontr) fix a :: 'a assume \\ card (UNIV :: 'a set) \ 2\ @@ -48,11 +53,12 @@ then have \a \ c\ \b \ c\ by auto with swap_distinct [of a b c] show False - by (simp add: \a \ b\) + by (simp add: \a \ b\) qed end -thm swap_distinct (*syntax from permutation_syntax only present in class specification and initial block*) +thm swap_distinct + \ \syntax from permutation_syntax only present in class specification and initial block\ -end \ No newline at end of file +end