Paper/Paper.thy
author Cezary Kaliszyk <kaliszyk@in.tum.de>
Wed, 10 Feb 2010 10:36:47 +0100
changeset 1111 ee276c9f12f0
parent 754 b85875d65b10
child 1473 b4216d0e109a
permissions -rw-r--r--
A concrete example, with a proof that rbv is not regular and with proofs of induction and pseudo-injectivity that require this

(*<*)
theory Paper
imports "../Quot/QuotMain"
begin
(*>*)

section {* Introduction *}

text {*
  Here can come any text.

*}

(*<*)
end
(*>*)