src/HOL/Random.thy
changeset 57242 25aff3b8d550
parent 57225 ff69e42ccf92
child 58101 e7ebe5554281
--- a/src/HOL/Random.thy	Thu Jun 12 17:02:03 2014 +0200
+++ b/src/HOL/Random.thy	Thu Jun 12 17:02:03 2014 +0200
@@ -4,7 +4,7 @@
 header {* A HOL random engine *}
 
 theory Random
-imports Code_Numeral List
+imports List
 begin
 
 notation fcomp (infixl "\<circ>>" 60)