| author | wenzelm |
| Wed, 15 Oct 2008 21:45:02 +0200 | |
| changeset 28605 | 12d6087ec18c |
| parent 28229 | 4f06fae6a55e |
| child 28952 | 15a4b2cf8c34 |
| permissions | -rw-r--r-- |
| 21917 | 1 |
(* ID: $Id$ |
2 |
Author: Florian Haftmann, TU Muenchen |
|
3 |
*) |
|
4 |
||
5 |
header {* A huge set of executable constants *}
|
|
6 |
||
7 |
theory ExecutableContent |
|
8 |
imports |
|
| 27421 | 9 |
Complex_Main |
| 21917 | 10 |
AssocList |
11 |
Binomial |
|
12 |
Commutative_Ring |
|
| 27421 | 13 |
Enum |
| 21917 | 14 |
List_Prefix |
15 |
Nat_Infinity |
|
|
24433
4a405457e9d6
added explicit equation for equality of nested environments
haftmann
parents:
24423
diff
changeset
|
16 |
Nested_Environment |
| 26515 | 17 |
Option_ord |
| 21917 | 18 |
Permutation |
19 |
Primes |
|
20 |
Product_ord |
|
21 |
SetsAndFunctions |
|
22 |
While_Combinator |
|
23 |
Word |
|
| 27421 | 24 |
"~~/src/HOL/ex/Commutative_Ring_Complete" |
25 |
"~~/src/HOL/ex/Records" |
|
| 21917 | 26 |
begin |
27 |
||
28 |
end |