src/HOL/Quickcheck_Random.thy
changeset 55147 bce3dbc11f95
parent 52435 6646bb548c6b
child 58152 6fe60a9a5bad
--- a/src/HOL/Quickcheck_Random.thy	Sat Jan 25 23:50:49 2014 +0100
+++ b/src/HOL/Quickcheck_Random.thy	Sat Jan 25 23:50:49 2014 +0100
@@ -9,7 +9,7 @@
 notation fcomp (infixl "\<circ>>" 60)
 notation scomp (infixl "\<circ>\<rightarrow>" 60)
 
-setup {* Code_Target.extend_target ("Quickcheck", (Code_Runtime.target, K I)) *}
+setup {* Code_Target.extend_target ("Quickcheck", (Code_Runtime.target, I)) *}
 
 subsection {* Catching Match exceptions *}