| author | wenzelm | 
| Wed, 21 Sep 2011 22:18:17 +0200 | |
| changeset 45028 | d608dd8cd409 | 
| parent 41886 | aa8dce9ab8a9 | 
| child 46691 | 72d81e789106 | 
| permissions | -rw-r--r-- | 
| 27368 | 1  | 
header {* Plain HOL *}
 | 
2  | 
||
3  | 
theory Plain  | 
|
| 
40178
 
00152d17855b
reverted e7a80c6752c9 -- there's not much point in putting a diagnosis tool (as opposed to a proof method) in Plain, but more importantly Sledgehammer must be in Main to use SMT solvers
 
blanchet 
parents: 
40121 
diff
changeset
 | 
4  | 
imports Datatype FunDef Extraction Metis  | 
| 27368 | 5  | 
begin  | 
6  | 
||
| 29304 | 7  | 
text {*
 | 
8  | 
Plain bootstrap of fundamental HOL tools and packages; does not  | 
|
9  | 
  include @{text Hilbert_Choice}.
 | 
|
10  | 
*}  | 
|
11  | 
||
| 27368 | 12  | 
end  |