doc-src/TutorialI/Misc/Tree.thy
author paulson
Wed, 24 May 2000 18:49:05 +0200
changeset 8962 633e1682455c
parent 8745 13b32661dde4
child 9458 c613cd06d5cf
permissions -rw-r--r--
setsum is now overloaded on plus_ac0

(*<*)
theory Tree = Main:
(*>*)

text{*\noindent
Define the datatype of binary trees
*}

datatype 'a tree = Tip | Node "'a tree" 'a "'a tree";(*<*)

consts mirror :: "'a tree \\<Rightarrow> 'a tree";
primrec
"mirror Tip = Tip"
"mirror (Node l x r) = Node (mirror l) x (mirror r)";(*>*)

text{*\noindent
and a function \isa{mirror} that mirrors a binary tree
by swapping subtrees (recursively). Prove
*}

lemma mirror_mirror: "mirror(mirror t) = t";
(*<*)
apply(induct_tac t);
apply(auto).;

end
(*>*)