author | Thomas Sewell <tsewell@nicta.com.au> |
Fri, 11 Sep 2009 20:58:29 +1000 | |
changeset 32749 | 3282c12a856c |
parent 32479 | 521cc9bf2958 |
child 33042 | ddf1f03a9ad9 |
permissions | -rw-r--r-- |
31378 | 1 |
|
2 |
(* Author: Florian Haftmann, TU Muenchen *) |
|
21917 | 3 |
|
31378 | 4 |
header {* A huge collection of equations to generate code from *} |
21917 | 5 |
|
31378 | 6 |
theory Codegenerator_Candidates |
21917 | 7 |
imports |
27421 | 8 |
Complex_Main |
21917 | 9 |
AssocList |
10 |
Binomial |
|
31849 | 11 |
Fset |
21917 | 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 |
32479 | 19 |
"~~/src/HOL/Number_Theory/Primes" |
21917 | 20 |
Product_ord |
21 |
SetsAndFunctions |
|
31459 | 22 |
Tree |
21917 | 23 |
While_Combinator |
24 |
Word |
|
27421 | 25 |
"~~/src/HOL/ex/Commutative_Ring_Complete" |
26 |
"~~/src/HOL/ex/Records" |
|
21917 | 27 |
begin |
28 |
||
31378 | 29 |
(*avoid popular infixes*) |
30 |
code_reserved SML union inter upto |
|
31 |
||
21917 | 32 |
end |