src/HOL/Computational_Algebra/Computation_Checks.thy
changeset 83357 d7c525fd68b2
child 83358 1cf4f1e930af
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Computational_Algebra/Computation_Checks.thy	Sun Nov 02 19:47:30 2025 +0100
@@ -0,0 +1,28 @@
+(*  Title:      HOL/Computational_Algebra/Computation_Checks.thy
+    Author:     Florian Haftmann, TU Muenchen
+*)
+
+section \<open>Computation checks\<close>
+
+theory Computation_Checks
+imports Primes Polynomial_Factorial
+begin
+
+text \<open>
+  @{lemma \<open>prime (997::nat)\<close> by eval}
+\<close>
+
+text \<open>
+  @{lemma \<open>prime (997::int)\<close> by eval}
+\<close>
+
+text \<open>
+  @{lemma \<open>Gcd {[:1, 2, 3:], [:2, 3, (4 :: int):]} = 1\<close> by eval}
+\<close>
+
+text \<open>
+  @{lemma \<open>Lcm {[:1, 2, 3:], [:2, 3, 4:]} = [:[:2:], [:7:], [:16:], [:17:], [:12 :: int:]:]\<close> by eval}
+\<close>
+
+end
+