diff -r 2025a17bb20f -r adaa430fc0f7 src/Doc/Isar_Ref/HOL_Specific.thy --- a/src/Doc/Isar_Ref/HOL_Specific.thy Fri Feb 06 19:17:17 2015 +0100 +++ b/src/Doc/Isar_Ref/HOL_Specific.thy Fri Feb 06 17:57:03 2015 +0100 @@ -1592,7 +1592,7 @@ \end{matharray} @{rail \ - @@{command (HOL) setup_lifting} ('(' 'no_code' ')')? \ + @@{command (HOL) setup_lifting} \ @{syntax thmref} @{syntax thmref}? (@'parametric' @{syntax thmref})?; \} @@ -1645,9 +1645,6 @@ The command @{command (HOL) "setup_lifting"} also sets up the code generator for the new type. Later on, when a new constant is defined by @{command (HOL) "lift_definition"}, the Lifting package proves and registers a code equation (if there is one) for the new constant. - If the option @{text "no_code"} is specified, the Lifting package does not set up the code - generator and as a consequence no code equations involving an abstract type are registered - by @{command (HOL) "lift_definition"}. \item @{command (HOL) "lift_definition"} @{text "f :: \"} @{keyword (HOL) "is"} @{text t} Defines a new function @{text f} with an abstract type @{text \}