| author | blanchet | 
| Wed, 04 Mar 2009 11:05:29 +0100 | |
| changeset 30242 | aea5d7fa7ef5 | 
| parent 30073 | a4ad0c08b7d9 | 
| child 30327 | 4d1185c77f4a | 
| 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