src/HOL/Number_Theory/Number_Theory.thy
author blanchet
Tue, 24 Apr 2012 13:56:13 +0200
changeset 47728 6ee015f6ea4b
parent 32479 521cc9bf2958
child 51173 3cbb4e95a565
permissions -rw-r--r--
reintroduce file offsets in Mirabelle output, but make sure they are not influenced by the length of the path


header {* Comprehensive number theory *}

theory Number_Theory
imports Fib Residues
begin

end