4 imports Predicate_Compile Nitpick Extraction Lifting_Sum List_Prefix Coinduction Cardinal_Arithmetic_FP
8 Classical Higher-order Logic -- only ``Main'', excluding real and
12 text {* See further \cite{Nipkow-et-al:2002:tutorial} *}
17 inf (infixl "\<sqinter>" 70) and
18 sup (infixl "\<squnion>" 65) and
19 Inf ("\<Sqinter>_" [900] 900) and
20 Sup ("\<Squnion>_" [900] 900)
23 "_INF1" :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Sqinter>_./ _)" [0, 10] 10)
24 "_INF" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Sqinter>_\<in>_./ _)" [0, 0, 10] 10)
25 "_SUP1" :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Squnion>_./ _)" [0, 10] 10)
26 "_SUP" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b" ("(3\<Squnion>_\<in>_./ _)" [0, 0, 10] 10)