# HG changeset patch # User wenzelm # Date 1494756412 -7200 # Node ID 3039d4aa71435abec8070b528c65dfb66524aa3a # Parent bdd17b18e10356f7078ff1b1946d06995597bf85 obsolete (see also bdd17b18e103, f533820e7248); diff -r bdd17b18e103 -r 3039d4aa7143 src/HOL/Main.thy --- a/src/HOL/Main.thy Fri May 12 20:03:50 2017 +0200 +++ b/src/HOL/Main.thy Sun May 14 12:06:52 2017 +0200 @@ -6,7 +6,42 @@ \ theory Main -imports Pre_Main +imports Predicate_Compile Quickcheck_Narrowing Extraction Nitpick BNF_Greatest_Fixpoint Filter Conditionally_Complete_Lattices Binomial GCD begin +text \ + Classical Higher-order Logic -- only ``Main'', excluding real and + complex numbers etc. +\ + +no_notation + bot ("\") and + top ("\") and + inf (infixl "\" 70) and + sup (infixl "\" 65) and + Inf ("\_" [900] 900) and + Sup ("\_" [900] 900) and + ordLeq2 (infix "<=o" 50) and + ordLeq3 (infix "\o" 50) and + ordLess2 (infix "(_,/ _)\") + +hide_const (open) + czero cinfinite cfinite csum cone ctwo Csum cprod cexp image2 image2p vimage2p Gr Grp collect + fsts snds setl setr convol pick_middlep fstOp sndOp csquare relImage relInvImage Succ Shift + shift proj id_bnf + +hide_fact (open) id_bnf_def type_definition_id_bnf_UNIV + +no_syntax + "_INF1" :: "pttrns \ 'b \ 'b" ("(3\_./ _)" [0, 10] 10) + "_INF" :: "pttrn \ 'a set \ 'b \ 'b" ("(3\_\_./ _)" [0, 0, 10] 10) + "_SUP1" :: "pttrns \ 'b \ 'b" ("(3\_./ _)" [0, 10] 10) + "_SUP" :: "pttrn \ 'a set \ 'b \ 'b" ("(3\_\_./ _)" [0, 0, 10] 10) + end diff -r bdd17b18e103 -r 3039d4aa7143 src/HOL/Pre_Main.thy --- a/src/HOL/Pre_Main.thy Fri May 12 20:03:50 2017 +0200 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,42 +0,0 @@ -section \Main HOL\ - -theory Pre_Main -imports Predicate_Compile Quickcheck_Narrowing Extraction Nitpick BNF_Greatest_Fixpoint Filter Conditionally_Complete_Lattices Binomial GCD -begin - -text \ - Classical Higher-order Logic -- only ``Main'', excluding real and - complex numbers etc. -\ - -no_notation - bot ("\") and - top ("\") and - inf (infixl "\" 70) and - sup (infixl "\" 65) and - Inf ("\_" [900] 900) and - Sup ("\_" [900] 900) and - ordLeq2 (infix "<=o" 50) and - ordLeq3 (infix "\o" 50) and - ordLess2 (infix "(_,/ _)\") - -hide_const (open) - czero cinfinite cfinite csum cone ctwo Csum cprod cexp image2 image2p vimage2p Gr Grp collect - fsts snds setl setr convol pick_middlep fstOp sndOp csquare relImage relInvImage Succ Shift - shift proj id_bnf - -hide_fact (open) id_bnf_def type_definition_id_bnf_UNIV - -no_syntax - "_INF1" :: "pttrns \ 'b \ 'b" ("(3\_./ _)" [0, 10] 10) - "_INF" :: "pttrn \ 'a set \ 'b \ 'b" ("(3\_\_./ _)" [0, 0, 10] 10) - "_SUP1" :: "pttrns \ 'b \ 'b" ("(3\_./ _)" [0, 10] 10) - "_SUP" :: "pttrn \ 'a set \ 'b \ 'b" ("(3\_\_./ _)" [0, 0, 10] 10) - -end