diff -r d7c525fd68b2 -r 1cf4f1e930af src/HOL/Computational_Algebra/Computation_Checks.thy --- a/src/HOL/Computational_Algebra/Computation_Checks.thy Sun Nov 02 19:47:30 2025 +0100 +++ b/src/HOL/Computational_Algebra/Computation_Checks.thy Sun Nov 02 19:47:30 2025 +0100 @@ -5,15 +5,19 @@ section \Computation checks\ theory Computation_Checks -imports Primes Polynomial_Factorial +imports Primes Polynomial_Factorial "HOL-Library.Discrete_Functions" "HOL-Library.Code_Target_Numeral" begin text \ - @{lemma \prime (997::nat)\ by eval} + @{lemma \floor_sqrt 16476148165462159 = 128359449\ by eval} \ text \ - @{lemma \prime (997::int)\ by eval} + @{lemma \prime (997 :: nat)\ by eval} +\ + +text \ + @{lemma \prime (997 :: int)\ by eval} \ text \