author | haftmann |
Wed, 21 Jan 2009 23:40:23 +0100 | |
changeset 29609 | a010aab5bed0 |
parent 29304 | 5c71a6da989d |
child 29820 | 07f53494cf20 |
permissions | -rw-r--r-- |
header {* Plain HOL *} theory Plain imports Datatype FunDef Record SAT 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