src/HOL/Pre_Main.thy
changeset 65814 3039d4aa7143
parent 65813 bdd17b18e103
child 65816 59b945ff5684
child 65818 94cad7590015
equal deleted inserted replaced
65813:bdd17b18e103 65814:3039d4aa7143
     1 section \<open>Main HOL\<close>
       
     2 
       
     3 theory Pre_Main
       
     4 imports Predicate_Compile Quickcheck_Narrowing Extraction Nitpick BNF_Greatest_Fixpoint Filter Conditionally_Complete_Lattices Binomial GCD
       
     5 begin
       
     6 
       
     7 text \<open>
       
     8   Classical Higher-order Logic -- only ``Main'', excluding real and
       
     9   complex numbers etc.
       
    10 \<close>
       
    11 
       
    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
       
    18   Sup ("\<Squnion>_" [900] 900) and
       
    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
       
    23   card_of ("|_|") and
       
    24   csum (infixr "+c" 65) and
       
    25   cprod (infixr "*c" 80) and
       
    26   cexp (infixr "^c" 90) and
       
    27   convol ("\<langle>(_,/ _)\<rangle>")
       
    28 
       
    29 hide_const (open)
       
    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
       
    32   shift proj id_bnf
       
    33 
       
    34 hide_fact (open) id_bnf_def type_definition_id_bnf_UNIV
       
    35 
       
    36 no_syntax
       
    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 
       
    42 end