src/HOL/Number_Theory/Number_Theory.thy
author traytel
Mon, 10 Nov 2014 10:29:19 +0100
changeset 58961 7c507e664047
parent 58889 5b7a9633cfa8
child 60526 fad653acf58f
permissions -rw-r--r--
dropped redundant transfer rules (now proved and registered by datatype and plugins)


section {* Comprehensive number theory *}

theory Number_Theory
imports Fib Residues Eratosthenes
begin

end