src/HOL/Number_Theory/Number_Theory.thy
author blanchet
Thu, 13 Mar 2014 13:18:13 +0100
changeset 56088 db61a0a62b2c
parent 51173 3cbb4e95a565
child 58889 5b7a9633cfa8
permissions -rw-r--r--
reintroduced old model reconstruction code -- still needs to be ported


header {* Comprehensive number theory *}

theory Number_Theory
imports Fib Residues Eratosthenes
begin

end