CookBook/FirstSteps.thy
changeset 138 e4d8dfb7e34a
parent 136 58277de8493c
child 149 253ea99c1441
--- a/CookBook/FirstSteps.thy	Tue Feb 24 22:23:07 2009 +0000
+++ b/CookBook/FirstSteps.thy	Wed Feb 25 10:09:18 2009 +0000
@@ -842,14 +842,13 @@
 
 @{ML_response_fake [display,gray]
 "let
-  val thy = @{theory}
 
-  val assm1 = cterm_of thy @{prop \"\<And>(x::nat). P x \<Longrightarrow> Q x\"}
-  val assm2 = cterm_of thy @{prop \"(P::nat\<Rightarrow>bool) t\"}
+  val assm1 = @{cprop \"\<And>(x::nat). P x \<Longrightarrow> Q x\"}
+  val assm2 = @{cprop \"(P::nat\<Rightarrow>bool) t\"}
 
   val Pt_implies_Qt = 
         assume assm1
-        |> forall_elim (cterm_of thy @{term \"t::nat\"});
+        |> forall_elim @{cterm \"t::nat\"};
   
   val Qt = implies_elim Pt_implies_Qt (assume assm2);
 in