| author | bulwahn | 
| Mon, 22 Mar 2010 08:30:13 +0100 | |
| changeset 35890 | 14a0993fe64b | 
| parent 35617 | a6528fb99641 | 
| child 36115 | 6601c227c5bf | 
| 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  | 
|
| 35303 | 11  | 
"~~/src/HOL/Decision_Procs/Commutative_Ring_Complete"  | 
12  | 
Dlist  | 
|
| 31849 | 13  | 
Fset  | 
| 27421 | 14  | 
Enum  | 
| 21917 | 15  | 
List_Prefix  | 
16  | 
Nat_Infinity  | 
|
| 
24433
 
4a405457e9d6
added explicit equation for equality of nested environments
 
haftmann 
parents: 
24423 
diff
changeset
 | 
17  | 
Nested_Environment  | 
| 26515 | 18  | 
Option_ord  | 
| 21917 | 19  | 
Permutation  | 
| 32479 | 20  | 
"~~/src/HOL/Number_Theory/Primes"  | 
| 21917 | 21  | 
Product_ord  | 
| 35303 | 22  | 
"~~/src/HOL/ex/Records"  | 
| 21917 | 23  | 
SetsAndFunctions  | 
| 35617 | 24  | 
Table  | 
| 31459 | 25  | 
Tree  | 
| 21917 | 26  | 
While_Combinator  | 
27  | 
Word  | 
|
28  | 
begin  | 
|
29  | 
||
| 33500 | 30  | 
inductive sublist :: "'a list \<Rightarrow> 'a list \<Rightarrow> bool" where  | 
31  | 
empty: "sublist [] xs"  | 
|
32  | 
| drop: "sublist ys xs \<Longrightarrow> sublist ys (x # xs)"  | 
|
33  | 
| take: "sublist ys xs \<Longrightarrow> sublist (x # ys) (x # xs)"  | 
|
34  | 
||
35  | 
code_pred sublist .  | 
|
36  | 
||
| 33042 | 37  | 
(*avoid popular infix*)  | 
38  | 
code_reserved SML upto  | 
|
| 31378 | 39  | 
|
| 21917 | 40  | 
end  |