src/HOL/Wellfounded.thy
changeset 61799 4cf66f21b764
parent 61424 c3658c18b7bc
child 61943 7fba644ed827
--- a/src/HOL/Wellfounded.thy	Mon Dec 07 10:23:50 2015 +0100
+++ b/src/HOL/Wellfounded.thy	Mon Dec 07 10:38:04 2015 +0100
@@ -233,7 +233,7 @@
 apply (rule_tac x = "{z. z:Q & (z,y) : r^*}" in allE)
  apply assumption
 apply (erule_tac V = "ALL Q. (EX x. x : Q) --> P Q" for P in thin_rl) 
-  --\<open>essential for speed\<close>
+  \<comment>\<open>essential for speed\<close>
 txt\<open>Blast with new substOccur fails\<close>
 apply (fast intro: converse_rtrancl_into_rtrancl)
 done
@@ -375,7 +375,7 @@
   qed
 qed
 
-lemma wf_comp_self: "wf R = wf (R O R)"  -- \<open>special case\<close>
+lemma wf_comp_self: "wf R = wf (R O R)"  \<comment> \<open>special case\<close>
   by (rule wf_union_merge [where S = "{}", simplified])
 
 
@@ -384,7 +384,7 @@
 text \<open>Bachmair and Dershowitz 1986, Lemma 2. [Provided by Tjark Weber]\<close>
 
 lemma qc_wf_relto_iff:
-  assumes "R O S \<subseteq> (R \<union> S)\<^sup>* O R" -- \<open>R quasi-commutes over S\<close>
+  assumes "R O S \<subseteq> (R \<union> S)\<^sup>* O R" \<comment> \<open>R quasi-commutes over S\<close>
   shows "wf (S\<^sup>* O R O S\<^sup>*) \<longleftrightarrow> wf R" (is "wf ?S \<longleftrightarrow> _")
 proof
   assume "wf ?S"