src/FOL/ex/Locale_Test/Locale_Test1.thy
changeset 61487 f8cb97e0fd0b
parent 61268 abe08fb15a12
child 61489 b8d375aee0df
equal deleted inserted replaced
61486:3590367b0ce9 61487:f8cb97e0fd0b
   160 \<close>
   160 \<close>
   161 
   161 
   162 declare [[show_hyps]]
   162 declare [[show_hyps]]
   163 
   163 
   164 ML \<open>
   164 ML \<open>
   165   check_syntax @{context} @{thm d1_def} "d1(?x) <-> ~ p2(p1(?x))";
   165   check_syntax @{context} @{thm d1_def} "d1(?x) \<longleftrightarrow> \<not> p2(p1(?x))";
   166   check_syntax @{context} @{thm d2_def} "d2(?x) <-> ~ p2(?x)";
   166   check_syntax @{context} @{thm d2_def} "d2(?x) \<longleftrightarrow> \<not> p2(?x)";
   167 \<close>
   167 \<close>
   168 
   168 
   169 end
   169 end
   170 
   170 
   171 locale syntax'' = "syntax" p3 p2 for p3 :: "'a => 'b" and p2 :: "'b => o"
   171 locale syntax'' = "syntax" p3 p2 for p3 :: "'a => 'b" and p2 :: "'b => o"
   173 
   173 
   174 thm d1_def d2_def
   174 thm d1_def d2_def
   175   (* should print as "syntax.d1(p3, p2, ?x) <-> ..." and "d2(?x) <-> ..." *)
   175   (* should print as "syntax.d1(p3, p2, ?x) <-> ..." and "d2(?x) <-> ..." *)
   176 
   176 
   177 ML \<open>
   177 ML \<open>
   178   check_syntax @{context} @{thm d1_def} "syntax.d1(p3, p2, ?x) <-> ~ p2(p3(?x))";
   178   check_syntax @{context} @{thm d1_def} "syntax.d1(p3, p2, ?x) \<longleftrightarrow> \<not> p2(p3(?x))";
   179   check_syntax @{context} @{thm d2_def} "d2(?x) <-> ~ p2(?x)";
   179   check_syntax @{context} @{thm d2_def} "d2(?x) \<longleftrightarrow> \<not> p2(?x)";
   180 \<close>
   180 \<close>
   181 
   181 
   182 end
   182 end
   183 
   183 
   184 
   184