doc-src/TutorialI/Overview/Isar.thy
changeset 12815 1f073030b97a
parent 11238 1d789889c922
child 13249 4b3de6370184
--- a/doc-src/TutorialI/Overview/Isar.thy	Fri Jan 18 17:46:17 2002 +0100
+++ b/doc-src/TutorialI/Overview/Isar.thy	Fri Jan 18 18:30:19 2002 +0100
@@ -9,7 +9,7 @@
       (is "lfp ?F = ?toA")
 proof
   show "lfp ?F \<subseteq> ?toA"
-  by (blast intro!: lfp_lowerbound intro:rtrancl_trans)
+  by (blast intro!: lfp_lowerbound intro: rtrancl_trans)
 
   show "?toA \<subseteq> lfp ?F"
   proof