| author | haftmann |
| Sun, 22 Feb 2009 22:32:50 +0100 | |
| changeset 30063 | e7723cb4b2a6 |
| parent 29837 | eb7e62c0f53c |
| child 30073 | a4ad0c08b7d9 |
| permissions | -rw-r--r-- |
header {* Plain HOL *} theory Plain imports Datatype FunDef Record Extraction Divides Fact 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