src/Doc/Implementation/Base.thy
author Manuel Eberl <eberlm@in.tum.de>
Wed, 07 Apr 2021 11:05:00 +0200
changeset 73537 56db8559eadb
parent 69605 a96320074298
permissions -rw-r--r--
fixed problematic addition operation in the 'approximation' package (previous version used much too high precision sometimes)

(*:maxLineLen=78:*)

theory Base
imports Main
begin

ML_file \<open>../antiquote_setup.ML\<close>

end