thys/Chap03.thy
changeset 52 d67149236738
parent 51 3810b37511cb
child 54 45274393f28c
equal deleted inserted replaced
51:3810b37511cb 52:d67149236738
       
     1 (* test *)
     1 theory Chap03
     2 theory Chap03
     2 imports Main
     3 imports Main
     3 begin
     4 begin
     4 
     5 
     5 lemma "\<lbrakk> xs @ zs = ys @ xs; [] @ xs = [] @ [] \<rbrakk> \<Longrightarrow> ys = zs"
     6 lemma "\<lbrakk> xs @ zs = ys @ xs; [] @ xs = [] @ [] \<rbrakk> \<Longrightarrow> ys = zs"