author | blanchet |
Mon, 20 Jan 2014 18:24:56 +0100 | |
changeset 55058 | 4e700eb471d4 |
parent 55057 | 6b0fcbeebaba |
child 55062 | 6d3fad6f01c9 |
permissions | -rw-r--r-- |
12024 | 1 |
header {* Main HOL *} |
2 |
||
15131 | 3 |
theory Main |
55058 | 4 |
imports Predicate_Compile Nitpick Extraction Lifting_Sum List_Prefix Coinduction BNF_LFP BNF_GFP |
15131 | 5 |
begin |
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
6 |
|
29304 | 7 |
text {* |
8 |
Classical Higher-order Logic -- only ``Main'', excluding real and |
|
9 |
complex numbers etc. |
|
10 |
*} |
|
11 |
||
27367 | 12 |
text {* See further \cite{Nipkow-et-al:2002:tutorial} *} |
25964 | 13 |
|
51112 | 14 |
no_notation |
15 |
bot ("\<bottom>") and |
|
16 |
top ("\<top>") and |
|
17 |
inf (infixl "\<sqinter>" 70) and |
|
18 |
sup (infixl "\<squnion>" 65) and |
|
19 |
Inf ("\<Sqinter>_" [900] 900) and |
|
55057 | 20 |
Sup ("\<Squnion>_" [900] 900) and |
21 |
ordLeq2 ("<=o") and |
|
22 |
ordLeq3 ("\<le>o") and |
|
23 |
ordLess2 ("<o") and |
|
24 |
ordIso2 ("=o") and |
|
25 |
csum (infixr "+c" 65) and |
|
26 |
cprod (infixr "*c" 80) and |
|
27 |
cexp (infixr "^c" 90) |
|
51112 | 28 |
|
29 |
no_syntax (xsymbols) |
|
30 |
"_INF1" :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Sqinter>_./ _)" [0, 10] 10) |
|
31 |
"_INF" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Sqinter>_\<in>_./ _)" [0, 0, 10] 10) |
|
32 |
"_SUP1" :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Squnion>_./ _)" [0, 10] 10) |
|
33 |
"_SUP" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Squnion>_\<in>_./ _)" [0, 0, 10] 10) |
|
34 |
||
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
35 |
end |