src/HOL/ex/ExecutableContent.thy
changeset 31407 689df1591793
parent 31406 e23dd3aac0fb
parent 31385 bc1f918ccf68
child 31408 9f2ca03ae7b7
--- a/src/HOL/ex/ExecutableContent.thy	Tue Jun 02 23:49:46 2009 -0700
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,27 +0,0 @@
-(*  Author:     Florian Haftmann, TU Muenchen
-*)
-
-header {* A huge set of executable constants *}
-
-theory ExecutableContent
-imports
-  Complex_Main
-  AssocList
-  Binomial
-  Commutative_Ring
-  Enum
-  List_Prefix
-  Nat_Infinity
-  Nested_Environment
-  Option_ord
-  Permutation
-  Primes
-  Product_ord
-  SetsAndFunctions
-  While_Combinator
-  Word
-  "~~/src/HOL/ex/Commutative_Ring_Complete"
-  "~~/src/HOL/ex/Records"
-begin
-
-end