diff -r 1c5dcba6925f -r f143d0a4cb6a src/HOL/ex/Sqrt_Script.thy --- a/src/HOL/ex/Sqrt_Script.thy Sat Jun 05 12:45:00 2021 +0200 +++ b/src/HOL/ex/Sqrt_Script.thy Sat Jun 05 12:57:52 2021 +0200 @@ -5,14 +5,14 @@ section \Square roots of primes are irrational (script version)\ -theory Sqrt_Script -imports Complex_Main "HOL-Computational_Algebra.Primes" -begin +text \ + Contrast this linear Isabelle/Isar script with the more mathematical version + in \<^file>\~~/src/HOL/Examples/Sqrt.thy\ by Makarius Wenzel. +\ -text \ - \medskip Contrast this linear Isabelle/Isar script with Markus - Wenzel's more mathematical version. -\ +theory Sqrt_Script + imports Complex_Main "HOL-Computational_Algebra.Primes" +begin subsection \Preliminaries\