src/HOL/ex/Codegenerator_Candidates.thy
author haftmann
Sat, 06 Mar 2010 15:31:30 +0100
changeset 35617 a6528fb99641
parent 35303 816e48d60b13
child 36115 6601c227c5bf
permissions -rw-r--r--
added Table.thy
     1 
     2 (* Author: Florian Haftmann, TU Muenchen *)
     3 
     4 header {* A huge collection of equations to generate code from *}
     5 
     6 theory Codegenerator_Candidates
     7 imports
     8   Complex_Main
     9   AssocList
    10   Binomial
    11   "~~/src/HOL/Decision_Procs/Commutative_Ring_Complete"
    12   Dlist
    13   Fset
    14   Enum
    15   List_Prefix
    16   Nat_Infinity
    17   Nested_Environment
    18   Option_ord
    19   Permutation
    20   "~~/src/HOL/Number_Theory/Primes"
    21   Product_ord
    22   "~~/src/HOL/ex/Records"
    23   SetsAndFunctions
    24   Table
    25   Tree
    26   While_Combinator
    27   Word
    28 begin
    29 
    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 
    37 (*avoid popular infix*)
    38 code_reserved SML upto
    39 
    40 end