src/HOL/Main.thy
changeset 70078 3a1b2d8c89aa
parent 69745 aec42cee2521
child 70336 559f45528804
--- a/src/HOL/Main.thy	Sun Apr 07 12:44:37 2019 +0200
+++ b/src/HOL/Main.thy	Sun Apr 07 08:26:57 2019 +0200
@@ -8,7 +8,7 @@
 theory Main
   imports
     Predicate_Compile
-    Quickcheck_Narrowing 
+    Quickcheck_Narrowing
     Extraction
     Nunchaku
     BNF_Greatest_Fixpoint
@@ -72,6 +72,23 @@
   BNF_Cardinal_Arithmetic.cexp (infixr "^c" 90) and
   BNF_Def.convol ("\<langle>(_,/ _)\<rangle>")
 
+bundle cardinal_syntax begin
+notation
+  ordLeq2 (infix "<=o" 50) and
+  ordLeq3 (infix "\<le>o" 50) and
+  ordLess2 (infix "<o" 50) and
+  ordIso2 (infix "=o" 50) and
+  card_of ("|_|") and
+  BNF_Cardinal_Arithmetic.csum (infixr "+c" 65) and
+  BNF_Cardinal_Arithmetic.cprod (infixr "*c" 80) and
+  BNF_Cardinal_Arithmetic.cexp (infixr "^c" 90)
+
+alias cinfinite = BNF_Cardinal_Arithmetic.cinfinite
+alias czero = BNF_Cardinal_Arithmetic.czero
+alias cone = BNF_Cardinal_Arithmetic.cone
+alias ctwo = BNF_Cardinal_Arithmetic.ctwo
+end
+
 no_syntax
   "_INF1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3\<Sqinter>_./ _)" [0, 10] 10)
   "_INF"      :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b"  ("(3\<Sqinter>_\<in>_./ _)" [0, 0, 10] 10)