src/CTT/ex/Typechecking.thy
changeset 60770 240563fbf41d
parent 59498 50b60f501b05
child 61337 4645502c3c64
--- a/src/CTT/ex/Typechecking.thy	Thu Jul 23 14:20:51 2015 +0200
+++ b/src/CTT/ex/Typechecking.thy	Thu Jul 23 14:25:05 2015 +0200
@@ -9,7 +9,7 @@
 imports "../CTT"
 begin
 
-subsection {* Single-step proofs: verifying that a type is well-formed *}
+subsection \<open>Single-step proofs: verifying that a type is well-formed\<close>
 
 schematic_lemma "?A type"
 apply (rule form_rls)
@@ -31,7 +31,7 @@
 done
 
 
-subsection {* Multi-step proofs: Type inference *}
+subsection \<open>Multi-step proofs: Type inference\<close>
 
 lemma "PROD w:N. N + N type"
 apply form
@@ -67,7 +67,7 @@
 (*Proofs involving arbitrary types.
   For concreteness, every type variable left over is forced to be N*)
 method_setup N =
-  {* Scan.succeed (fn ctxt => SIMPLE_METHOD (TRYALL (resolve_tac ctxt @{thms NF}))) *}
+  \<open>Scan.succeed (fn ctxt => SIMPLE_METHOD (TRYALL (resolve_tac ctxt @{thms NF})))\<close>
 
 schematic_lemma "lam w. <w,w> : ?A"
 apply typechk