diff -r a80d8ec6c998 -r 3dda49e08b9d src/HOL/Quickcheck_Random.thy --- a/src/HOL/Quickcheck_Random.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/HOL/Quickcheck_Random.thy Fri Jan 04 23:22:53 2019 +0100 @@ -127,7 +127,7 @@ subsection \Complex generators\ -text \Towards @{typ "'a \ 'b"}\ +text \Towards \<^typ>\'a \ 'b\\ axiomatization random_fun_aux :: "typerep \ typerep \ ('a \ 'a \ bool) \ ('a \ term) \ (Random.seed \ ('b \ (unit \ term)) \ Random.seed) @@ -217,7 +217,7 @@ code_printing constant random_fun_aux \ (Quickcheck) "Random'_Generators.random'_fun" - \ \With enough criminal energy this can be abused to derive @{prop False}; + \ \With enough criminal energy this can be abused to derive \<^prop>\False\; for this reason we use a distinguished target \Quickcheck\ not spoiling the regular trusted code generation\