doc-src/IsarImplementation/Thy/Base.thy
author haftmann
Mon, 20 Apr 2009 09:32:40 +0200
changeset 30954 cf50e67bc1d1
parent 30272 2d612824e642
child 39846 cb6634eb8926
permissions -rw-r--r--
power operation on functions in theory Nat; power operation on relations in theory Transitive_Closure

theory Base
imports Pure
uses "../../antiquote_setup.ML"
begin

end