src/HOL/ex/Sqrt_Script.thy
changeset 58889 5b7a9633cfa8
parent 57514 bdc2c6b40bf2
child 61343 5b5656a63bd6
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (*  Title:      HOL/ex/Sqrt_Script.thy
     1 (*  Title:      HOL/ex/Sqrt_Script.thy
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     3     Copyright   2001  University of Cambridge
     3     Copyright   2001  University of Cambridge
     4 *)
     4 *)
     5 
     5 
     6 header {* Square roots of primes are irrational (script version) *}
     6 section {* Square roots of primes are irrational (script version) *}
     7 
     7 
     8 theory Sqrt_Script
     8 theory Sqrt_Script
     9 imports Complex_Main "~~/src/HOL/Number_Theory/Primes"
     9 imports Complex_Main "~~/src/HOL/Number_Theory/Primes"
    10 begin
    10 begin
    11 
    11