src/HOL/ex/Antiquote.thy
changeset 61933 cf58b5b794b2
parent 59031 4c3bb56b8ce7
child 69597 ff784d5a5bfb
--- a/src/HOL/ex/Antiquote.thy	Sat Dec 26 15:44:14 2015 +0100
+++ b/src/HOL/ex/Antiquote.thy	Sat Dec 26 15:59:27 2015 +0100
@@ -31,9 +31,9 @@
 term "EXPR (a + b + c + VAR x + VAR y + 1)"
 term "EXPR (VAR (f w) + VAR x)"
 
-term "Expr (\<lambda>env. env x)"    -- \<open>improper\<close>
+term "Expr (\<lambda>env. env x)"    \<comment> \<open>improper\<close>
 term "Expr (\<lambda>env. f env)"
-term "Expr (\<lambda>env. f env + env x)"    -- \<open>improper\<close>
+term "Expr (\<lambda>env. f env + env x)"    \<comment> \<open>improper\<close>
 term "Expr (\<lambda>env. f env y z)"
 term "Expr (\<lambda>env. f env + g y env)"
 term "Expr (\<lambda>env. f env + g env y + h a env z)"