author | wenzelm |
Sat, 17 Sep 2005 18:11:21 +0200 | |
changeset 17461 | 83f1dd9d901d |
parent 17421 | 0382f6877b98 |
child 17509 | 054cd8972095 |
permissions | -rw-r--r-- |
17461 | 1 |
(* $Id$ *) |
9619 | 2 |
|
12024 | 3 |
header {* Main HOL *} |
4 |
||
15131 | 5 |
theory Main |
17461 | 6 |
imports Refute Reconstruction |
15131 | 7 |
begin |
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
8 |
|
12024 | 9 |
text {* |
10 |
Theory @{text Main} includes everything. Note that theory @{text |
|
11 |
PreList} already includes most HOL theories. |
|
12 |
*} |
|
13 |
||
17395
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
14 |
|
17461 | 15 |
subsection {* Special hacks, late package setup etc. *} |
17395
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
16 |
|
17461 | 17 |
text {* \medskip Hide the rather generic names used in theory @{text |
18 |
Commutative_Ring}. *} |
|
17395
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
19 |
|
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
20 |
hide (open) const |
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
21 |
Pc Pinj PX |
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
22 |
Pol Add Sub Mul Pow Neg |
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
23 |
add mul neg sqr pow sub |
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
24 |
norm |
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
25 |
|
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
26 |
|
17461 | 27 |
text {* \medskip Default values for rufute, see also theory @{text |
28 |
Refute}. |
|
16770
1f1b1fae30e4
Auxiliary functions to be used in generated code are now defined using "attach".
berghofe
parents:
16635
diff
changeset
|
29 |
*} |
13093
ab0335307905
code generator: wfrec combinator is now implemented by ML function wf_rec.
berghofe
parents:
12554
diff
changeset
|
30 |
|
17461 | 31 |
refute_params |
32 |
["itself"=1, |
|
33 |
minsize=1, |
|
34 |
maxsize=8, |
|
35 |
maxvars=10000, |
|
36 |
maxtime=60, |
|
37 |
satsolver="auto"] |
|
12554
671b4d632c34
Declared characteristic equations for < on nat for code generation.
berghofe
parents:
12439
diff
changeset
|
38 |
|
17395
a05e20f6a31a
hide the rather generic names used in theory Commutative_Ring;
wenzelm
parents:
17386
diff
changeset
|
39 |
|
17461 | 40 |
text {* \medskip Clause setup: installs \emph{all} simprules and |
41 |
claset rules into the clause cache; cf.\ theory @{text |
|
42 |
Reconstruction}. *} |
|
14350 | 43 |
|
17461 | 44 |
setup ResAxioms.clause_setup |
14350 | 45 |
|
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
46 |
end |