diff -r 5eb932e604a2 -r eab6ce8368fa src/Doc/Isar_Ref/HOL_Specific.thy --- a/src/Doc/Isar_Ref/HOL_Specific.thy Wed Jan 10 15:21:49 2018 +0100 +++ b/src/Doc/Isar_Ref/HOL_Specific.thy Wed Jan 10 15:25:09 2018 +0100 @@ -1452,7 +1452,7 @@ \Quotient_thm\). Optional theorems \pcr_def\ and \pcr_cr_eq_thm\ can be specified to register the parametrized correspondence relation for \\\. E.g.\ for @{typ "'a dlist"}, \pcr_def\ is \pcr_dlist A \ list_all2 A \\ - cr_dlist\ and \pcr_cr_eq_thm\ is \pcr_dlist (op =) = (op =)\. This attribute + cr_dlist\ and \pcr_cr_eq_thm\ is \pcr_dlist (=) = (=)\. This attribute is rather used for low-level manipulation with set-up of the Lifting package because using of the bundle \\.lifting\ together with the commands @{command (HOL) lifting_forget} and @{command (HOL) lifting_update} is preferred for @@ -1539,7 +1539,7 @@ Lemmas involving predicates on relations can also be registered using the same attribute. For example: - \bi_unique A \ (list_all2 A ===> op =) distinct distinct\ \\ + \bi_unique A \ (list_all2 A ===> (=)) distinct distinct\ \\ \\bi_unique A; bi_unique B\ \ bi_unique (rel_prod A B)\ Preservation of predicates on relations (\bi_unique, bi_total, right_unique, @@ -1555,7 +1555,7 @@ quantifiers are transferred. \<^descr> @{attribute (HOL) relator_eq} attribute collects identity laws for - relators of various type constructors, e.g. @{term "rel_set (op =) = (op =)"}. + relators of various type constructors, e.g. @{term "rel_set (=) = (=)"}. The @{method (HOL) transfer} method uses these lemmas to infer transfer rules for non-polymorphic constants on the fly. For examples see \<^file>\~~/src/HOL/Lifting_Set.thy\ or \<^file>\~~/src/HOL/Lifting.thy\. This property @@ -1894,7 +1894,7 @@ @{term "Quickcheck_Narrowing.sum (Quickcheck_Narrowing.cons []) (Quickcheck_Narrowing.apply (Quickcheck_Narrowing.apply - (Quickcheck_Narrowing.cons (op #)) + (Quickcheck_Narrowing.cons (#)) narrowing) narrowing)"}. If a symbolic variable of type @{typ "_ list"} is evaluated, it is @@ -1909,7 +1909,7 @@ "Quickcheck_Narrowing.Narrowing_constructor i args"}, where @{term "i :: integer"} denotes the index in the sum of refinements. In the above example for lists, @{term "0"} corresponds to @{term "[]"} and @{term "1"} - to @{term "op #"}. + to @{term "(#)"}. The command @{command (HOL) "code_datatype"} sets up @{const partial_term_of} such that the @{term "i"}-th refinement is interpreted as