src/HOL/Isar_examples/MultisetOrder.thy
changeset 7968 964b65b4e433
parent 7874 180364256231
child 7982 d534b897ce39
--- a/src/HOL/Isar_examples/MultisetOrder.thy	Thu Oct 28 19:53:24 1999 +0200
+++ b/src/HOL/Isar_examples/MultisetOrder.thy	Thu Oct 28 19:57:34 1999 +0200
@@ -3,15 +3,17 @@
     Author:     Markus Wenzel
 
 Wellfoundedness proof for the multiset order.
-
-Original tactic script by Tobias Nipkow (see also
-HOL/Induct/Multiset).  Pen-and-paper proof by Wilfried Buchholz.
 *)
 
 header {* Wellfoundedness of multiset ordering *};
 
 theory MultisetOrder = Multiset:;
 
+text_raw {*
+ \footnote{Original tactic script by Tobias Nipkow (see also
+ \url{http://isabelle.in.tum.de/library/HOL/Induct/Multiset.html}),
+ based on a pen-and-paper proof due to Wilfried Buchholz.}
+*};
 
 subsection {* A technical lemma *};