| author | nipkow | 
| Mon, 09 Feb 2009 18:50:10 +0100 | |
| changeset 29849 | a2baf1b221be | 
| parent 29820 | 07f53494cf20 | 
| child 29837 | eb7e62c0f53c | 
| permissions | -rw-r--r-- | 
header {* Plain HOL *} theory Plain imports Datatype FunDef Record Extraction Divides begin text {* Plain bootstrap of fundamental HOL tools and packages; does not include @{text Hilbert_Choice}. *} instance option :: (finite) finite by default (simp add: insert_None_conv_UNIV [symmetric]) ML {* path_add "~~/src/HOL/Library" *} end