doc-src/IsarImplementation/Thy/base.thy
author webertj
Wed, 26 Jul 2006 19:23:04 +0200
changeset 20217 25b068a99d2b
parent 18537 2681f9e34390
child 21374 27ae6bc4102a
permissions -rw-r--r--
linear arithmetic splits certain operators (e.g. min, max, abs)


(* $Id$ *)

theory base
imports CPure
uses "setup.ML"
begin

end