Tutorial/Tutorial5.thy
changeset 2698 96f3ac5d11ad
parent 2691 abb6c3ac2df2
child 2701 7b2691911fbc
equal deleted inserted replaced
2697:b9e2a66a317c 2698:96f3ac5d11ad
   130 theorem progress:
   130 theorem progress:
   131   assumes a: "[] \<turnstile> t : T"
   131   assumes a: "[] \<turnstile> t : T"
   132   shows "(\<exists>t'. t \<longrightarrow>cbv t') \<or> (val t)"
   132   shows "(\<exists>t'. t \<longrightarrow>cbv t') \<or> (val t)"
   133 using a
   133 using a
   134 by (induct \<Gamma>\<equiv>"[]::ty_ctx" t T)
   134 by (induct \<Gamma>\<equiv>"[]::ty_ctx" t T)
   135    (auto elim: canonical_tArr)
   135    (auto elim: canonical_tArr simp add: val.simps)
   136 
   136 
   137 text {*
   137 text {*
   138   Done! Congratulations!
   138   Done! Congratulations!
   139 *}
   139 *}
   140 
   140