doc-src/TutorialI/Misc/Tree.thy
changeset 16417 9bc16273c2d4
parent 11456 7eb63f63e6c6
child 27015 f8537d69f514
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     1 (*<*)
     1 (*<*)
     2 theory Tree = Main:
     2 theory Tree imports Main begin
     3 (*>*)
     3 (*>*)
     4 
     4 
     5 text{*\noindent
     5 text{*\noindent
     6 Define the datatype of \rmindex{binary trees}:
     6 Define the datatype of \rmindex{binary trees}:
     7 *}
     7 *}