src/HOL/ex/Lagrange.thy
changeset 58889 5b7a9633cfa8
parent 58776 95e58e04e534
child 61343 5b5656a63bd6
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (*  Title:      HOL/ex/Lagrange.thy
     1 (*  Title:      HOL/ex/Lagrange.thy
     2     Author:     Tobias Nipkow
     2     Author:     Tobias Nipkow
     3     Copyright   1996 TU Muenchen
     3     Copyright   1996 TU Muenchen
     4 *)
     4 *)
     5 
     5 
     6 header {* A lemma for Lagrange's theorem *}
     6 section {* A lemma for Lagrange's theorem *}
     7 
     7 
     8 theory Lagrange imports Main begin
     8 theory Lagrange imports Main begin
     9 
     9 
    10 text {* This theory only contains a single theorem, which is a lemma
    10 text {* This theory only contains a single theorem, which is a lemma
    11 in Lagrange's proof that every natural number is the sum of 4 squares.
    11 in Lagrange's proof that every natural number is the sum of 4 squares.