src/HOL/IMP/Poly_Types.thy
changeset 45200 1f1897ac7877
parent 45015 fdac1e9880eb
child 45212 e87feee00a4c
--- a/src/HOL/IMP/Poly_Types.thy	Wed Oct 19 09:11:21 2011 +0200
+++ b/src/HOL/IMP/Poly_Types.thy	Wed Oct 19 16:32:12 2011 +0200
@@ -18,7 +18,7 @@
 
 inductive btyping :: "tyenv \<Rightarrow> bexp \<Rightarrow> bool" (infix "\<turnstile>p" 50)
 where
-"\<Gamma> \<turnstile>p B bv" |
+"\<Gamma> \<turnstile>p Bc v" |
 "\<Gamma> \<turnstile>p b \<Longrightarrow> \<Gamma> \<turnstile>p Not b" |
 "\<Gamma> \<turnstile>p b1 \<Longrightarrow> \<Gamma> \<turnstile>p b2 \<Longrightarrow> \<Gamma> \<turnstile>p And b1 b2" |
 "\<Gamma> \<turnstile>p a1 : \<tau> \<Longrightarrow> \<Gamma> \<turnstile>p a2 : \<tau> \<Longrightarrow> \<Gamma> \<turnstile>p Less a1 a2"