src/HOL/Bali/WellType.thy
changeset 13384 a34e38154413
parent 13337 f75dfc606ac7
child 13462 56610e2ba220
--- a/src/HOL/Bali/WellType.thy	Tue Jul 16 18:52:26 2002 +0200
+++ b/src/HOL/Bali/WellType.thy	Tue Jul 16 20:25:21 2002 +0200
@@ -216,6 +216,8 @@
 "binop_type Xor      = Boolean"
 "binop_type BitOr    = Integer"
 "binop_type Or       = Boolean"
+"binop_type CondAnd  = Boolean"
+"binop_type CondOr   = Boolean"
 
 consts wt_binop :: "prog \<Rightarrow> binop \<Rightarrow> ty \<Rightarrow> ty \<Rightarrow> bool"
 primrec
@@ -239,8 +241,10 @@
 "wt_binop G Xor     t1 t2 = ((t1 = PrimT Boolean) \<and> (t2 = PrimT Boolean))"
 "wt_binop G BitOr   t1 t2 = ((t1 = PrimT Integer) \<and> (t2 = PrimT Integer))"
 "wt_binop G Or      t1 t2 = ((t1 = PrimT Boolean) \<and> (t2 = PrimT Boolean))"
+"wt_binop G CondAnd t1 t2 = ((t1 = PrimT Boolean) \<and> (t2 = PrimT Boolean))"
+"wt_binop G CondOr  t1 t2 = ((t1 = PrimT Boolean) \<and> (t2 = PrimT Boolean))"
 
-      
+
 types tys  =        "ty + ty list"
 translations
   "tys"   <= (type) "ty + ty list"