diff -r 5eb932e604a2 -r eab6ce8368fa src/HOL/Library/Countable_Set_Type.thy --- a/src/HOL/Library/Countable_Set_Type.thy Wed Jan 10 15:21:49 2018 +0100 +++ b/src/HOL/Library/Countable_Set_Type.thy Wed Jan 10 15:25:09 2018 +0100 @@ -81,7 +81,7 @@ lemma less_cset_transfer[transfer_rule]: includes lifting_syntax assumes [transfer_rule]: "bi_unique A" - shows "((pcr_cset A) ===> (pcr_cset A) ===> op =) op \ op <" + shows "((pcr_cset A) ===> (pcr_cset A) ===> (=)) (\) (<)" unfolding less_cset_def[abs_def] psubset_eq[abs_def] by transfer_prover lift_definition sup_cset :: "'a cset \ 'a cset \ 'a cset" @@ -104,12 +104,12 @@ abbreviation cInt :: "'a cset \ 'a cset \ 'a cset" where "cInt xs ys \ inf xs ys" abbreviation cDiff :: "'a cset \ 'a cset \ 'a cset" where "cDiff xs ys \ minus xs ys" -lift_definition cin :: "'a \ 'a cset \ bool" is "op \" parametric member_transfer +lift_definition cin :: "'a \ 'a cset \ bool" is "(\)" parametric member_transfer . lift_definition cinsert :: "'a \ 'a cset \ 'a cset" is insert parametric Lifting_Set.insert_transfer by (rule countable_insert) abbreviation csingle :: "'a \ 'a cset" where "csingle x \ cinsert x cempty" -lift_definition cimage :: "('a \ 'b) \ 'a cset \ 'b cset" is "op `" parametric image_transfer +lift_definition cimage :: "('a \ 'b) \ 'a cset \ 'b cset" is "(`)" parametric image_transfer by (rule countable_image) lift_definition cBall :: "'a cset \ ('a \ bool) \ bool" is Ball parametric Ball_transfer . lift_definition cBex :: "'a cset \ ('a \ bool) \ bool" is Bex parametric Bex_transfer . @@ -480,15 +480,15 @@ unfolding rel_fun_def rel_cset_iff by blast lemma cBall_parametric [transfer_rule]: - "(rel_cset A ===> (A ===> op =) ===> op =) cBall cBall" + "(rel_cset A ===> (A ===> (=)) ===> (=)) cBall cBall" unfolding rel_cset_iff rel_fun_def by blast lemma cBex_parametric [transfer_rule]: - "(rel_cset A ===> (A ===> op =) ===> op =) cBex cBex" + "(rel_cset A ===> (A ===> (=)) ===> (=)) cBex cBex" unfolding rel_cset_iff rel_fun_def by blast lemma rel_cset_parametric [transfer_rule]: - "((A ===> B ===> op =) ===> rel_cset A ===> rel_cset B ===> op =) rel_cset rel_cset" + "((A ===> B ===> (=)) ===> rel_cset A ===> rel_cset B ===> (=)) rel_cset rel_cset" unfolding rel_fun_def using rel_set_transfer[unfolded rel_fun_def, rule_format, Transfer.transferred, where A = A and B = B] by simp @@ -496,7 +496,7 @@ text \Rules requiring bi-unique, bi-total or right-total relations\ lemma cin_parametric [transfer_rule]: - "bi_unique A \ (A ===> rel_cset A ===> op =) cin cin" + "bi_unique A \ (A ===> rel_cset A ===> (=)) cin cin" unfolding rel_fun_def rel_cset_iff bi_unique_def by metis lemma cInt_parametric [transfer_rule]: @@ -511,7 +511,7 @@ using Diff_transfer[unfolded rel_fun_def, rule_format, Transfer.transferred] by blast lemma csubset_parametric [transfer_rule]: - "bi_unique A \ (rel_cset A ===> rel_cset A ===> op =) csubset_eq csubset_eq" + "bi_unique A \ (rel_cset A ===> rel_cset A ===> (=)) csubset_eq csubset_eq" unfolding rel_fun_def using subset_transfer[unfolded rel_fun_def, rule_format, Transfer.transferred] by blast @@ -595,7 +595,7 @@ fix C f g assume eq: "\a. a \ rcset C \ f a = g a" thus "cimage f C = cimage g C" including cset.lifting by transfer force next - fix f show "rcset \ cimage f = op ` f \ rcset" including cset.lifting by transfer' fastforce + fix f show "rcset \ cimage f = (`) f \ rcset" including cset.lifting by transfer' fastforce next show "card_order natLeq" by (rule natLeq_card_order) next