src/HOL/ex/Seq.thy
changeset 58310 91ea607a34d8
parent 58249 180f1b3508ed
child 58616 4257a7f2bf39
equal deleted inserted replaced
58309:a09ec6daaa19 58310:91ea607a34d8
     6 
     6 
     7 theory Seq
     7 theory Seq
     8 imports Main
     8 imports Main
     9 begin
     9 begin
    10 
    10 
    11 datatype_new 'a seq = Empty | Seq 'a "'a seq"
    11 datatype 'a seq = Empty | Seq 'a "'a seq"
    12 
    12 
    13 fun conc :: "'a seq \<Rightarrow> 'a seq \<Rightarrow> 'a seq"
    13 fun conc :: "'a seq \<Rightarrow> 'a seq \<Rightarrow> 'a seq"
    14 where
    14 where
    15   "conc Empty ys = ys"
    15   "conc Empty ys = ys"
    16 | "conc (Seq x xs) ys = Seq x (conc xs ys)"
    16 | "conc (Seq x xs) ys = Seq x (conc xs ys)"