src/HOL/ex/Quickcheck_Generators.thy
changeset 30364 577edc39b501
parent 30280 eb98b49ef835
child 30945 0418e9bffbba
--- a/src/HOL/ex/Quickcheck_Generators.thy	Sun Mar 08 17:19:15 2009 +0100
+++ b/src/HOL/ex/Quickcheck_Generators.thy	Sun Mar 08 17:26:14 2009 +0100
@@ -138,7 +138,7 @@
     let
       val this_ty = Type (hd tycos, map TFree vs);
       val this_ty' = StateMonad.liftT (term_ty this_ty) @{typ seed};
-      val random_name = NameSpace.base_name @{const_name random};
+      val random_name = Long_Name.base_name @{const_name random};
       val random'_name = random_name ^ "_" ^ Class.type_name (hd tycos) ^ "'";
       fun random ty = Sign.mk_const thy (@{const_name random}, [ty]);
       val random' = Free (random'_name,