src/HOL/Number_Theory/Number_Theory.thy
author kuncar
Tue, 25 Feb 2014 19:07:14 +0100
changeset 55736 f1ed1e9cd080
parent 51173 3cbb4e95a565
child 58889 5b7a9633cfa8
permissions -rw-r--r--
unregister lifting setup following the best practice of Lifting


header {* Comprehensive number theory *}

theory Number_Theory
imports Fib Residues Eratosthenes
begin

end