diff -r a705f42b244d -r 2332d9be352b src/CTT/ex/Typechecking.thy --- a/src/CTT/ex/Typechecking.thy Sat Oct 10 21:14:00 2015 +0200 +++ b/src/CTT/ex/Typechecking.thy Sat Oct 10 21:43:07 2015 +0200 @@ -22,7 +22,7 @@ apply (rule form_rls) done -schematic_goal "PROD z:?A . N + ?B(z) type" +schematic_goal "\z:?A . N + ?B(z) type" apply (rule form_rls) apply (rule form_rls) apply (rule form_rls) @@ -33,7 +33,7 @@ subsection \Multi-step proofs: Type inference\ -lemma "PROD w:N. N + N type" +lemma "\w:N. N + N type" apply form done @@ -41,26 +41,26 @@ apply intr done -schematic_goal "PROD w:N . Eq(?A,w,w) type" +schematic_goal "\w:N . Eq(?A,w,w) type" apply typechk done -schematic_goal "PROD x:N . PROD y:N . Eq(?A,x,y) type" +schematic_goal "\x:N . \y:N . Eq(?A,x,y) type" apply typechk done text "typechecking an application of fst" -schematic_goal "(lam u. split(u, \v w. v)) ` <0, succ(0)> : ?A" +schematic_goal "(\<^bold>\u. split(u, \v w. v)) ` <0, succ(0)> : ?A" apply typechk done text "typechecking the predecessor function" -schematic_goal "lam n. rec(n, 0, \x y. x) : ?A" +schematic_goal "\<^bold>\n. rec(n, 0, \x y. x) : ?A" apply typechk done text "typechecking the addition function" -schematic_goal "lam n. lam m. rec(n, m, \x y. succ(y)) : ?A" +schematic_goal "\<^bold>\n. \<^bold>\m. rec(n, m, \x y. succ(y)) : ?A" apply typechk done @@ -69,18 +69,18 @@ method_setup N = \Scan.succeed (fn ctxt => SIMPLE_METHOD (TRYALL (resolve_tac ctxt @{thms NF})))\ -schematic_goal "lam w. : ?A" +schematic_goal "\<^bold>\w. : ?A" apply typechk apply N done -schematic_goal "lam x. lam y. x : ?A" +schematic_goal "\<^bold>\x. \<^bold>\y. x : ?A" apply typechk apply N done text "typechecking fst (as a function object)" -schematic_goal "lam i. split(i, \j k. j) : ?A" +schematic_goal "\<^bold>\i. split(i, \j k. j) : ?A" apply typechk apply N done