changeset 55017 | 2df6ad1dbd66 |
parent 44918 | 6a80fbc4e72c |
child 58112 | 8081087096ad |
--- a/src/HOL/Induct/Sexp.thy Thu Jan 16 15:47:33 2014 +0100 +++ b/src/HOL/Induct/Sexp.thy Thu Jan 16 16:20:17 2014 +0100 @@ -6,7 +6,9 @@ structures by hand. *) -theory Sexp imports Main "~~/src/HOL/Library/Wfrec" begin +theory Sexp +imports Main +begin type_synonym 'a item = "'a Datatype.item" abbreviation "Leaf == Datatype.Leaf"