doc-src/TutorialI/Overview/LNCS/FP0.thy
author haftmann
Wed, 06 Feb 2008 08:34:32 +0100
changeset 26041 c2e15e65165f
parent 16417 9bc16273c2d4
permissions -rw-r--r--
locales ACf, ACIf, ACIfSL and ACIfSLlin have been abandoned in favour of the existing algebraic classes ab_semigroup_mult, ab_semigroup_idem_mult, lower_semilattice (resp. uper_semilattice) and linorder

theory FP0 imports PreList begin

datatype 'a list = Nil                          ("[]")
                 | Cons 'a "'a list"            (infixr "#" 65)

consts app :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list"   (infixr "@" 65)
       rev :: "'a list \<Rightarrow> 'a list"

primrec
"[] @ ys       = ys"
"(x # xs) @ ys = x # (xs @ ys)"

primrec
"rev []        = []"
"rev (x # xs)  = (rev xs) @ (x # [])"

theorem rev_rev [simp]: "rev(rev xs) = xs"
(*<*)oops(*>*)text_raw{*\isanewline\isanewline*}

end