src/HOL/Computational_Algebra/Computation_Checks.thy
changeset 83358 1cf4f1e930af
parent 83357 d7c525fd68b2
child 83359 518a1464f1ac
--- 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 \<open>Computation checks\<close>
 
 theory Computation_Checks
-imports Primes Polynomial_Factorial
+imports Primes Polynomial_Factorial "HOL-Library.Discrete_Functions" "HOL-Library.Code_Target_Numeral"
 begin
 
 text \<open>
-  @{lemma \<open>prime (997::nat)\<close> by eval}
+  @{lemma \<open>floor_sqrt 16476148165462159 = 128359449\<close> by eval}
 \<close>
 
 text \<open>
-  @{lemma \<open>prime (997::int)\<close> by eval}
+  @{lemma \<open>prime (997 :: nat)\<close> by eval}
+\<close>
+
+text \<open>
+  @{lemma \<open>prime (997 :: int)\<close> by eval}
 \<close>
 
 text \<open>