src/Doc/Isar_Ref/HOL_Specific.thy
changeset 68484 59793df7f853
parent 68254 3a7f257dcac7
child 69484 ed6b100a9c7d
equal deleted inserted replaced
68483:087d32a40129 68484:59793df7f853
  1873 
  1873 
  1874     \<^descr>[\<open>random\<close>] The operation @{const Quickcheck_Random.random} of the type
  1874     \<^descr>[\<open>random\<close>] The operation @{const Quickcheck_Random.random} of the type
  1875     class @{class random} generates a pseudo-random value of the given size
  1875     class @{class random} generates a pseudo-random value of the given size
  1876     and a lazy term reconstruction of the value in the type @{typ
  1876     and a lazy term reconstruction of the value in the type @{typ
  1877     Code_Evaluation.term}. A pseudo-randomness generator is defined in theory
  1877     Code_Evaluation.term}. A pseudo-randomness generator is defined in theory
  1878     @{theory Random}.
  1878     @{theory HOL.Random}.
  1879 
  1879 
  1880     \<^descr>[\<open>narrowing\<close>] implements Haskell's Lazy Smallcheck @{cite
  1880     \<^descr>[\<open>narrowing\<close>] implements Haskell's Lazy Smallcheck @{cite
  1881     "runciman-naylor-lindblad"} using the type classes @{class narrowing} and
  1881     "runciman-naylor-lindblad"} using the type classes @{class narrowing} and
  1882     @{class partial_term_of}. Variables in the current goal are initially
  1882     @{class partial_term_of}. Variables in the current goal are initially
  1883     represented as symbolic variables. If the execution of the goal tries to
  1883     represented as symbolic variables. If the execution of the goal tries to
  1995   third argument inherits the allowance of coercsion insertion from the
  1995   third argument inherits the allowance of coercsion insertion from the
  1996   position of the constant \<open>c\<close> (policy \<open>0\<close>). The standard usage of policies is
  1996   position of the constant \<open>c\<close> (policy \<open>0\<close>). The standard usage of policies is
  1997   the definition of syntatic constructs (usually extralogical, i.e., processed
  1997   the definition of syntatic constructs (usually extralogical, i.e., processed
  1998   and stripped during type inference), that should not be destroyed by the
  1998   and stripped during type inference), that should not be destroyed by the
  1999   insertion of coercions (see, for example, the setup for the case syntax in
  1999   insertion of coercions (see, for example, the setup for the case syntax in
  2000   @{theory Ctr_Sugar}).
  2000   @{theory HOL.Ctr_Sugar}).
  2001 
  2001 
  2002   \<^descr> @{attribute (HOL) "coercion_enabled"} enables the coercion inference
  2002   \<^descr> @{attribute (HOL) "coercion_enabled"} enables the coercion inference
  2003   algorithm.
  2003   algorithm.
  2004 \<close>
  2004 \<close>
  2005 
  2005