Paper/Paper.thy
author Christian Urban <urbanc@in.tum.de>
Wed, 17 Mar 2010 15:13:03 +0100
changeset 1483 2ca8e43b53c5
parent 1473 b4216d0e109a
child 1484 dc7b049d9072
permissions -rw-r--r--
added partial proof for the strong induction principle

(*<*)
theory Paper
imports "../Nominal/Test"
begin
(*>*)

section {* Introduction *}

text {*
  Here can come any text.

*}

(*<*)
end
(*>*)