| author | haftmann |
| Mon, 28 May 2012 13:38:07 +0200 | |
| changeset 48003 | 1d11af40b106 |
| parent 41884 | 335895ffbd94 |
| child 49077 | 154f25a162e3 |
| 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 |
|
|
37695
71e84a203c19
introduced distinct session HOL-Codegenerator_Test
haftmann
parents:
37407
diff
changeset
|
6 |
theory Candidates |
| 21917 | 7 |
imports |
| 27421 | 8 |
Complex_Main |
|
37695
71e84a203c19
introduced distinct session HOL-Codegenerator_Test
haftmann
parents:
37407
diff
changeset
|
9 |
Library |
| 41884 | 10 |
"~~/src/HOL/Library/List_Prefix" |
| 32479 | 11 |
"~~/src/HOL/Number_Theory/Primes" |
| 35303 | 12 |
"~~/src/HOL/ex/Records" |
| 21917 | 13 |
begin |
14 |
||
| 33500 | 15 |
inductive sublist :: "'a list \<Rightarrow> 'a list \<Rightarrow> bool" where |
16 |
empty: "sublist [] xs" |
|
17 |
| drop: "sublist ys xs \<Longrightarrow> sublist ys (x # xs)" |
|
18 |
| take: "sublist ys xs \<Longrightarrow> sublist (x # ys) (x # xs)" |
|
19 |
||
20 |
code_pred sublist . |
|
21 |
||
| 33042 | 22 |
(*avoid popular infix*) |
23 |
code_reserved SML upto |
|
| 31378 | 24 |
|
| 21917 | 25 |
end |