nipkow@8563: (* Title: HOL/List.thy nipkow@8563: ID: $Id$ nipkow@8563: Author: Tobias Nipkow nipkow@8563: Copyright 2000 TU Muenchen nipkow@8563: nipkow@8563: A basis for building theory List on. Is defined separately to serve as a nipkow@8563: basis for theory ToyList in the documentation. nipkow@8563: *) wenzelm@8490: wenzelm@8490: theory PreList = nipkow@10212: Option + Wellfounded_Relations + NatSimprocs + Recdef + Record + wenzelm@10261: Relation_Power + Calculation + SVC_Oracle: wenzelm@8490: wenzelm@10261: (*belongs to theory HOL*) wenzelm@10261: declare case_split [cases type: bool] wenzelm@10261: wenzelm@10261: (*belongs to theory Wellfounded_Recursion*) wenzelm@10261: declare wf_induct [induct set: wf] wenzelm@9066: wenzelm@8490: end