src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy
changeset 67226 ec32cdaab97b
parent 66453 cc19f7ca2ed6
child 67399 eab6ce8368fa
--- a/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy	Tue Dec 19 14:51:27 2017 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy	Tue Dec 19 13:58:12 2017 +0100
@@ -125,7 +125,7 @@
 
 code_pred predicate_where_argument_is_neg_condition_and_in_equation .
 
-text {* Another related example that required slight adjustment of the proof procedure *}
+text \<open>Another related example that required slight adjustment of the proof procedure\<close>
 
 inductive if_as_predicate :: "bool \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"
 where