author | wenzelm |
Thu, 01 Sep 2016 21:28:46 +0200 | |
changeset 63763 | 0f61ea70d384 |
parent 63655 | d31650b377c4 |
permissions | -rw-r--r-- |
60758 | 1 |
section \<open>Main HOL\<close> |
12024 | 2 |
|
15131 | 3 |
theory Main |
63655 | 4 |
imports Predicate_Compile Quickcheck_Narrowing Extraction Nitpick BNF_Greatest_Fixpoint Filter Conditionally_Complete_Lattices |
15131 | 5 |
begin |
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
6 |
|
60758 | 7 |
text \<open> |
29304 | 8 |
Classical Higher-order Logic -- only ``Main'', excluding real and |
9 |
complex numbers etc. |
|
60758 | 10 |
\<close> |
29304 | 11 |
|
51112 | 12 |
no_notation |
13 |
bot ("\<bottom>") and |
|
14 |
top ("\<top>") and |
|
15 |
inf (infixl "\<sqinter>" 70) and |
|
16 |
sup (infixl "\<squnion>" 65) and |
|
17 |
Inf ("\<Sqinter>_" [900] 900) and |
|
55057 | 18 |
Sup ("\<Squnion>_" [900] 900) and |
55065 | 19 |
ordLeq2 (infix "<=o" 50) and |
20 |
ordLeq3 (infix "\<le>o" 50) and |
|
21 |
ordLess2 (infix "<o" 50) and |
|
22 |
ordIso2 (infix "=o" 50) and |
|
55078 | 23 |
card_of ("|_|") and |
55057 | 24 |
csum (infixr "+c" 65) and |
25 |
cprod (infixr "*c" 80) and |
|
55086 | 26 |
cexp (infixr "^c" 90) and |
57641
dc59f147b27d
more robust notation BNF_Def.convol, which is private to main HOL, but may cause syntax ambiguities nonetheless (e.g. List.thy);
wenzelm
parents:
57208
diff
changeset
|
27 |
convol ("\<langle>(_,/ _)\<rangle>") |
51112 | 28 |
|
55087
252c7fec4119
renamed 'regular' to 'regularCard' to avoid clashes (e.g. in Meson_Test)
blanchet
parents:
55086
diff
changeset
|
29 |
hide_const (open) |
58152 | 30 |
czero cinfinite cfinite csum cone ctwo Csum cprod cexp image2 image2p vimage2p Gr Grp collect |
31 |
fsts snds setl setr convol pick_middlep fstOp sndOp csquare relImage relInvImage Succ Shift |
|
58353 | 32 |
shift proj id_bnf |
33 |
||
34 |
hide_fact (open) id_bnf_def type_definition_id_bnf_UNIV |
|
55087
252c7fec4119
renamed 'regular' to 'regularCard' to avoid clashes (e.g. in Meson_Test)
blanchet
parents:
55086
diff
changeset
|
35 |
|
61955
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
60758
diff
changeset
|
36 |
no_syntax |
51112 | 37 |
"_INF1" :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Sqinter>_./ _)" [0, 10] 10) |
38 |
"_INF" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Sqinter>_\<in>_./ _)" [0, 0, 10] 10) |
|
39 |
"_SUP1" :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Squnion>_./ _)" [0, 10] 10) |
|
40 |
"_SUP" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Squnion>_\<in>_./ _)" [0, 0, 10] 10) |
|
41 |
||
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
42 |
end |