src/Doc/Datatypes/Datatypes.thy
changeset 53691 fa103abdbade
parent 53677 b51ebeda414d
child 53694 7b453b619b5f
equal deleted inserted replaced
53690:a3ad5a0350f9 53691:fa103abdbade
  1719     begin
  1719     begin
  1720 (*>*)
  1720 (*>*)
  1721     primcorec lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where
  1721     primcorec lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where
  1722       "lnull xs \<Longrightarrow> lnull ys \<Longrightarrow> lnull (lappend xs ys)" |
  1722       "lnull xs \<Longrightarrow> lnull ys \<Longrightarrow> lnull (lappend xs ys)" |
  1723       "lhd (lappend xs ys) = lhd (if lnull xs then ys else xs)" |
  1723       "lhd (lappend xs ys) = lhd (if lnull xs then ys else xs)" |
  1724       "ltl (lappend xs ys) = ltl (if lnull xs then ys else xs)"
  1724       "ltl (lappend xs ys) = (if xs = LNil then ltl ys else lappend (ltl xs) ys)"
  1725     .
  1725     .
  1726 (*<*)
  1726 (*<*)
  1727     end
  1727     end
  1728 (*>*)
  1728 (*>*)
  1729 
  1729